Skip to content

Commit

Permalink
feat(data/subtype): subtype.coe_ext
Browse files Browse the repository at this point in the history
  • Loading branch information
digama0 committed Sep 20, 2018
1 parent 9815239 commit 1758092
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions data/subtype.lean
Expand Up @@ -13,6 +13,9 @@ protected lemma subtype.eq' : ∀ {a1 a2 : {x // β x}}, a1.val = a2.val → a1
lemma subtype.ext {a1 a2 : {x // β x}} : a1 = a2 ↔ a1.val = a2.val :=
⟨congr_arg _, subtype.eq'⟩

lemma subtype.coe_ext {a1 a2 : {x // β x}} : a1 = a2 ↔ (a1 : α) = a2 :=
subtype.ext

theorem subtype.val_injective : function.injective (@subtype.val _ β) :=
λ a b, subtype.eq'

Expand Down

0 comments on commit 1758092

Please sign in to comment.