Weights and roots of Lie modules and Lie algebras #
Just as a key tool when studying the behaviour of a linear operator is to decompose the space on
which it acts into a sum of (generalised) eigenspaces, a key tool when studying a representation M
of Lie algebra L
is to decompose M
into a sum of simultaneous eigenspaces of x
as x
ranges
over L
. These simultaneous generalised eigenspaces are known as the weight spaces of M
.
When L
is nilpotent, it follows from the binomial theorem that weight spaces are Lie submodules.
Even when L
is not nilpotent, it may be useful to study its representations by restricting them
to a nilpotent subalgebra (e.g., a Cartan subalgebra). In the particular case when we view L
as a
module over itself via the adjoint action, the weight spaces of L
restricted to a nilpotent
subalgebra are known as root spaces.
Basic definitions and properties of the above ideas are provided in this file.
Main definitions #
LieModule.weightSpaceOf
LieModule.weightSpace
LieModule.IsWeight
LieAlgebra.rootSpace
LieAlgebra.IsRoot
LieAlgebra.rootSpaceWeightSpaceProduct
LieAlgebra.rootSpaceProduct
LieAlgebra.zeroRootSubalgebra_eq_iff_is_cartan
References #
Tags #
lie character, eigenvalue, eigenspace, weight, weight vector, root, root vector
See also bourbaki1975b
Chapter VII §1.1, Proposition 2 (ii).
If M
is a representation of a nilpotent Lie algebra L
, χ
is a scalar, and x : L
, then
weightSpaceOf M χ x
is the maximal generalized χ
-eigenspace of the action of x
on M
.
It is a Lie submodule because L
is nilpotent.
Instances For
If M
is a representation of a nilpotent Lie algebra L
and χ : L → R
is a family of
scalars, then weightSpace M χ
is the intersection of the maximal generalized χ x
-eigenspaces of
the action of x
on M
as x
ranges over L
.
It is a Lie submodule because L
is nilpotent.
Instances For
See also the more useful form LieModule.zero_weightSpace_eq_top_of_nilpotent
.
Given a Lie module M
of a Lie algebra L
, a weight of M
with respect to a nilpotent
subalgebra H ⊆ L
is a Lie character whose corresponding weight space is non-empty.
Instances For
For a non-trivial nilpotent Lie module over a nilpotent Lie algebra, the zero character is a
weight with respect to the ⊤
Lie subalgebra.
A (nilpotent) Lie algebra acts nilpotently on the zero weight space of a Noetherian Lie module.
By Engel's theorem, the zero weight space of a Noetherian Lie module is nilpotent.
Given a nilpotent Lie subalgebra H ⊆ L
, the root space of a map χ : H → R
is the weight
space of L
regarded as a module of H
via the adjoint action.
Instances For
A root of a Lie algebra L
with respect to a nilpotent subalgebra H ⊆ L
is a weight of L
,
regarded as a module of H
via the adjoint action.
Instances For
Auxiliary definition for rootSpaceWeightSpaceProduct
,
which is close to the deterministic timeout limit.
Instances For
Given a nilpotent Lie subalgebra H ⊆ L
together with χ₁ χ₂ : H → R
, there is a natural
R
-bilinear product of root vectors and weight vectors, compatible with the actions of H
.
Instances For
Given a nilpotent Lie subalgebra H ⊆ L
together with χ₁ χ₂ : H → R
, there is a natural
R
-bilinear product of root vectors, compatible with the actions of H
.
Instances For
Given a nilpotent Lie subalgebra H ⊆ L
, the root space of the zero map 0 : H → R
is a Lie
subalgebra of L
.
Instances For
If the zero root subalgebra of a nilpotent Lie subalgebra H
is just H
then H
is a Cartan
subalgebra.
When L
is Noetherian, it follows from Engel's theorem that the converse holds. See
LieAlgebra.zeroRootSubalgebra_eq_iff_is_cartan