The simplex category #
We construct a skeletal model of the simplex category, with objects ℕ and the
morphisms n ⟶ m being the monotone maps from Fin (n + 1) to Fin (m + 1).
In Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean, we show that this category
is equivalent to NonemptyFinLinOrd.
Remarks #
The definitions SimplexCategory and SimplexCategory.Hom are marked as irreducible.
We provide the following functions to work with these objects:
- SimplexCategory.mkcreates an object of- SimplexCategoryout of a natural number. Use the notation- ⦋n⦌in the- Simpliciallocale.
- SimplexCategory.lengives the "length" of an object of- SimplexCategory, as a natural.
- SimplexCategory.Hom.mkmakes a morphism out of a monotone map between- Fin's.
- SimplexCategory.Hom.toOrderHomgives the underlying monotone map associated to a term of- SimplexCategory.Hom.
Notation #
- ⦋n⦌denotes the- n-dimensional simplex. This notation is available with- open Simplicial.
- ⦋m⦌ₙdenotes the- m-dimensional simplex in the- n-truncated simplex category. The truncation proof- p : m ≤ ncan also be provided using the syntax- ⦋m, p⦌ₙ. This notation is available with- open SimplexCategory.Truncated.
Interpret a natural number as an object of the simplex category.
Equations
- SimplexCategory.mk n = n
Instances For
the n-dimensional simplex can be denoted ⦋n⦌
Equations
- One or more equations did not get rendered due to their size.
Instances For
The length of an object of SimplexCategory.
Instances For
A recursor for SimplexCategory. Use it as induction Δ using SimplexCategory.rec.
Equations
- SimplexCategory.rec h n = h n.len
Instances For
Make a morphism in SimplexCategory from a monotone map of Fin's.
Equations
Instances For
Recover the monotone map from a morphism in the simplex category.
Equations
- f.toOrderHom = f
Instances For
Composition of morphisms of SimplexCategory.
Equations
- f.comp g = SimplexCategory.Hom.mk (f.toOrderHom.comp g.toOrderHom)
Instances For
Equations
- One or more equations did not get rendered due to their size.
The truncated simplex category.
Equations
- SimplexCategory.Truncated n = CategoryTheory.ObjectProperty.FullSubcategory fun (a : SimplexCategory) => a.len ≤ n
Instances For
Equations
Equations
- SimplexCategory.Truncated.instInhabited = { default := { obj := SimplexCategory.mk 0, property := ⋯ } }
The fully faithful inclusion of the truncated simplex category into the usual simplex category.
Equations
- SimplexCategory.Truncated.inclusion n = CategoryTheory.ObjectProperty.ι fun (a : SimplexCategory) => a.len ≤ n
Instances For
A proof that the full subcategory inclusion is fully faithful
Equations
Instances For
A quick attempt to prove that ⦋m⦌ is n-truncated (⦋m⦌.len ≤ n).
Equations
- SimplexCategory.Truncated.tacticTrunc = Lean.ParserDescr.node `SimplexCategory.Truncated.tacticTrunc 1024 (Lean.ParserDescr.nonReservedSymbol "trunc" false)
Instances For
For m ≤ n, ⦋m⦌ₙ is the m-dimensional simplex in Truncated n. The
proof p : m ≤ n can also be provided using the syntax ⦋m, p⦌ₙ.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Make a morphism in Truncated n from a morphism in SimplexCategory. This
is equivalent to @id (⦋a⦌ₙ ⟶ ⦋b⦌ₙ) f.
Equations
- SimplexCategory.Truncated.Hom.tr f ha hb = f
Instances For
The inclusion of Truncated n into Truncated m when n ≤ m.
Equations
- One or more equations did not get rendered due to their size.
Instances For
For all n ≤ m, inclusion n factors through Truncated m.