Documentation

Mathlib.CategoryTheory.Presentable.Directed

κ-filtered categories and κ-directed poset #

In this file, we shall formalize the proof by Deligne (SGA 4 I 8.1.6) that for any (small) filtered category J, there exists a final functor F : α ⥤ J where α is a directed partially ordered set (TODO). The construction applies more generally to κ-filtered categories and κ-directed posets (TODO).

Note: the argument by Deligne is reproduced (without reference) in the book by Adámek and Rosický (theorem 1.5), but with a mistake: the construction by Deligne involves considering diagrams (see CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.DiagramWithUniqueTerminal) which are not necessarily subcategories (the class of morphisms W does not have to be multiplicative.)

References #

Let J is a κ-filtered category. In order to construct a cofinal functor α ⥤ J with a κ-directed poset α, we first consider the case where there is no object m : J such that for any object j : J, there exists a map j ⟶ m. Under this assumption (hJ), the partially ordered type DiagramWithUniqueTerminal J κ of κ-bounded diagrams with a unique terminal object in J shall be a possible choice for α.

If κ is a cardinal, this structure contains the data of a κ-bounded diagram in a category J.

Instances For
    theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.ext {J : Type w} {inst✝ : SmallCategory J} {κ : Cardinal.{w}} {x y : Diagram J κ} (W : x.W = y.W) (P : x.P = y.P) :
    x = y

    Given a κ-bounded diagram D in a category J, an object e : J is terminal if 𝟙 e belongs to D and for any object j of D, there is a unique morphism j ⟶ e in D, such that these unique morphisms are compatible with precomposition with morphisms in D.

    Instances For
      theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.IsTerminal.comm_assoc {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} {D : Diagram J κ} {e : J} (self : D.IsTerminal e) {i j : J} (f : i j) (hf : D.W f) {Z : J} (h : e Z) :
      noncomputable def CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.IsTerminal.ofExistsUnique {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} {D : Diagram J κ} {e : J} (prop_id : D.W (CategoryStruct.id e)) (h₁ : ∀ ⦃j : J⦄, D.P j∃ (lift : j e), D.W lift) (h₂ : ∀ ⦃j : J⦄, D.P j∀ (l₁ l₂ : j e), D.W l₁D.W l₂l₁ = l₂) (h₃ : ∀ ⦃i j : J⦄ (f : i j), D.W f∃ (li : i e) (lj : j e), D.W li D.W lj CategoryStruct.comp f lj = li) :

      Constructor for Diagram.IsTerminal for which no data is provided, but only its existence.

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

        If κ is a cardinal, this structure contains the data of a κ-bounded diagram with a unique terminal object in a category J.

        Instances For
          @[simp]
          theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.functorMap_comp {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} {D₁ D₂ D₃ : DiagramWithUniqueTerminal J κ} (h₁₂ : D₁ D₂) (h₂₃ : D₂ D₃) :
          @[simp]
          theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.functorMap_comp_assoc {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} {D₁ D₂ D₃ : DiagramWithUniqueTerminal J κ} (h₁₂ : D₁ D₂) (h₂₃ : D₂ D₃) {Z : J} (h : D₃.top Z) :

          The functor which sends a κ-bounded diagram with a unique terminal object to its terminal object.

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

            The diagram containing a single object (and its identity morphism).

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

              The diagram with a unique terminal object containing a single object (and its identity morphism).

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

                The union of a κ-bounded family of κ-bounded diagrams.

                Equations
                Instances For
                  @[simp]
                  theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.iSup_W {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} [Fact κ.IsRegular] {ι : Type u_1} (D : ιDiagram J κ) ( : HasCardinalLT ι κ) :
                  (iSup D ).W = ⨆ (i : ι), (D i).W
                  @[simp]
                  theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.iSup_P {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} [Fact κ.IsRegular] {ι : Type u_1} (D : ιDiagram J κ) ( : HasCardinalLT ι κ) (a✝ : J) :
                  (iSup D ).P a✝ = (⨆ (i : ι), (D i).P) a✝

                  The union of two κ-bounded diagrams.

                  Equations
                  • D₁.sup D₂ = { W := D₁.WD₂.W, P := D₁.PD₂.P, src := , tgt := , hW := , hP := }
                  Instances For
                    @[simp]
                    theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.sup_P {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} [Fact κ.IsRegular] (D₁ D₂ : Diagram J κ) (a✝ : J) :
                    (D₁.sup D₂).P a✝ = Max.max D₁.P D₂.P a✝
                    @[simp]
                    theorem CategoryTheory.IsCardinalFiltered.exists_cardinal_directed.Diagram.sup_W {J : Type w} [SmallCategory J] {κ : Cardinal.{w}} [Fact κ.IsRegular] (D₁ D₂ : Diagram J κ) :
                    (D₁.sup D₂).W = D₁.WD₂.W