Documentation

Mathlib.CategoryTheory.Limits.Yoneda

Limit properties relating to the (co)yoneda embedding. #

We calculate the colimit of Y ↦ (X ⟶ Y), which is just PUnit. (This is used in characterising cofinal functors.)

We also show the (co)yoneda embeddings preserve limits and jointly reflect them.

The colimit cocone over coyoneda.obj X, with cocone point PUnit.

Equations
Instances For
    @[simp]
    theorem CategoryTheory.Coyoneda.colimitCocone_ι_app {C : Type u} [Category.{v, u} C] (X : Cᵒᵖ) (X_1 : C) (a : (coyoneda.obj X).obj X_1) :
    (colimitCocone X).app X_1 a = id PUnit.unit

    The proposed colimit cocone over coyoneda.obj X is a colimit cocone.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      The colimit of coyoneda.obj X is isomorphic to PUnit.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def CategoryTheory.Limits.coneOfSectionCompYoneda {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J Cᵒᵖ) (X : C) (s : (F.comp (yoneda.obj X)).sections) :

        The cone of F corresponding to an element in (F ⋙ yoneda.obj X).sections.

        Equations
        Instances For
          @[simp]
          theorem CategoryTheory.Limits.coneOfSectionCompYoneda_π {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J Cᵒᵖ) (X : C) (s : (F.comp (yoneda.obj X)).sections) :
          @[simp]
          theorem CategoryTheory.Limits.coneOfSectionCompYoneda_pt {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J Cᵒᵖ) (X : C) (s : (F.comp (yoneda.obj X)).sections) :
          def CategoryTheory.yonedaJointlyReflectsLimits {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J Cᵒᵖ) (c : Limits.Cone F) (hc : (X : C) → Limits.IsLimit ((yoneda.obj X).mapCone c)) :

          The yoneda embeddings jointly reflect limits.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            noncomputable def CategoryTheory.Limits.Cocone.isColimitYonedaEquiv {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] {F : Functor J C} (c : Cocone F) :
            IsColimit c ((X : C) → IsLimit ((yoneda.obj X).mapCone c.op))

            A cocone is colimit iff it becomes limit after the application of yoneda.obj X for all X : C.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def CategoryTheory.Limits.coneOfSectionCompCoyoneda {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J C) (X : Cᵒᵖ) (s : (F.comp (coyoneda.obj X)).sections) :

              The cone of F corresponding to an element in (F ⋙ coyoneda.obj X).sections.

              Equations
              Instances For
                @[simp]
                theorem CategoryTheory.Limits.coneOfSectionCompCoyoneda_pt {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J C) (X : Cᵒᵖ) (s : (F.comp (coyoneda.obj X)).sections) :
                @[simp]
                theorem CategoryTheory.Limits.coneOfSectionCompCoyoneda_π {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J C) (X : Cᵒᵖ) (s : (F.comp (coyoneda.obj X)).sections) :
                def CategoryTheory.coyonedaJointlyReflectsLimits {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] (F : Functor J C) (c : Limits.Cone F) (hc : (X : Cᵒᵖ) → Limits.IsLimit ((coyoneda.obj X).mapCone c)) :

                The coyoneda embeddings jointly reflect limits.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  noncomputable def CategoryTheory.Limits.Cone.isLimitCoyonedaEquiv {C : Type u} [Category.{v, u} C] {J : Type w} [Category.{t, w} J] {F : Functor J C} (c : Cone F) :
                  IsLimit c ((X : Cᵒᵖ) → IsLimit ((coyoneda.obj X).mapCone c))

                  A cone is limit iff it is so after the application of coyoneda.obj X for all X : Cᵒᵖ.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    The yoneda embedding yoneda.obj X : Cᵒᵖ ⥤ Type v for X : C preserves limits.

                    The coyoneda embedding coyoneda.obj X : C ⥤ Type v for X : Cᵒᵖ preserves limits.