Extensions of Lie algebras #
This file defines extensions of Lie algebras, given by short exact sequences of Lie algebra
homomorphisms. They are implemented in two ways: IsExtension
is a Prop
-valued class taking two
homomorphisms as parameters, and Extension
is a structure that includes the middle Lie algebra.
Main definitions #
LieAlgebra.IsExtension
: AProp
-valued class characterizing an extension of Lie algebras.LieAlgebra.Extension
: A bundled structure giving an extension of Lie algebras.LieAlgebra.IsExtension.extension
: A function that builds the bundled structure from the class.
TODO #
IsCentral
- central extensionsEquiv
- equivalence of extensionsofTwoCocycle
- construction of extensions from 2-cocycles
References #
A sequence of two Lie algebra homomorphisms is an extension if it is short exact.
- exact : i.range = LieIdeal.toLieSubalgebra R L p.ker
Instances
The type of all Lie extensions of M
by N
. That is, short exact sequences of R
-Lie algebra
homomorphisms 0 → N → L → M → 0
where R
, M
, and N
are fixed.
- L : Type u_5
The middle object in the sequence.
- instLieRing : LieRing self.L
L
is a Lie ring. - instLieAlgebra : LieAlgebra R self.L
L
is a Lie algebra overR
. The inclusion homomorphism
N →ₗ⁅R⁆ L
The projection homomorphism
L →ₗ⁅R⁆ M
- IsExtension : LieAlgebra.IsExtension self.incl self.proj
Instances For
The bundled LieAlgebra.Extension
corresponding to LieAlgebra.IsExtension
Equations
- h.extension = { L := L, instLieRing := inst✝⁵, instLieAlgebra := inst✝⁴, incl := i, proj := p, IsExtension := h }
Instances For
A surjective Lie algebra homomorphism yields an extension.