Documentation

Mathlib.AlgebraicTopology.SimplicialSet.StrictSegal

Strict Segal simplicial sets #

A simplicial set X satisfies the StrictSegal condition if for all n, the map X.spine n : X _[n] → X.Path n is an equivalence, with equivalence inverse spineToSimplex {n : ℕ} : Path X n → X _[n].

Examples of StrictSegal simplicial sets are given by nerves of categories.

TODO: Show that these are the only examples: that a StrictSegal simplicial set is isomorphic to the nerve of its homotopy category.

class SSet.StrictSegal (X : SSet) :

A simplicial set X satisfies the strict Segal condition if its simplices are uniquely determined by their spine.

Instances
    def SSet.StrictSegal.spineEquiv {X : SSet} [X.StrictSegal] (n : ) :
    X.obj (Opposite.op (SimplexCategory.mk n)) X.Path n

    The fields of StrictSegal define an equivalence between X _[n] and Path X n.

    Equations
    Instances For
      @[simp]
      theorem SSet.StrictSegal.spineToSimplex_vertex {X : SSet} [X.StrictSegal] {n : } (i : Fin (n + 1)) (f : X.Path n) :
      @[simp]
      theorem SSet.StrictSegal.spineToSimplex_arrow {X : SSet} [X.StrictSegal] {n : } (i : Fin n) (f : X.Path n) :
      def SSet.StrictSegal.spineToDiagonal {X : SSet} [X.StrictSegal] {n : } (f : X.Path n) :

      In the presence of the strict Segal condition, a path of length n can be "composed" by taking the diagonal edge of the resulting n-simplex.

      Equations
      Instances For
        @[simp]
        theorem SSet.StrictSegal.spineToSimplex_interval {X : SSet} [X.StrictSegal] {n : } (f : X.Path n) (j l : ) (hjl : j + l n) :
        theorem SSet.StrictSegal.spineToSimplex_edge {X : SSet} [X.StrictSegal] {n : } (f : X.Path n) (j l : ) (hjl : j + l n) :
        noncomputable instance Nerve.strictSegal (C : Type u) [CategoryTheory.Category.{v, u} C] :
        (CategoryTheory.nerve C).StrictSegal

        Simplices in the nerve of categories are uniquely determined by their spine. Indeed, this property describes the essential image of the nerve functor.

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