A simplicial set is just a simplicial object in Type
,
i.e. a Type
-valued presheaf on the simplex category.
(One might be tempted to call these "simplicial types" when working in type-theoretic foundations, but this would be unnecessarily confusing given the existing notion of a simplicial type in homotopy type theory.)
We define the standard simplices Δ[n]
as simplicial sets,
and their boundaries ∂Δ[n]
and horns Λ[n, i]
.
(The notations are available via open_locale simplicial
.)
Future work #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
There isn't yet a complete API for simplices, boundaries, and horns.
As an example, we should have a function that constructs
from a non-surjective order preserving function fin n → fin n
a morphism Δ[n] ⟶ ∂Δ[n]
.
The category of simplicial sets.
This is the category of contravariant functors from
simplex_category
to Type u
.
Equations
Instances for sSet
The n
-th standard simplex Δ[n]
associated with a nonempty finite linear order n
is the Yoneda embedding of n
.
Equations
Equations
The m
-simplices of the n
-th standard simplex are
the monotone maps from fin (m+1)
to fin (n+1)
.
Equations
The boundary ∂Δ[n]
of the n
-th standard simplex consists of
all m
-simplices of standard_simplex n
that are not surjective
(when viewed as monotone function m → n
).
Equations
- sSet.boundary n = {obj := λ (m : simplex_categoryᵒᵖ), {α // ¬function.surjective ⇑(sSet.as_order_hom α)}, map := λ (m₁ m₂ : simplex_categoryᵒᵖ) (f : m₁ ⟶ m₂) (α : {α // ¬function.surjective ⇑(sSet.as_order_hom α)}), ⟨f.unop ≫ ↑α, _⟩, map_id' := _, map_comp' := _}
The inclusion of the boundary of the n
-th standard simplex into that standard simplex.
Equations
- sSet.boundary_inclusion n = {app := λ (m : simplex_categoryᵒᵖ) (α : {α // ¬function.surjective ⇑(sSet.as_order_hom α)}), ↑α, naturality' := _}
horn n i
(or Λ[n, i]
) is the i
-th horn of the n
-th standard simplex, where i : n
.
It consists of all m
-simplices α
of Δ[n]
for which the union of {i}
and the range of α
is not all of n
(when viewing α
as monotone function m → n
).
The inclusion of the i
-th horn of the n
-th standard simplex into that standard simplex.
Equations
- sSet.horn_inclusion n i = {app := λ (m : simplex_categoryᵒᵖ) (α : {α // set.range ⇑(sSet.as_order_hom α) ∪ {i} ≠ set.univ}), ↑α, naturality' := _}
The simplicial circle.
Truncated simplicial sets.
Equations
Instances for sSet.truncated
The skeleton functor on simplicial sets.
Equations
Equations
The category of augmented simplicial sets, as a particular case of augmented simplicial objects.
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
- sSet.augmented.standard_simplex = {obj := λ (Δ : simplex_category), {left := sSet.standard_simplex.obj Δ, right := ⊤_ Type, hom := {app := λ (Δ' : simplex_categoryᵒᵖ), category_theory.limits.terminal.from (((𝟭 (category_theory.simplicial_object Type)).obj (sSet.standard_simplex.obj Δ)).obj Δ'), naturality' := _}}, map := λ (Δ₁ Δ₂ : simplex_category) (θ : Δ₁ ⟶ Δ₂), {left := sSet.standard_simplex.map θ, right := category_theory.limits.terminal.from {left := sSet.standard_simplex.obj Δ₁, right := ⊤_ Type, hom := {app := λ (Δ' : simplex_categoryᵒᵖ), category_theory.limits.terminal.from (((𝟭 (category_theory.simplicial_object Type)).obj (sSet.standard_simplex.obj Δ₁)).obj Δ'), naturality' := _}}.right, w' := _}, map_id' := sSet.augmented.standard_simplex._proof_10, map_comp' := sSet.augmented.standard_simplex._proof_11}
The functor associating the singular simplicial set to a topological space.
The geometric realization functor.
Geometric realization is left adjoint to the singular simplicial set construction.
The geometric realization of the representable simplicial sets agree with the usual topological simplices.