Documentation

Mathlib.CategoryTheory.Limits.Indization.Category

The category of Ind-objects #

We define the v-category of Ind-objects of a category C, called Ind C, as well as the functors Ind.yoneda : C ⥤ Ind C and Ind.inclusion C : Ind C ⥤ Cᵒᵖ ⥤ Type v.

This file will mainly collect results about ind-objects (stated in terms of IsIndObject) and reinterpret them in terms of Ind C.

Adopting the theorem numbering of [KS06], we show that

More limit-colimit properties will follow.

Note that:

References #

The category of Ind-objects of C.

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

    The defining properties of Ind C are that its morphisms live in v and that it is equivalent to the full subcategory of Cᵒᵖ ⥤ Type v containing the ind-objects.

    Equations
    Instances For

      The canonical inclusion of ind-objects into presheaves.

      Equations
      Instances For

        The functor Ind C ⥤ Cᵒᵖ ⥤ Type v is fully faithful.

        Equations
        Instances For

          The inclusion of C into Ind C induced by the Yoneda embedding.

          Equations
          Instances For
            instance CategoryTheory.instFullIndYoneda {C : Type u} [CategoryTheory.Category.{v, u} C] :
            CategoryTheory.Ind.yoneda.Full
            instance CategoryTheory.instFaithfulIndYoneda {C : Type u} [CategoryTheory.Category.{v, u} C] :
            CategoryTheory.Ind.yoneda.Faithful
            noncomputable def CategoryTheory.Ind.yoneda.fullyFaithful {C : Type u} [CategoryTheory.Category.{v, u} C] :
            CategoryTheory.Ind.yoneda.FullyFaithful

            The functor C ⥤ Ind C is fully faithful.

            Equations
            Instances For
              noncomputable def CategoryTheory.Ind.yonedaCompInclusion {C : Type u} [CategoryTheory.Category.{v, u} C] :
              CategoryTheory.Ind.yoneda.comp (CategoryTheory.Ind.inclusion C) CategoryTheory.yoneda

              The composition C ⥤ Ind C ⥤ (Cᵒᵖ ⥤ Type v) is just the Yoneda embedding.

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

                Pick a presentation of an ind-object X using choice.

                Equations
                • X.presentation = .presentation
                Instances For
                  noncomputable def CategoryTheory.Ind.colimitPresentationCompYoneda {C : Type u} [CategoryTheory.Category.{v, u} C] (X : CategoryTheory.Ind C) :
                  CategoryTheory.Limits.colimit (X.presentation.F.comp CategoryTheory.Ind.yoneda) X

                  An ind-object X is the colimit (in Ind C!) of the filtered diagram presenting it.

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