The category of commutative bialgebras over a commutative ring #
This file defines the bundled category CommBialgCat R
of commutative bialgebras over a fixed
commutative ring R
along with the forgetful functor to CommAlgCat
.
Equations
Turn an unbundled R
-bialgebra into the corresponding object in the category of R
-bialgebras.
This is the preferred way to construct a term of CommBialgCat R
.
Equations
- CommBialgCat.of R X = { carrier := X, commRing := inst✝¹, bialgebra := inst✝ }
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.
Turn a morphism in CommBialgCat
back into a BialgHom
.
Equations
Instances For
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- CommBialgCat.Hom.Simps.hom A B f = f.hom
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- CommBialgCat.instInhabited = { default := CommBialgCat.of R R }
Equations
Equations
Equations
- One or more equations did not get rendered due to their size.
Forgetting to the underlying type and then building the bundled object returns the original bialgebra.
Equations
- M.ofSelfIso = { hom := CategoryTheory.CategoryStruct.id M, inv := CategoryTheory.CategoryStruct.id M, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build an isomorphism in the category CommBialgCat R
from a BialgEquiv
between
Bialgebra
s.
Equations
- CommBialgCat.isoMk e = { hom := CommBialgCat.ofHom ↑e, inv := CommBialgCat.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build a BialgEquiv
from an isomorphism in the category CommBialgCat R
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Bialgebra equivalences between Bialgebra
s are the same as isomorphisms in CommBialgCat
.
Equations
- CommBialgCat.isoEquivBialgEquiv = { toFun := CommBialgCat.bialgEquivOfIso, invFun := CommBialgCat.isoMk, left_inv := ⋯, right_inv := ⋯ }
Instances For
Equations
- CommAlgCat.mon_ClassOpOf = { one := (CommAlgCat.ofHom (Bialgebra.counitAlgHom R A)).op, mul := (CommAlgCat.ofHom (Bialgebra.comulAlgHom R A)).op, one_mul := ⋯, mul_one := ⋯, mul_assoc := ⋯ }
Commutative bialgebras over a commutative ring R
are the same thing as comonoid
R
-algebras.
Equations
- One or more equations did not get rendered due to their size.