Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit e6ff367

Browse files
kim-emVierkantor
andcommitted
feat(logic/embedding): simp lemma for injectivity for embeddings (#7881)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com> Co-authored-by: Vierkantor <vierkantor@vierkantor.com>
1 parent 728eefe commit e6ff367

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/logic/embedding.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -66,6 +66,9 @@ by { ext, simp }
6666

6767
theorem injective {α β} (f : α ↪ β) : injective f := f.inj'
6868

69+
@[simp] lemma apply_eq_iff_eq {α β : Type*} (f : α ↪ β) (x y : α) : f x = f y ↔ x = y :=
70+
f.injective.eq_iff
71+
6972
@[refl, simps {simp_rhs := tt}]
7073
protected def refl (α : Sort*) : α ↪ α :=
7174
⟨id, injective_id⟩

0 commit comments

Comments
 (0)