Skip to content

Commit

Permalink
feat(category_theory): equivalences preserve epis and monos (#6994)
Browse files Browse the repository at this point in the history
Note that these don't follow from the results in `limits/constructions/epi_mono.lean`, since the results in that file are less universe polymorphic.
  • Loading branch information
TwoFX committed Apr 6, 2021
1 parent 89ea423 commit fe16235
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/category_theory/epi_mono.lean
Expand Up @@ -40,6 +40,14 @@ begin
cancel_mono, equiv.apply_eq_iff_eq] at H
end

instance is_equivalence.epi_map {F : C ⥤ D} [is_left_adjoint F] {X Y : C} {f : X ⟶ Y}
[h : epi f] : epi (F.map f) :=
left_adjoint_preserves_epi (adjunction.of_left_adjoint F) h

instance is_equivalence.mono_map {F : C ⥤ D} [is_right_adjoint F] {X Y : C} {f : X ⟶ Y}
[h : mono f] : mono (F.map f) :=
right_adjoint_preserves_mono (adjunction.of_right_adjoint F) h

lemma faithful_reflects_epi (F : C ⥤ D) [faithful F] {X Y : C} {f : X ⟶ Y}
(hf : epi (F.map f)) : epi f :=
⟨λ Z g h H, F.map_injective $
Expand Down

0 comments on commit fe16235

Please sign in to comment.