Documentation

Mathlib.Algebra.Category.BialgebraCat.Monoidal

The monoidal structure on the category of bialgebras #

In Mathlib.RingTheory.Bialgebra.TensorProduct, given two R-bialgebras A, B, we define a bialgebra instance on A ⊗[R] B as well as the tensor product of two BialgHoms as a BialgHom, and the associator and left/right unitors for bialgebras as BialgEquivs. In this file, we declare a MonoidalCategory instance on the category of bialgebras, with data fields given by the definitions in Mathlib.RingTheory.Bialgebra.TensorProduct, and Prop fields proved by pulling back the MonoidalCategory instance on the category of algebras, using Monoidal.induced.

Equations
  • One or more equations did not get rendered due to their size.
@[simp]
theorem BialgebraCat.instMonoidalCategoryStruct_tensorHom (R : Type u) [CommRing R] {X₁✝ Y₁✝ X₂✝ Y₂✝ : BialgebraCat R} (f : X₁✝ Y₁✝) (g : X₂✝ Y₂✝) :

The data needed to induce a MonoidalCategory structure via BialgebraCat.instMonoidalCategoryStruct and the forgetful functor to algebras.

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

    forget₂ (BialgebraCat R) (AlgebraCat R) as a monoidal functor.

    Equations

    forget₂ (BialgebraCat R) (CoalgebraCat R) as a monoidal functor.

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