Preservation and reflection of monomorphisms and epimorphisms #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We provide typeclasses that state that a functor preserves or reflects monomorphisms or epimorphisms.
- preserves : ∀ {X Y : C} (f : X ⟶ Y) [_inst_4 : category_theory.mono f], category_theory.mono (F.map f)
A functor preserves monomorphisms if it maps monomorphisms to monomorphisms.
Instances of this typeclass
- category_theory.functor.preserves_monomorphisms_of_is_right_adjoint
- category_theory.preserves_monomorphisms_of_preserves_limits_of_shape
- category_theory.functor.preserves_monomorphisms_comp
- category_theory.forget₂_preserves_monomorphisms
- Module.forget_preserves_monomorphisms
- Group.forget_Group_preserves_mono
- AddGroup.forget_Group_preserves_mono
- CommGroup.forget_CommGroup_preserves_mono
- AddCommGroup.forget_CommGroup_preserves_mono
- Top.presheaf.stalk_functor_preserves_mono
- preserves : ∀ {X Y : C} (f : X ⟶ Y) [_inst_4 : category_theory.epi f], category_theory.epi (F.map f)
A functor preserves epimorphisms if it maps epimorphisms to epimorphisms.
Instances of this typeclass
- category_theory.functor.preserves_epimorphisms_of_is_left_adjoint
- category_theory.preserves_epimorphisms_of_preserves_colimits_of_shape
- category_theory.functor.preserves_epimorphisms_comp
- category_theory.forget₂_preserves_epimorphisms
- Module.forget_preserves_epimorphisms
- Group.forget_Group_preserves_epi
- AddGroup.forget_Group_preserves_epi
- CommGroup.forget_CommGroup_preserves_epi
- AddCommGroup.forget_CommGroup_preserves_epi
- reflects : ∀ {X Y : C} (f : X ⟶ Y), category_theory.mono (F.map f) → category_theory.mono f
A functor reflects monomorphisms if morphisms that are mapped to monomorphisms are themselves monomorphisms.
- reflects : ∀ {X Y : C} (f : X ⟶ Y), category_theory.epi (F.map f) → category_theory.epi f
A functor reflects epimorphisms if morphisms that are mapped to epimorphisms are themselves epimorphisms.
If F
is a fully faithful functor, split epimorphisms are preserved and reflected by F
.
If F
is a fully faithful functor, split monomorphisms are preserved and reflected by F
.
Equations
- F.split_mono_equiv f = {to_fun := λ (f_1 : category_theory.split_mono f), f_1.map F, inv_fun := λ (s : category_theory.split_mono (F.map f)), {retraction := F.preimage s.retraction, id' := _}, left_inv := _, right_inv := _}
If F : C ⥤ D
is an equivalence of categories and C
is a split_epi_category
,
then D
also is.