Documentation

Mathlib.AlgebraicTopology.SimplicialSet.SubcomplexColimits

Colimits involving subcomplexes of a simplicial set #

If X is a simplicial set, and we have subcomplexes A, U i (for i : ι) and V i j which satisfy Subcomplex.MulticoequalizerDiagram A U V (an abbreviation for CompleteLattice.MulticoequalizerDiagram), we show that the simplicial sset corresponding to A is the multicoequalizer of the U i along the V i j.

Similarly, bicartesian squares in the lattice Subcomplex X give pushout squares in the category of simplicial sets.

@[reducible, inline]
abbrev SSet.Subcomplex.MulticoequalizerDiagram {X : SSet} (A : X.Subcomplex) {ι : Type u_1} (U : ιX.Subcomplex) (V : ιιX.Subcomplex) :

Abbreviation for multicoequalizer diagrams in the complete lattice of subcomplexes of a simplicial set.

Equations
Instances For

    The colimit multicofork attached to a MulticoequalizerDiagram structure in the complete lattice of subcomplexes of a simplicial set.

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

      A colimit multicofork attached to a MulticoequalizerDiagram structure in the complete lattice of subcomplexes of a simplicial set. In this variant, we assume that the index type ι has a linear order. This allows to consider only the "relations" given by tuples (i, j) such that i < j.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[reducible, inline]
        abbrev SSet.Subcomplex.BicartSq {X : SSet} (A₁ A₂ A₃ A₄ : X.Subcomplex) :

        Abbreviation for bicartesian squares in the lattice of subcomplexes of a simplicial set.

        Equations
        Instances For
          theorem SSet.Subcomplex.BicartSq.isPushout {X : SSet} {A₁ A₂ A₃ A₄ : X.Subcomplex} (sq : A₁.BicartSq A₂ A₃ A₄) :