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.

@[simp]
theorem CategoryTheory.Coyoneda.colimitCocone_ι_app {C : Type u} [CategoryTheory.Category.{v, u} C] (X : Cᵒᵖ) (X_1 : C) (a : (CategoryTheory.coyoneda.obj X).obj X_1) :

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

Equations
Instances For

    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

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

        Equations
        Instances For
          Equations

          The yoneda embeddings jointly reflect limits.

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

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

            Equations
            Instances For
              Equations

              The coyoneda embeddings jointly reflect limits.

              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.

                Equations

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

                Equations
                Equations
                Equations
                Equations
                • CategoryTheory.yonedaFunctorReflectsLimits = inferInstance
                Equations
                • CategoryTheory.coyonedaFunctorReflectsLimits = inferInstance