IsRepresentedBy predicate #
In this file we define the predicate IsRepresentedBy: A presheaf F is represented by X
with universal element x : F.obj X if the natural transformation yoneda.obj X ⟶ F induced
by x is an isomorphism.
For other declarations expressing a functor is representable, see also:
CategoryTheory.Functor.RepresentableBy: Structure bundling an explicit natural isomorphismyoneda.obj X ⟶ F.CategoryTheory.Functor.IsRepresentable: Predicate asserting the existence of a representing object.
The relations to these other notions are given as
CategoryTheory.Functor.IsRepresentable.iff_exists_isRepresentedBy and
CategoryTheory.Functor.IsRepresentedBy.iff_exists_representableBy.
TODOs #
- Dualize to
IsCorepresentedBy.
A presheaf F is represented by X with universal element x : F.obj X
if the natural transformation yoneda.obj X ⟶ F induced by x is an isomorphism.
For better universe generality, we state this manually as for every Y, the
induced map (Y ⟶ X) → F.obj Y is bijective.
- map_bijective {Y : C} : Function.Bijective fun (f : Y ⟶ X) => F.map f.op x
Instances For
If F is represented by X with universal element x : F.obj X, modulo universe
lifting, it is isomorphic to yoneda.obj X.
Equations
- h.uliftYonedaIso = CategoryTheory.asIso (CategoryTheory.uliftYonedaEquiv.symm { down := x })
Instances For
The canonical representation induced by the universal element x : F.obj X.
Equations
- One or more equations did not get rendered due to their size.