Documentation

Mathlib.Algebra.Category.AlgebraCat.Monoidal

The monoidal category structure on R-algebras #

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

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

Equations
Instances For
    @[reducible, inline]
    noncomputable abbrev AlgebraCat.instMonoidalCategory.tensorHom {R : Type u} [CommRing R] {W X Y Z : AlgebraCat R} (f : W X) (g : Y Z) :

    Auxiliary definition used to fight a timeout when building AlgebraCat.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.