Documentation

Mathlib.Algebra.Lie.Semisimple.Basic

Semisimple Lie algebras #

The famous Cartan-Dynkin-Killing classification of semisimple Lie algebras renders them one of the most important classes of Lie algebras. In this file we prove basic results abot simple and semisimple Lie algebras.

Main declarations #

Tags #

lie algebra, radical, simple, semisimple

Equations
  • =
theorem LieAlgebra.IsSimple.eq_top_of_isAtom {R : Type u_1} {L : Type u_2} [CommRing R] [LieRing L] [LieAlgebra R L] [LieAlgebra.IsSimple R L] (I : LieIdeal R L) (hI : IsAtom I) :
I =
@[simp]
theorem LieAlgebra.IsSimple.isAtom_iff_eq_top {R : Type u_1} {L : Type u_2} [CommRing R] [LieRing L] [LieAlgebra R L] [LieAlgebra.IsSimple R L] (I : LieIdeal R L) :
@[instance 100]
Equations
  • LieAlgebra.IsSemisimple.instDistribLattice = .distribLattice_of_sSup_eq_top
@[instance 100]
Equations
  • LieAlgebra.IsSemisimple.instBooleanAlgebra = .booleanAlgebra_of_sSup_eq_top
@[instance 100]

A semisimple Lie algebra has trivial radical.

Equations
  • =
@[instance 100]

A simple Lie algebra is semisimple.

Equations
  • =

An abelian Lie algebra with trivial radical is trivial.

The two properties shown to be equivalent here are possible definitions for a Lie algebra to be reductive.

Note that there is absolutely no agreement on what the label 'reductive' should mean when the coefficients are not a field of characteristic zero.