Documentation

Mathlib.RepresentationTheory.Tannaka

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 #

https://math.leidenuniv.nl/scripties/1bachCommelin.pdf

@[simp]
theorem TannakaDuality.FiniteGroup.forget_obj {k G : Type u} [CommRing k] [Group G] (X : FDRep k G) :
(forget k G).obj X = X.V
@[simp]
theorem TannakaDuality.FiniteGroup.forget_map {k G : Type u} [CommRing k] [Group G] (X Y : FDRep k G) (f : X Y) :
(forget k G).map f = f.hom
def TannakaDuality.FiniteGroup.equivApp {k G : Type u} [CommRing k] [Group G] (g : G) (X : FDRep k G) :
X.V X.V

Definition of equivHom g : Aut (forget k G) by its components.

Equations
Instances For
    @[simp]
    theorem TannakaDuality.FiniteGroup.equivApp_hom {k G : Type u} [CommRing k] [Group G] (g : G) (X : FDRep k G) :
    @[simp]
    theorem TannakaDuality.FiniteGroup.equivApp_inv {k G : Type u} [CommRing k] [Group G] (g : G) (X : FDRep k G) :

    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
      Instances For
        @[simp]
        theorem TannakaDuality.FiniteGroup.rightRegular_apply {k G : Type u} [CommRing k] [Group G] (s t : G) (f : Gk) :
        (rightRegular s) f t = f (t * s)

        The representation on G → k induced by multiplication on the left in G.

        Equations
        Instances For
          @[simp]
          theorem TannakaDuality.FiniteGroup.leftRegular_apply {k G : Type u} [CommRing k] [Group G] (s t : G) (f : Gk) :
          (leftRegular s) f t = f (s⁻¹ * t)

          The right regular representation rightRegular on G → k as a FDRep k G.

          Equations
          Instances For

            The FDRep k G morphism induced by multiplication on G → k.

            Equations
            Instances For
              theorem TannakaDuality.FiniteGroup.map_mul_toRightFDRepComp {k G : Type u} [CommRing k] [Group G] [Fintype G] (η : CategoryTheory.Aut (forget k G)) (f g : Gk) :
              let α := ModuleCat.Hom.hom (η.hom.hom.app rightFDRep); α (f * g) = α f * α g

              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).

              Equations
              Instances For