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

Commit eca55c9

Browse files
committed
feat(category_theory/equivalence): injectivity simp lemmas for equivalences (#3437)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent eb68f4c commit eca55c9

File tree

1 file changed

+14
-0
lines changed

1 file changed

+14
-0
lines changed

src/category_theory/equivalence.lean

Lines changed: 14 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -388,6 +388,20 @@ is_equivalence.mk (equivalence_inverse F)
388388
(λ Y, F.fun_obj_preimage_iso Y)
389389
(by obviously))
390390

391+
@[simp] lemma functor_map_inj_iff (e : C ≌ D) {X Y : C} (f g : X ⟶ Y) : e.functor.map f = e.functor.map g ↔ f = g :=
392+
begin
393+
split,
394+
{ intro w, apply e.functor.map_injective, exact w, },
395+
{ rintro ⟨rfl⟩, refl, }
396+
end
397+
398+
@[simp] lemma inverse_map_inj_iff (e : C ≌ D) {X Y : D} (f g : X ⟶ Y) : e.inverse.map f = e.inverse.map g ↔ f = g :=
399+
begin
400+
split,
401+
{ intro w, apply e.inverse.map_injective, exact w, },
402+
{ rintro ⟨rfl⟩, refl, }
403+
end
404+
391405
end equivalence
392406

393407
end category_theory

0 commit comments

Comments
 (0)