mathlib3 documentation

algebra.lie.universal_enveloping

Universal enveloping algebra #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Given a commutative ring R and a Lie algebra L over R, we construct the universal enveloping algebra of L, together with its universal property.

Main definitions #

Tags #

lie algebra, universal enveloping algebra, tensor algebra

inductive universal_enveloping_algebra.rel (R : Type u₁) (L : Type u₂) [comm_ring R] [lie_ring L] [lie_algebra R L] :

The quotient by the ideal generated by this relation is the universal enveloping algebra.

Note that we have avoided using the more natural expression: | lie_compat (x y : L) : rel (ιₜ ⁅x, y⁆) ⁅ιₜ x, ιₜ y⁆ so that our construction needs only the semiring structure of the tensor algebra.

def universal_enveloping_algebra (R : Type u₁) (L : Type u₂) [comm_ring R] [lie_ring L] [lie_algebra R L] :
Type (max u₁ u₂)

The universal enveloping algebra of a Lie algebra.

Equations
Instances for universal_enveloping_algebra
@[protected, instance]
@[protected, instance]
@[protected, instance]

The quotient map from the tensor algebra to the universal enveloping algebra as a morphism of associative algebras.

Equations

The natural Lie algebra morphism from a Lie algebra to its universal enveloping algebra.

Equations
def universal_enveloping_algebra.lift (R : Type u₁) {L : Type u₂} [comm_ring R] [lie_ring L] [lie_algebra R L] {A : Type u₃} [ring A] [algebra R A] :

The universal property of the universal enveloping algebra: Lie algebra morphisms into associative algebras lift to associative algebra morphisms from the universal enveloping algebra.

Equations
@[simp]