Documentation

Mathlib.Algebra.Category.AlgCat.Monoidal

The monoidal category structure on R-algebras #

@[reducible, inline]
noncomputable abbrev AlgCat.instMonoidalCategory.tensorObj {R : Type u} [CommRing R] (X Y : AlgCat R) :

Auxiliary definition used to fight a timeout when building AlgCat.instMonoidalCategory.

Equations
Instances For
    @[simp]
    theorem AlgCat.instMonoidalCategory.tensorObj_carrier {R : Type u} [CommRing R] (X Y : AlgCat R) :
    (tensorObj X Y) = TensorProduct R X Y
    @[reducible, inline]
    noncomputable abbrev AlgCat.instMonoidalCategory.tensorHom {R : Type u} [CommRing R] {W X Y Z : AlgCat R} (f : W X) (g : Y Z) :

    Auxiliary definition used to fight a timeout when building AlgCat.instMonoidalCategory.

    Equations
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      • One or more equations did not get rendered due to their size.