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.
A simplicial set X
satisfies the strict Segal condition if its simplices are uniquely
determined by their spine.
- spineToSimplex : {n : ℕ} → X.Path n → X.obj (Opposite.op (SimplexCategory.mk n))
The inverse to
X.spine n
. - spine_spineToSimplex : ∀ {n : ℕ} (f : X.Path n), X.spine n (SSet.StrictSegal.spineToSimplex f) = f
spineToSimplex
is a right inverse toX.spine n
. - spineToSimplex_spine : ∀ {n : ℕ} (Δ : X.obj (Opposite.op (SimplexCategory.mk n))), SSet.StrictSegal.spineToSimplex (X.spine n Δ) = Δ
spineToSimplex
is a left inverse toX.spine n
.
Instances
The fields of StrictSegal
define an equivalence between X _[n]
and Path X n
.
Equations
- SSet.StrictSegal.spineEquiv n = { toFun := X.spine n, invFun := SSet.StrictSegal.spineToSimplex, left_inv := ⋯, right_inv := ⋯ }
Instances For
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
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.