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.

For a small filtered category I, we also define Ind.lim I : (I ⥤ C) ⥤ Ind C and show that it preserves finite limits and finite colimits.

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 [Kashiwara2006], we show the following properties:

Limits:

Colimits:

Note that:

References #

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 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
      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      • One or more equations did not get rendered due to their size.

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

      Equations
      Instances For

        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
          noncomputable def CategoryTheory.Ind.lim {C : Type u} [Category.{v, u} C] (I : Type v) [SmallCategory I] [IsFiltered I] :
          Functor (Functor I C) (Ind C)

          This is the functor (I ⥤ C) ⥤ Ind C that sends a functor F to colim (Y ∘ F), where Y is the Yoneda embedding. It is known as "ind-lim" and denoted “colim” in [Kashiwara2006].

          Equations
          Instances For

            Computing ind-lims in Ind C is the same as computing them in Cᵒᵖ ⥤ Type v.

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

              Given an IndParallelPairPresentation f g, we can understand the parallel pair (f, g) as the colimit of (P.φ, P.ψ) in Ind C.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                theorem CategoryTheory.Ind.exists_nonempty_arrow_mk_iso_ind_lim {C : Type u} [Category.{v, u} C] {A B : Ind C} {f : A B} :
                ∃ (I : Type v) (x : SmallCategory I) (x_1 : IsFiltered I) (F : Functor I C) (G : Functor I C) (φ : F G), Nonempty (Arrow.mk f Arrow.mk ((Ind.lim I).map φ))

                A way to understand morphisms in Ind C: every morphism is induced by a natural transformation of diagrams.

                For small finitely cocomplete categories C : Type u, the category of Ind-objects Ind C is equivalent to the category of left-exact functors Cᵒᵖ ⥤ Type u

                Equations
                Instances For