Paths in simplicial sets #
A path in a simplicial set X
of length n
is a directed path comprised of n + 1
0-simplices
and n
1-simplices, together with identifications between 0-simplices and the sources and targets
of the 1-simplices.
An n
-simplex has a maximal path, the spine
of the simplex, which is a path of length n
.
A path in a simplicial set X
of length n
is a directed path of n
edges.
- vertex : Fin (n + 1) → X.obj (Opposite.op (SimplexCategory.mk 0))
A path includes the data of
n+1
0-simplices inX
. - arrow : Fin n → X.obj (Opposite.op (SimplexCategory.mk 1))
A path includes the data of
n
1-simplices inX
. - arrow_src : ∀ (i : Fin n), CategoryTheory.SimplicialObject.δ X 1 (self.arrow i) = self.vertex i.castSucc
The sources of the 1-simplices in a path are identified with appropriate 0-simplices.
- arrow_tgt : ∀ (i : Fin n), CategoryTheory.SimplicialObject.δ X 0 (self.arrow i) = self.vertex i.succ
The targets of the 1-simplices in a path are identified with appropriate 0-simplices.
Instances For
For j + l ≤ n
, a path of length n
restricts to a path of length l
, namely the subpath
spanned by the vertices j ≤ i ≤ j + l
and edges j ≤ i < j + l
.
Equations
Instances For
The spine of an n
-simplex in X
is the path of edges of length n
formed by
traversing through its vertices in order.
Equations
- One or more equations did not get rendered due to their size.