The Lie algebra of a Lie group #
Given a Lie group, we define GroupLieAlgebra I G
as its tangent space at the identity, and we
endow it with a Lie bracket, as follows. Given two vectors v, w : GroupLieAlgebra I G
, consider
the associated left-invariant vector fields mulInvariantVectorField v
(given at a point g
by
the image of v
under the derivative of left-multiplication by g
) and
mulInvariantVectorField w
. Then take their Lie bracket at the identity: this is by definition
the bracket of v
and w
.
Due to general properties of the Lie bracket of vector fields, this gives a Lie algebra structure
on GroupLieAlgebra I G
.
Note that one can also define a Lie algebra on the space of left-invariant derivations on C^∞
functions (see LeftInvariantDerivation.instLieAlgebra
). For finite-dimensional C^∞
real
manifolds, this space of derivations can be canonically identified with the tangent space, and we
recover the same Lie algebra structure (TODO: prove this). In other smoothness classes or on other
fields, this identification is not always true, though, so the derivations point of view does not
work in these settings. Therefore, the point of view in the current file is more general, and
should be favored when possible.
The standing assumption in this file is that the group is C^n
for n = minSmoothness 𝕜 3
, i.e.,
it is C^3
over ℝ
or ℂ
, and analytic otherwise.
The Lie algebra of a Lie group, i.e., its tangent space at the identity. We use the word
GroupLieAlgebra
instead of LieAlgebra
as the latter is taken as a generic class.
Equations
- GroupLieAlgebra I G = TangentSpace I 1
Instances For
The Lie algebra of an additive Lie group, i.e., its tangent space at zero. We use
the word AddGroupLieAlgebra
instead of LieAlgebra
as the latter is taken as a generic class.
Equations
- AddGroupLieAlgebra I G = TangentSpace I 0
Instances For
The invariant vector field associated to a vector v
in the Lie alebra. At a point g
, it
is given by the image of v
under left-multiplication by g
.
Equations
- mulInvariantVectorField v g = (mfderiv I I (fun (x : G) => g * x) 1) v
Instances For
The invariant vector field associated to a vector v
in the Lie alebra. At a
point g
, it is given by the image of v
under left-addition by g
.
Equations
- addInvariantVectorField v g = (mfderiv I I (fun (x : G) => g + x) 0) v
Instances For
The Lie bracket of two vectors v
and w
in the Lie algebra of a Lie group is obtained by
taking the Lie bracket of the associated invariant vector fields, at the identity.
Equations
- instBracketGroupLieAlgebra = { bracket := fun (v w : GroupLieAlgebra I G) => VectorField.mlieBracket I (mulInvariantVectorField v) (mulInvariantVectorField w) 1 }
The Lie bracket of two vectors v
and w
in the Lie algebra of an additive Lie
group is obtained by taking the Lie bracket of the associated invariant vector fields, at zero.
Equations
- instBracketAddGroupLieAlgebra = { bracket := fun (v w : AddGroupLieAlgebra I G) => VectorField.mlieBracket I (addInvariantVectorField v) (addInvariantVectorField w) 0 }
Invariant vector fields are invariant under pullbacks.
Invariant vector fields are invariant under pullbacks.
The invariant vector field associated to the value at the identity of the Lie bracket of two invariant vector fields, is everywhere the Lie bracket of the invariant vector fields.
The invariant vector field associated to the value at zero of the Lie bracket of two invariant vector fields, is everywhere the Lie bracket of the invariant vector fields.
The tangent space at the identity of a Lie group is a Lie ring, for the bracket given by the Lie bracket of invariant vector fields.
Equations
- instLieRingGroupLieAlgebra = { toAddCommGroup := instAddCommGroupTangentSpace I, toBracket := instBracketGroupLieAlgebra, add_lie := ⋯, lie_add := ⋯, lie_self := ⋯, leibniz_lie := ⋯ }
The tangent space at the identity of an additive Lie group is a Lie ring, for the bracket given by the Lie bracket of invariant vector fields.
Equations
- instLieRingAddGroupLieAlgebra = { toAddCommGroup := instAddCommGroupTangentSpace I, toBracket := instBracketAddGroupLieAlgebra, add_lie := ⋯, lie_add := ⋯, lie_self := ⋯, leibniz_lie := ⋯ }
The tangent space at the identity of an additive Lie group is a Lie algebra, for the bracket given by the Lie bracket of invariant vector fields.
Equations
- instLieAlgebraAddGroupLieAlgebra = { toModule := instModuleTangentSpace I, lie_smul := ⋯ }
The tangent space at the identity of a Lie group is a Lie algebra, for the bracket given by the Lie bracket of invariant vector fields.
Equations
- instLieAlgebraGroupLieAlgebra = { toModule := instModuleTangentSpace I, lie_smul := ⋯ }