Monoidal structure on the augmented simplex category #
This file defines a monoidal structure on AugmentedSimplexCategory
.
The tensor product of objects is characterized by the fact that the initial object star
is
also the unit, and the fact that ⦋m⦌ ⊗ ⦋n⦌ = ⦋m + n + 1⦌
for n m : ℕ
.
Through the (not in mathlib) equivalence between AugmentedSimplexCategory
and the category
of finite ordinals, the tensor products corresponds to ordinal sum.
As the unit of this structure is an initial object, for every x y : AugmentedSimplexCategory
,
there are maps AugmentedSimplexCategory.inl x y : x ⟶ x ⊗ y
and
AugmentedSimplexCategory.inr x y : y ⟶ x ⊗ y
. The main API for working with the tensor product
of maps is given by AugmentedSimplexCategory.tensorObj_hom_ext
, which characterizes maps
x ⊗ y ⟶ z
in terms of their composition with these two maps. We also characterize the behaviour
of the associator isomorphism with respect to these maps.
An auxiliary definition for the tensor product of two objects in AugmentedSimplexCategory
.
Equations
- AugmentedSimplexCategory.tensorObjOf m n = SimplexCategory.mk (m.len + n.len + 1)
Instances For
The tensor product of two objects of AugmentedSimplexCategory
.
Equations
- AugmentedSimplexCategory.tensorObj (CategoryTheory.WithInitial.of m_2) (CategoryTheory.WithInitial.of n_2) = CategoryTheory.WithInitial.of (AugmentedSimplexCategory.tensorObjOf m_2 n_2)
- AugmentedSimplexCategory.tensorObj CategoryTheory.WithInitial.star n = n
- m.tensorObj CategoryTheory.WithInitial.star = m
Instances For
The action of the tensor product on maps coming from SimplexCategory
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The action of the tensor product on maps of AugmentedSimplexCategory
.
Equations
- One or more equations did not get rendered due to their size.
- AugmentedSimplexCategory.tensorHom f₁_2 f₂_2 = AugmentedSimplexCategory.tensorHomOf f₁_2 f₂_2
- AugmentedSimplexCategory.tensorHom x f₂_2 = f₂_2
- AugmentedSimplexCategory.tensorHom f₁_2 x = f₁_2
- AugmentedSimplexCategory.tensorHom f₁ f₂ = CategoryTheory.WithInitial.starInitial.to (y₁.tensorObj y₂)
Instances For
The unit for the monoidal structure on AugmentedSimplexCategory
is the initial object.
Instances For
The associator isomorphism for the monoidal structure on AugmentedSimplexCategory
Equations
- One or more equations did not get rendered due to their size.
- AugmentedSimplexCategory.associator (CategoryTheory.WithInitial.of x_2) (CategoryTheory.WithInitial.of y_2) (CategoryTheory.WithInitial.of z_2) = CategoryTheory.eqToIso ⋯
Instances For
The left unitor isomorphism for the monoidal structure in AugmentedSimplexCategory
Equations
- AugmentedSimplexCategory.leftUnitor (CategoryTheory.WithInitial.of a) = CategoryTheory.Iso.refl (AugmentedSimplexCategory.tensorUnit.tensorObj (CategoryTheory.WithInitial.of a))
- AugmentedSimplexCategory.leftUnitor CategoryTheory.WithInitial.star = CategoryTheory.Iso.refl (AugmentedSimplexCategory.tensorUnit.tensorObj CategoryTheory.WithInitial.star)
Instances For
The right unitor isomorphism for the monoidal structure in AugmentedSimplexCategory
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Thanks to tensorUnit
being initial in AugmentedSimplexCategory
, we get
a morphism Δ ⟶ Δ ⊗ Δ'
for every pair of objects Δ, Δ'
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Thanks to tensorUnit
being initial in AugmentedSimplexCategory
, we get
a morphism Δ' ⟶ Δ ⊗ Δ'
for every pair of objects Δ, Δ'
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
To ease type checking, we also provide a version of inl that lives in
SimplexCategory
.
Equations
Instances For
To ease type checking, we also provide a version of inr that lives in
SimplexCategory
.
Equations
Instances For
We can characterize morphisms out of a tensor product via their precomposition with inl
and
inr
.
Equations
- One or more equations did not get rendered due to their size.