Documentation

Mathlib.CategoryTheory.Monoidal.Preadditive

Preadditive monoidal categories #

A monoidal category is MonoidalPreadditive if it is preadditive and tensor product of morphisms is linear in both factors.

A category is MonoidalPreadditive if tensoring is additive in both factors.

Note we don't extend Preadditive C here, as Abelian C already extends it, and we'll need to have both typeclasses sometimes.

Instances

    A faithful additive monoidal functor to a monoidal preadditive category ensures that the domain is monoidal preadditive.

    theorem CategoryTheory.whiskerLeft_sum {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] [MonoidalCategory C] [MonoidalPreadditive C] (P : C) {Q R : C} {J : Type u_2} (s : Finset J) (g : J(Q R)) :
    theorem CategoryTheory.sum_whiskerRight {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] [MonoidalCategory C] [MonoidalPreadditive C] {Q R : C} {J : Type u_2} (s : Finset J) (g : J(Q R)) (P : C) :
    theorem CategoryTheory.tensor_sum {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] [MonoidalCategory C] [MonoidalPreadditive C] {P Q R S : C} {J : Type u_2} (s : Finset J) (f : P Q) (g : J(R S)) :
    MonoidalCategoryStruct.tensorHom f (∑ js, g j) = js, MonoidalCategoryStruct.tensorHom f (g j)
    theorem CategoryTheory.sum_tensor {C : Type u_1} [Category.{u_3, u_1} C] [Preadditive C] [MonoidalCategory C] [MonoidalPreadditive C] {P Q R S : C} {J : Type u_2} (s : Finset J) (f : P Q) (g : J(R S)) :
    MonoidalCategoryStruct.tensorHom (∑ js, g j) f = js, MonoidalCategoryStruct.tensorHom (g j) f

    The isomorphism showing how tensor product on the left distributes over direct sums.

    Equations
    Instances For

      The isomorphism showing how tensor product on the right distributes over direct sums.

      Equations
      Instances For