Documentation

Mathlib.RingTheory.HopfAlgebra

Hopf algebras #

In this file we define HopfAlgebra, and provide instances for:

Main definitions #

TODO #

References #

class HopfAlgebra (R : Type u) (A : Type v) [CommSemiring R] [Semiring A] extends Bialgebra :
Type (max u v)

A Hopf algebra over a commutative (semi)ring R is a bialgebra over R equipped with an R-linear endomorphism antipode satisfying the antipode axioms.

Instances
    @[simp]
    theorem HopfAlgebra.mul_antipode_rTensor_comul_apply {R : Type u} {A : Type v} [CommSemiring R] [Semiring A] [HopfAlgebra R A] (a : A) :
    (LinearMap.mul' R A) ((LinearMap.rTensor A HopfAlgebra.antipode) (Coalgebra.comul a)) = (algebraMap R A) (Coalgebra.counit a)
    @[simp]
    theorem HopfAlgebra.mul_antipode_lTensor_comul_apply {R : Type u} {A : Type v} [CommSemiring R] [Semiring A] [HopfAlgebra R A] (a : A) :
    (LinearMap.mul' R A) ((LinearMap.lTensor A HopfAlgebra.antipode) (Coalgebra.comul a)) = (algebraMap R A) (Coalgebra.counit a)
    noncomputable instance CommSemiring.toHopfAlgebra (R : Type u) [CommSemiring R] :

    Every commutative (semi)ring is a Hopf algebra over itself

    Equations
    @[simp]
    theorem CommSemiring.antipode_eq_id (R : Type u) [CommSemiring R] :
    HopfAlgebra.antipode = LinearMap.id