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.
StrictSegal
simplicial sets have an important property of being 2-coskeletal which is proven
in Mathlib.AlgebraicTopology.SimplicialSet.Coskeletal
.
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
. 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
For any σ : X ⟶ Y
between StrictSegal
simplicial sets, spineToSimplex
commutes with Path.map
.
If we take the path along the spine of the j
th face of a spineToSimplex
,
the common vertices will agree with those of the original path f
. In particular,
a vertex i
with i < j
can be identified with the same vertex in f
.
If we take the path along the spine of the j
th face of a spineToSimplex
,
a vertex i
with i ≥ j
can be identified with vertex i + 1
in the original
path.
If we take the path along the spine of the j
th face of a spineToSimplex
,
the common arrows will agree with those of the original path f
. In particular,
an arrow i
with i + 1 < j
can be identified with the same arrow in f
.
If we take the path along the spine of the j
th face of a spineToSimplex
,
an arrow i
with i + 1 > j
can be identified with arrow i + 1
in the
original path.
If we take the path along the spine of a face of a spineToSimplex
, the
arrows not contained in the original path can be recovered as the diagonal edge
of the spineToSimplex
that "composes" arrows i
and i + 1
.
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.