The standard simplex #
We define the standard simplices Δ[n] as simplicial sets.
See files SimplicialSet.Boundary and SimplicialSet.Horn
for their boundaries∂Δ[n] and horns Λ[n, i].
(The notations are available via open Simplicial.)
The functor SimplexCategory ⥤ SSet which sends ⦋n⦌ to the standard simplex Δ[n] is a
cosimplicial object in the category of simplicial sets. (This functor is essentially given by the
Yoneda embedding).
Instances For
The functor SimplexCategory ⥤ SSet which sends ⦋n⦌ to the standard simplex Δ[n] is a
cosimplicial object in the category of simplicial sets. (This functor is essentially given by the
Yoneda embedding).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- SSet.instInhabited = { default := SSet.stdSimplex.obj (SimplexCategory.mk 0) }
Equations
- SSet.instInhabitedTruncated = { default := (SSet.truncation n).obj (SSet.stdSimplex.obj (SimplexCategory.mk 0)) }
Simplices of the standard simplex identify to morphisms in SimplexCategory.
Equations
Instances For
If x : Δ[n] _⦋d⦌ and i : Fin (d + 1), we may evaluate x i : Fin (n + 1).
Equations
- One or more equations did not get rendered due to their size.
Constructor for simplices of the standard simplex which takes a OrderHom as an input.
Equations
Instances For
The m-simplices of the n-th standard simplex are
the monotone maps from Fin (m+1) to Fin (n+1).
Equations
Instances For
The canonical bijection (stdSimplex.obj n ⟶ X) ≃ X.obj (op n).
Instances For
The (degenerate) m-simplex in the standard simplex concentrated in vertex k.
Equations
- SSet.stdSimplex.const n k m = SSet.stdSimplex.objMk ((OrderHom.const (Fin ((Opposite.unop m).len + 1))) k)
Instances For
The 0-simplices of Δ[n] identify to the elements in Fin (n + 1).
Equations
- One or more equations did not get rendered due to their size.
Instances For
The edge of the standard simplex with endpoints a and b.
Equations
- SSet.stdSimplex.edge n a b hab = SSet.stdSimplex.objMk { toFun := ![a, b], monotone' := ⋯ }
Instances For
The triangle in the standard simplex with vertices a, b, and c.
Equations
- SSet.stdSimplex.triangle a b c hab hbc = SSet.stdSimplex.objMk { toFun := ![a, b, c], monotone' := ⋯ }
Instances For
If S : Finset (Fin (n + 1)) is order isomorphic to Fin (m + 1),
then the face face S of Δ[n] is representable by m,
i.e. face S is isomorphic to Δ[m], see stdSimplex.isoOfRepresentableBy.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If a simplicial set X is representable by ⦋m⦌ for some m : ℕ, then this is the
corresponding isomorphism Δ[m] ≅ X.
Equations
Instances For
The standard simplex identifies to the nerve to the preordered type
ULift (Fin (n + 1)).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Nondegenerate d-dimensional simplices of the standard simplex Δ[n]
identify to order embeddings Fin (d + 1) ↪o Fin (n + 1).
Equations
- One or more equations did not get rendered due to their size.
Instances For
The simplicial circle.
Equations
Instances For
The functor which sends ⦋n⦌ to the simplicial set Δ[n] equipped by
the obvious augmentation towards the terminal object of the category of sets.
Equations
- One or more equations did not get rendered due to their size.