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.
Because our sign convention for differentials is opposite that of Chevalley-Eilenberg, there is a change of signs in the "action" part of the Lie bracket.
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.LieAlgebra.ofTwoCocycle: The Lie algebra built from a direct product, but whose bracket product is sheared by a 2-cocycle.LieAlgebra.Extension.ofTwoCocycle- The Lie algebra extension constructed from a 2-cocycle.
TODO #
IsCentral- central extensionsEquiv- equivalence of extensions- The 2-cocycle given by a linear splitting of an extension.
- The 2-coboundary from two linear splittings of an extension.
References #
A sequence of two Lie algebra homomorphisms is an extension if it is short exact.
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.
Lis a Lie ring.- instLieAlgebra : LieAlgebra R self.L
Lis a Lie algebra overR. The inclusion homomorphism
N →ₗ⁅R⁆ LThe projection homomorphism
L →ₗ⁅R⁆ M- IsExtension : LieAlgebra.IsExtension self.incl self.proj
Instances For
The bundled LieAlgebra.Extension corresponding to LieAlgebra.IsExtension
Equations
Instances For
A surjective Lie algebra homomorphism yields an extension.
A one-field structure giving a type synonym for a direct product. We use this to describe an alternative Lie algebra structure on the product, where the bracket is shifted by a 2-cocycle.
The underlying type.
Instances For
An equivalence between the direct product and the corresponding one-field structure. This is used to transfer the additive and scalar-multiple structure on the direct product to the type synonym.
Equations
- LieAlgebra.ofProd c = { toFun := fun (a : L × M) => { carrier := a }, invFun := fun (a : LieAlgebra.ofTwoCocycle c) => a.carrier, left_inv := ⋯, right_inv := ⋯ }
Instances For
Equations
Equations
Equations
- One or more equations did not get rendered due to their size.
Equations
- LieAlgebra.instOfTwoCocycle c = { toModule := LieAlgebra.instModuleOfTwoCocycle c, lie_smul := ⋯ }
The extension of Lie algebras defined by a 2-cocycle.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The Lie algebra isomorphism given by the type synonym.