Documentation

Mathlib.AlgebraicTopology.SimplexCategory.Augmented.Monoidal

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.

@[reducible, inline]

An auxiliary definition for the tensor product of two objects in AugmentedSimplexCategory.

Equations
Instances For
    def AugmentedSimplexCategory.tensorHomOf {x₁ y₁ x₂ y₂ : SimplexCategory} (f₁ : x₁ y₁) (f₂ : x₂ y₂) :
    tensorObjOf x₁ x₂ tensorObjOf y₁ y₂

    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
      def AugmentedSimplexCategory.tensorHom {x₁ y₁ x₂ y₂ : AugmentedSimplexCategory} (f₁ : x₁ y₁) (f₂ : x₂ y₂) :
      x₁.tensorObj x₂ y₁.tensorObj y₂

      The action of the tensor product on maps of AugmentedSimplexCategory.

      Equations
      Instances For
        @[reducible, inline]

        The unit for the monoidal structure on AugmentedSimplexCategory is the initial object.

        Equations
        Instances For

          The associator isomorphism for the monoidal structure on AugmentedSimplexCategory

          Equations
          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
                  @[reducible, inline]

                  To ease type checking, we also provide a version of inl that lives in SimplexCategory.

                  Equations
                  Instances For
                    @[reducible, inline]

                    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.