Documentation

Mathlib.Algebra.Lie.CartanSubalgebra

Cartan subalgebras #

Cartan subalgebras are one of the most important concepts in Lie theory. We define them here. The standard example is the set of diagonal matrices in the Lie algebra of matrices.

Main definitions #

Tags #

lie subalgebra, normalizer, idealizer, cartan subalgebra

def LieSubmodule.IsUcsLimit {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] {M : Type u_1} [AddCommGroup M] [Module R M] [LieRingModule L M] [LieModule R L M] (N : LieSubmodule R L M) :

Given a Lie module M of a Lie algebra L, LieSubmodule.IsUcsLimit is the proposition that a Lie submodule N ⊆ M is the limiting value for the upper central series.

This is a characteristic property of Cartan subalgebras with the roles of L, M, N played by H, L, H, respectively. See LieSubalgebra.isCartanSubalgebra_iff_isUcsLimit.

Equations
Instances For

    A Cartan subalgebra is a nilpotent, self-normalizing subalgebra.

    A splitting Cartan subalgebra can be defined by mixing in LieModule.IsTriangularizable R H L.

    Instances
      theorem LieSubalgebra.IsCartanSubalgebra.nilpotent {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] {H : LieSubalgebra R L} [self : H.IsCartanSubalgebra] :
      theorem LieSubalgebra.IsCartanSubalgebra.self_normalizing {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] {H : LieSubalgebra R L} [self : H.IsCartanSubalgebra] :
      H.normalizer = H
      instance LieSubalgebra.instIsNilpotentSubtypeMemOfIsCartanSubalgebra {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] (H : LieSubalgebra R L) [H.IsCartanSubalgebra] :
      Equations
      • =
      @[simp]
      theorem LieSubalgebra.normalizer_eq_self_of_isCartanSubalgebra {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] (H : LieSubalgebra R L) [H.IsCartanSubalgebra] :
      H.toLieSubmodule.normalizer = H.toLieSubmodule
      @[simp]
      theorem LieSubalgebra.ucs_eq_self_of_isCartanSubalgebra {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] (H : LieSubalgebra R L) [H.IsCartanSubalgebra] (k : ) :
      LieSubmodule.ucs k H.toLieSubmodule = H.toLieSubmodule
      theorem LieSubalgebra.isCartanSubalgebra_iff_isUcsLimit {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] (H : LieSubalgebra R L) :
      H.IsCartanSubalgebra H.toLieSubmodule.IsUcsLimit
      @[simp]
      theorem LieIdeal.normalizer_eq_top {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] (I : LieIdeal R L) :
      (lieIdealSubalgebra R L I).normalizer =
      instance LieAlgebra.top_isCartanSubalgebra_of_nilpotent {R : Type u} {L : Type v} [CommRing R] [LieRing L] [LieAlgebra R L] [LieAlgebra.IsNilpotent R L] :
      .IsCartanSubalgebra

      A nilpotent Lie algebra is its own Cartan subalgebra.

      Equations
      • =