Weights and roots of Lie modules and Lie algebras with respect to Cartan subalgebras #
Given a Lie algebra L
which is not necessarily 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 #
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.
Equations
Instances For
Auxiliary definition for rootSpaceWeightSpaceProduct
,
which is close to the deterministic timeout limit.
Equations
- One or more equations did not get rendered due to their size.
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
.
Equations
- One or more equations did not get rendered due to their size.
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
.
Equations
- LieAlgebra.rootSpaceProduct R L H χ₁ χ₂ χ₃ hχ = LieAlgebra.rootSpaceWeightSpaceProduct R L H L χ₁ χ₂ χ₃ 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
.
Equations
- LieAlgebra.zeroRootSubalgebra R L H = { toSubmodule := ↑(LieAlgebra.rootSpace H 0), lie_mem' := ⋯ }
Instances For
This enables the instance Zero (Weight R H L)
.
Equations
- ⋯ = ⋯
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
Given a root α
relative to a Cartan subalgebra H
, this is the span of all products of
an element of the α
root space and an element of the -α
root space. Informally it is often
denoted ⁅H(α), H(-α)⁆
.
If the Killing form is non-degenerate and the coefficients are a perfect field, this space is
one-dimensional. See LieAlgebra.IsKilling.coe_corootSpace_eq_span_singleton
and
LieAlgebra.IsKilling.coe_corootSpace_eq_span_singleton'
.
Note that the name "coroot space" is not standard as this space does not seem to have a name in the informal literature.
Equations
- LieAlgebra.corootSpace α = (LieModuleHom.codRestrict H.toLieSubmodule ((LieAlgebra.rootSpace H 0).incl.comp (LieAlgebra.rootSpaceProduct R L H α (-α) 0 ⋯)) ⋯).range