Group-like elements in a Hopf algebra #
This file proves that group-like elements in a Hopf algebra form a group.
@[simp]
theorem
IsGroupLikeElem.antipode_mul_cancel
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
{a : A}
(ha : IsGroupLikeElem R a)
:
@[simp]
theorem
IsGroupLikeElem.mul_antipode_cancel
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
{a : A}
(ha : IsGroupLikeElem R a)
:
def
GroupLike.toUnits
(R : Type u_1)
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
:
Turn a group-like element a into a unit with inverse its antipode.
Equations
- GroupLike.toUnits R = { toFun := fun (a : GroupLike R A) => { val := ↑a, inv := (HopfAlgebraStruct.antipode R) ↑a, val_inv := ⋯, inv_val := ⋯ }, map_one' := ⋯, map_mul' := ⋯ }
Instances For
@[simp]
theorem
GroupLike.val_inv_toUnits_apply
(R : Type u_1)
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
(a : GroupLike R A)
:
@[simp]
theorem
GroupLike.val_toUnits_apply
(R : Type u_1)
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
(a : GroupLike R A)
:
theorem
IsGroupLikeElem.isUnit
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
{a : A}
(ha : IsGroupLikeElem R a)
:
IsUnit a
@[simp]
theorem
IsGroupLikeElem.antipode
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
{a : A}
(ha : IsGroupLikeElem R a)
:
IsGroupLikeElem R ((HopfAlgebraStruct.antipode R) a)
@[simp]
theorem
IsGroupLikeElem.antipode_antipode
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
{a : A}
(ha : IsGroupLikeElem R a)
:
instance
GroupLike.instInv
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
:
Equations
- GroupLike.instInv = { inv := fun (a : GroupLike R A) => { val := (HopfAlgebraStruct.antipode R) ↑a, isGroupLikeElem_val := ⋯ } }
@[simp]
theorem
GroupLike.val_inv
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
(a : GroupLike R A)
:
instance
GroupLike.instGroup
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[Semiring A]
[HopfAlgebra R A]
:
Equations
- One or more equations did not get rendered due to their size.
instance
GroupLike.instCommGroup
{R : Type u_1}
{A : Type u_2}
[CommSemiring R]
[CommSemiring A]
[HopfAlgebra R A]
:
Equations
- One or more equations did not get rendered due to their size.