Documentation

MyProject.Addenda_monoid_algebra_theory

Addenda to the monoid algebra theory in mathlib #

This file adds some properties about monoid algebra theory in mathlib.

Main results #

The goal of this file is to add to the monoid algebra theory some preliminary results to construct the character on the induced representation by the center of a finite group. The main theorem proved here is the decomposition of MonoidAlgebra k G as a direct sum of g • MonoidAlgebra k (Subgroup.center G) indexed by elements of a system of representatives of G⧸ (Subgroup.center G) as defined in system_of_repr_center.set.

Contents #

instance Finite_H (G : Type) [inst2 : Group G] [inst3 : Finite G] (H : Subgroup G) :
Finite H
noncomputable instance Fintype_G (G : Type) [inst3 : Finite G] :
Equations
noncomputable def Map_kHkG (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) :

The trivial map from MonoidAlgebra k H to MonoidAlgebra k G, ie elements from MonoidAlgebra k H are seen as MonoidAlgebra k G.

Equations
Instances For
    @[simp]
    theorem Map_kHkG_single_apply (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) (h : H) (c : k) :
    @[simp]
    theorem Map_kHkG_k_linear (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) (c : k) (x : MonoidAlgebra k H) :
    (Map_kHkG k G H) (c x) = c (Map_kHkG k G H) x

    Map_kHkG is indeed a k linear map.

    noncomputable instance Coe_kH_kG (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) :

    Coercion from MonoidAlgebra k H to MonoidAlgebra k G when H is a subgroup of G

    Equations
    noncomputable instance Smul_kHkG (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) :

    Scalar multiplication between MonoidAlgebra k H and MonoidAlgebra k G, ie classical mulitplication between an element of MonoidAlgebra k H seen as an element of MonoidAlgebra k G and an element of MonoidAlgebra k G.

    Equations
    noncomputable instance kG_is_kCenter_Algebra (k G : Type) [inst1 : Field k] [inst2 : Group G] :

    MonoidAlgebra k G is a MonoidAlgebra k (Subgroup.center G) algebra.

    Equations
    noncomputable instance kG_is_kH_Algebra (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) [instH : IsMulCommutative H] (ϕ : H →* (Subgroup.center G)) :

    If we have a homomorphism H →* Subgroup.center G, then we have Algebra (MonoidAlgebra k H) (MonoidAlgebra k G).

    Equations
    @[simp]
    theorem center_commutes_single (k G : Type) [inst1 : Field k] [inst2 : Group G] (x : MonoidAlgebra k (Subgroup.center G)) (g : G) :

    For every g : G, x : MonoidAlgebra k (Subgroup.center G) commutes with MonoidAlgebra.single g (1:k).

    noncomputable instance Set_Coe (k G : Type) [inst1 : Field k] [inst2 : Group G] (H : Subgroup G) :

    Coercion from Set (MonoidAlgebra k H) to (Set (MonoidAlgebra k G)).

    Equations
    noncomputable def center_sub_module (k G : Type) [inst1 : Field k] [inst2 : Group G] :

    (MonoidAlgebra k (Subgroup.center G)) seen as a subset of MonoidAlgebra k G is a (MonoidAlgebra k (Subgroup.center G)) submodule of (MonoidAlgebra k (Subgroup.center G)).

    Equations
    Instances For
      noncomputable instance hmul_g_kH_kG (k G : Type) [inst1 : Field k] [inst2 : Group G] :

      We define the multiplication of an element g : G by kH : MonoidAlgebra k (Subgroup.center G) by MonoidAlgebra.single g (1:k) * kH.

      Equations
      noncomputable instance hmul_g_kG (k G : Type) [inst1 : Field k] [inst2 : Group G] :

      We define the multiplication of an element g: G by kG : MonoidAlgebra k G by MonoidAlgebra.single g (1:k) * kG.

      Equations
      theorem hmul_g_kH_kG_simp (k G : Type) [inst1 : Field k] [inst2 : Group G] (g : G) (kH : MonoidAlgebra k (Subgroup.center G)) :
      noncomputable def gkH_map (k G : Type) [inst1 : Field k] [inst2 : Group G] (g : G) :

      Let g : G. We define a k linear map on MonoidAlgebra k (Subgroup.center G) by x ↦ g*x

      Equations
      Instances For
        @[simp]
        theorem gkH_map_eq (k G : Type) [inst1 : Field k] [inst2 : Group G] (g : G) (x : MonoidAlgebra k (Subgroup.center G)) :
        (gkH_map k G g) x = g * x

        For every x : MonoidAlgebra k (Subgroup.center G), we have gkH_map k G g x = g * x.

        noncomputable def gkH_set (k G : Type) [inst1 : Field k] [inst2 : Group G] (g : G) :

        The set of the image of gKh_map k G g, or in an equivalent manner the set of elements g*MonoidAlgebra k (Subgroup.center G) for g in G.

        Equations
        Instances For
          @[simp]
          theorem gkH_map_gkh_set (k G : Type) [inst1 : Field k] [inst2 : Group G] {g : G} (x : (gkH_set k G g)) :
          (gkH_map k G g) (Exists.choose ) = x

          simp lemma for gkH_map.

          noncomputable def gkH_set_iso_kH_k (k G : Type) [inst1 : Field k] [inst2 : Group G] (g : G) :

          We have a k linear equivalence between MonoidAlgebra k (Subgroup.center G) and gkH_set k G g given by the map gkH_map.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            noncomputable instance gkH_set_SMul (k G : Type) [inst1 : Field k] [inst2 : Group G] {g : G} :
            Equations
            noncomputable instance gkH_set_MulAction (k G : Type) [inst1 : Field k] [inst2 : Group G] {g : G} :
            Equations
            noncomputable instance gkH_set_DistribMulAction (k G : Type) [inst1 : Field k] [inst2 : Group G] {g : G} :
            Equations
            noncomputable instance gkH_set_Module (k G : Type) [inst1 : Field k] [inst2 : Group G] {g : G} :

            gkH_set k G g is a MonoidAlgebra k (Subgroup.center G) module.

            Equations
            noncomputable def gkH_set_iso_kH_module (k G : Type) [inst1 : Field k] [inst2 : Group G] (g : G) :

            We define a MonoidAlgebra k (Subgroup.center G) linear equivalence between gkH_set k G g and MonoidAlgebra k (Subgroup.center G) by $x ↦ g ⬝ x$.

            Equations
            Instances For
              @[simp]
              theorem Map_kHkG_single_simp (k G : Type) [inst1 : Field k] [inst2 : Group G] {x : (Subgroup.center G)} :

              Coercion on the natural basis of MonoidAlgebra k G when g : Subgroup.center G.

              noncomputable def MonoidAlgebra_MulAction_basis (k G : Type) [inst1 : Field k] [inst2 : Group G] [inst3 : Finite G] :

              A system of representatives system_of_repr_center.set G of G⧸ (Subgroup.center G) defines a basis of MonoidAlgebra k G on MonoidAlgebra k (Subgroup.center G).

              Equations
              Instances For
                @[simp]
                theorem MonoidAlgebra_single_basis_simp (k G : Type) [inst1 : Field k] [inst2 : Group G] [inst3 : Finite G] {i : (system_of_repr_center.set G)} (x1 : (system_of_repr_center.set G)) :

                Given a representative x1 : system_of_repr_center G, the coefficients of x1 in the basis MonoidAlgebra_MulAction_basis is 0 unless on the vector x1.

                noncomputable def G_to_direct_sum (k G : Type) [inst1 : Field k] [inst2 : Group G] :

                We define a map between system_of_repr_center.set G and ⨁ (_ : ↑(system_of_repr_center.set G)), MonoidAlgebra k ↥(Subgroup.center G)) given by MonoidAlgebra.single 1 1 on the g-th component and 0 elsewhere.

                Equations
                Instances For

                  We define a MonoidAlgebra k (Subgroup.center G) linear map by extending the map G_to_direct_sum k G which is define on the basis MonoidAlgebra_MulAction_basis k G.

                  Equations
                  Instances For
                    noncomputable def MonoidAlgebra_direct_sum_1 (k G : Type) [inst1 : Field k] [inst2 : Group G] [inst3 : Finite G] :

                    The map MonoidAlgebra_direct_sum_linear k G is in fact a linear bijection.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      noncomputable def MonoidAlgebra_direct_sum_system_of_repr_center_set (k G : Type) [inst1 : Field k] [inst2 : Group G] [inst3 : Finite G] :

                      Given a representative system system_of_repr_center.set G of G⧸ (Subgroup.center G), we have a MonoidAlgebra k (Subgroup.center G) linear bijection between MonoidAlgebra k G and the direct sum of g • (MonoidAlgebra k (Subgroup.center G)) for g : system_of_repr_center.set G.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For