Skip to content

Commit

Permalink
feat(data/quot): quotient.out is injective (#13584)
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Apr 22, 2022
1 parent 821e7c8 commit 40fc58c
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion src/data/quot.lean
Expand Up @@ -255,9 +255,12 @@ end
x.out ≈ y.out ↔ x = y :=
by rw [← quotient.eq_mk_iff_out, quotient.out_eq]

lemma quotient.out_injective {s : setoid α} : function.injective (@quotient.out α s) :=
λ a b h, quotient.out_equiv_out.1 $ h ▸ setoid.refl _

@[simp] lemma quotient.out_inj {s : setoid α} {x y : quotient s} :
x.out = y.out ↔ x = y :=
⟨λ h, quotient.out_equiv_out.1 $ h ▸ setoid.refl _, λ h, h ▸ rfl⟩
⟨λ h, quotient.out_injective h, λ h, h ▸ rfl⟩

section pi

Expand Down

0 comments on commit 40fc58c

Please sign in to comment.