Documentation

Mathlib.CategoryTheory.GradedObject.Monoidal

The monoidal category structures on graded objects #

Assuming that C is a monoidal category and that I is an additive monoid, we introduce a partially defined tensor product on the category GradedObject I C: given X₁ and X₂ two objects in GradedObject I C, we define GradedObject.Monoidal.tensorObj X₁ X₂ under the assumption HasTensor X₁ X₂ that the coproduct of X₁ i ⊗ X₂ j for i + j = n exists for any n : I.

@[reducible, inline]

The tensor product of two graded objects X₁ and X₂ exists if for any n, the coproduct of the objects X₁ i ⊗ X₂ j for i + j = n exists.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[reducible, inline]

    The tensor product of two graded objects.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      noncomputable def CategoryTheory.GradedObject.Monoidal.ιTensorObj {I : Type u} [AddMonoid I] {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.MonoidalCategory C] (X₁ : CategoryTheory.GradedObject I C) (X₂ : CategoryTheory.GradedObject I C) [X₁.HasTensor X₂] (i₁ : I) (i₂ : I) (i₁₂ : I) (h : i₁ + i₂ = i₁₂) :

      The inclusion of a summand in a tensor product of two graded objects.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        noncomputable def CategoryTheory.GradedObject.Monoidal.tensorObjDesc {I : Type u} [AddMonoid I] {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.MonoidalCategory C] {X₁ : CategoryTheory.GradedObject I C} {X₂ : CategoryTheory.GradedObject I C} [X₁.HasTensor X₂] {A : C} {k : I} (f : (i₁ i₂ : I) → i₁ + i₂ = k(CategoryTheory.MonoidalCategory.tensorObj (X₁ i₁) (X₂ i₂) A)) :

        Constructor for morphisms from a tensor product of two graded objects.

        Equations
        Instances For
          @[simp]
          theorem CategoryTheory.GradedObject.Monoidal.ι_tensorObjDesc_assoc {I : Type u} [AddMonoid I] {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.MonoidalCategory C] {X₁ : CategoryTheory.GradedObject I C} {X₂ : CategoryTheory.GradedObject I C} [X₁.HasTensor X₂] {A : C} {k : I} (f : (i₁ i₂ : I) → i₁ + i₂ = k(CategoryTheory.MonoidalCategory.tensorObj (X₁ i₁) (X₂ i₂) A)) (i₁ : I) (i₂ : I) (hi : i₁ + i₂ = k) {Z : C} (h : A Z) :
          @[simp]
          theorem CategoryTheory.GradedObject.Monoidal.ι_tensorObjDesc {I : Type u} [AddMonoid I] {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.MonoidalCategory C] {X₁ : CategoryTheory.GradedObject I C} {X₂ : CategoryTheory.GradedObject I C} [X₁.HasTensor X₂] {A : C} {k : I} (f : (i₁ i₂ : I) → i₁ + i₂ = k(CategoryTheory.MonoidalCategory.tensorObj (X₁ i₁) (X₂ i₂) A)) (i₁ : I) (i₂ : I) (hi : i₁ + i₂ = k) :

          The morphism tensorObj X₁ Y₁ ⟶ tensorObj X₂ Y₂ induced by morphisms of graded objects f : X₁ ⟶ X₂ and g : Y₁ ⟶ Y₂.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem CategoryTheory.GradedObject.Monoidal.ι_tensorHom {I : Type u} [AddMonoid I] {C : Type u_1} [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.MonoidalCategory C] {X₁ : CategoryTheory.GradedObject I C} {X₂ : CategoryTheory.GradedObject I C} {Y₁ : CategoryTheory.GradedObject I C} {Y₂ : CategoryTheory.GradedObject I C} (f : X₁ X₂) (g : Y₁ Y₂) [X₁.HasTensor Y₁] [X₂.HasTensor Y₂] (i₁ : I) (i₂ : I) (i₁₂ : I) (h : i₁ + i₂ = i₁₂) :
            @[reducible, inline]

            The morphism tensorObj X Y₁ ⟶ tensorObj X Y₂ induced by a morphism of graded objects φ : Y₁ ⟶ Y₂.

            Equations
            Instances For
              @[reducible, inline]

              The morphism tensorObj X₁ Y ⟶ tensorObj X₂ Y induced by a morphism of graded objects φ : X₁ ⟶ X₂.

              Equations
              Instances For