Tannaka duality for finite groups #
In this file we prove Tannaka duality for finite groups.
The theorem can be formulated as follows: for any integral domain k
, a finite group G
can be
recovered from FDRep k G
, the monoidal category of finite dimensional k
-linear representations
of G
, and the monoidal forgetful functor forget : FDRep k G ⥤ FGModuleCat k
.
More specifically, the main result is the isomorphism equiv : G ≃* Aut (forget k G)
.
Reference #
The monoidal forgetful functor from FDRep k G
to FGModuleCat k
.
Equations
Instances For
Definition of equivHom g : Aut (forget k G)
by its components.
Equations
- TannakaDuality.FiniteGroup.equivApp g X = { hom := ModuleCat.ofHom (X.ρ g), inv := ModuleCat.ofHom (X.ρ g⁻¹), hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
The group homomorphism G →* Aut (forget k G)
shown to be an isomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The representation on G → k
induced by multiplication on the right in G
.
Equations
- TannakaDuality.FiniteGroup.rightRegular = { toFun := fun (s : G) => { toFun := fun (f : G → k) (t : G) => f (t * s), map_add' := ⋯, map_smul' := ⋯ }, map_one' := ⋯, map_mul' := ⋯ }
Instances For
The representation on G → k
induced by multiplication on the left in G
.
Equations
- TannakaDuality.FiniteGroup.leftRegular = { toFun := fun (s : G) => { toFun := fun (f : G → k) (t : G) => f (s⁻¹ * t), map_add' := ⋯, map_smul' := ⋯ }, map_one' := ⋯, map_mul' := ⋯ }
Instances For
The right regular representation rightRegular
on G → k
as a FDRep k G
.
Instances For
The FDRep k G
morphism induced by multiplication on G → k
.
Equations
- TannakaDuality.FiniteGroup.mulRepHom = { hom := ModuleCat.ofHom (LinearMap.mul' k (G → k)), comm := ⋯ }
Instances For
The rightFDRep
component of η : Aut (forget k G)
preserves multiplication
The rightFDRep
component of η : Aut (forget k G)
gives rise to
an algebra morphism (G → k) →ₐ[k] (G → k)
.