- preimage : Π {X Y : C}, (F.obj X ⟶ F.obj Y) → (X ⟶ Y)
- witness' : (∀ {X Y : C} (f : F.obj X ⟶ F.obj Y), F.map (category_theory.full.preimage f) = f) . "obviously"
A functor F : C ⥤ D
is full if for each X Y : C
, F.map
is surjective.
In fact, we use a constructive definition, so the full F
typeclass contains data,
specifying a particular preimage of each f : F.obj X ⟶ F.obj Y
.
Instances
- category_theory.equivalence.full_of_equivalence
- category_theory.reflective.to_full
- category_theory.full.id
- category_theory.full.comp
- category_theory.ulift_functor_full
- category_theory.functor.category_theory.full
- category_theory.induced_category.full
- category_theory.full_subcategory.full
- category_theory.bundled_hom.forget₂_full
- CommRing.category_theory.full
- category_theory.yoneda.yoneda_full
- category_theory.coyoneda.coyoneda_full
- category_theory.limits.cones.functoriality_full
- category_theory.limits.cocones.functoriality_full
- category_theory.forget₂.category_theory.full
- Mon.to_Cat_full
- category_theory.Groupoid.forget_to_Cat_full
- category_theory.reflective.comparison_full
- Top.sheaf.forget.full
- map_injective' : (∀ {X Y : C}, function.injective F.map) . "obviously"
A functor F : C ⥤ D
is faithful if for each X Y : C
, F.map
is injective.
Instances
- category_theory.equivalence.faithful_of_equivalence
- category_theory.reflective.to_faithful
- category_theory.faithful.id
- category_theory.faithful.comp
- category_theory.ulift_functor_faithful
- category_theory.functor.category_theory.faithful
- category_theory.functor.right_op_faithful
- category_theory.functor.left_op_faithful
- category_theory.induced_category.faithful
- category_theory.full_subcategory.faithful
- category_theory.concrete_category.forget_faithful
- category_theory.forget_faithful
- category_theory.yoneda.yoneda_faithful
- category_theory.coyoneda.coyoneda_faithful
- category_theory.limits.cones.functoriality_faithful
- category_theory.limits.cocones.functoriality_faithful
- category_theory.monoidal_category.category_theory.faithful
- category_theory.graded_object.category_theory.faithful
- category_theory.differential_object.forget_faithful
- Mon.to_Cat_faithful
- category_theory.Groupoid.forget_to_Cat_faithful
- category_theory.reflective.comparison_faithful
- Top.sheaf.forget.faithful
The specified preimage of a morphism under a full functor.
Equations
If F : C ⥤ D
is fully faithful, every isomorphism F.obj X ≅ F.obj Y
has a preimage.
Equations
- category_theory.preimage_iso f = {hom := F.preimage f.hom, inv := F.preimage f.inv, hom_inv_id' := _, inv_hom_id' := _}
If the image of a morphism under a fully faithful functor in an isomorphism, then the original morphisms is also an isomorphism.
Equations
- category_theory.is_iso_of_fully_faithful F f = {inv := F.preimage (category_theory.is_iso.inv (F.map f)), hom_inv_id' := _, inv_hom_id' := _}
If F
is fully faithful, we have an equivalence of hom-sets X ⟶ Y
and F X ⟶ F Y
.
Equations
Equations
- _ = _
“Divide” a functor by a faithful functor.
Given a natural isomorphism between F ⋙ H
and G ⋙ H
for a fully faithful functor H
, we
can 'cancel' it to give a natural iso between F
and G
.
Equations
- category_theory.fully_faithful_cancel_right H comp_iso = category_theory.nat_iso.of_components (λ (X : C), category_theory.preimage_iso (comp_iso.app X)) _