Skip to content

Commit

Permalink
feat(category_theory/equivalence): injectivity simp lemmas for equiva…
Browse files Browse the repository at this point in the history
…lences (#3437)






Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Jul 19, 2020
1 parent eb68f4c commit eca55c9
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/category_theory/equivalence.lean
Expand Up @@ -388,6 +388,20 @@ is_equivalence.mk (equivalence_inverse F)
(λ Y, F.fun_obj_preimage_iso Y)
(by obviously))

@[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 :=
begin
split,
{ intro w, apply e.functor.map_injective, exact w, },
{ rintro ⟨rfl⟩, refl, }
end

@[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 :=
begin
split,
{ intro w, apply e.inverse.map_injective, exact w, },
{ rintro ⟨rfl⟩, refl, }
end

end equivalence

end category_theory

0 comments on commit eca55c9

Please sign in to comment.