Skip to content

Commit

Permalink
coercion
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 19, 2024
1 parent b486c67 commit 5ef7407
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/Init/Coe.lean
Original file line number Diff line number Diff line change
Expand Up @@ -313,6 +313,12 @@ instance optionCoe {α : Type u} : Coe α (Option α) where
instance subtypeCoe {α : Sort u} {p : α → Prop} : CoeOut (Subtype p) α where
coe v := v.val

instance boolPredToPred : Coe (α → Bool) (α → Prop) where
coe r := fun a => Eq (r a) true

instance boolRelToRel : Coe (α → α → Bool) (α → α → Prop) where
coe r := fun a b => Eq (r a b) true

/-! # Coe bridge -/

/--
Expand Down

0 comments on commit 5ef7407

Please sign in to comment.