mathlib3 documentation

algebra.lie.abelian

Trivial Lie modules and Abelian Lie algebras #

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

The action of a Lie algebra L on a module M is trivial if ⁅x, m⁆ = 0 for all x ∈ L and m ∈ M. In the special case that M = L with the adjoint action, triviality corresponds to the concept of an Abelian Lie algebra.

In this file we define these concepts and provide some related definitions and results.

Main definitions #

Tags #

lie algebra, abelian, commutative, center

@[class]
structure lie_module.is_trivial (L : Type v) (M : Type w) [has_bracket L M] [has_zero M] :
Prop

A Lie (ring) module is trivial iff all brackets vanish.

Instances of this typeclass
@[simp]
theorem trivial_lie_zero (L : Type v) (M : Type w) [has_bracket L M] [has_zero M] [lie_module.is_trivial L M] (x : L) (m : M) :
x, m = 0
@[reducible]
def is_lie_abelian (L : Type v) [has_bracket L L] [has_zero L] :
Prop

A Lie algebra is Abelian iff it is trivial as a Lie module over itself.

@[protected, instance]
theorem function.injective.is_lie_abelian {R : Type u} {L₁ : Type v} {L₂ : Type w} [comm_ring R] [lie_ring L₁] [lie_ring L₂] [lie_algebra R L₁] [lie_algebra R L₂] {f : L₁ →ₗ⁅R L₂} (h₁ : function.injective f) (h₂ : is_lie_abelian L₂) :
theorem function.surjective.is_lie_abelian {R : Type u} {L₁ : Type v} {L₂ : Type w} [comm_ring R] [lie_ring L₁] [lie_ring L₂] [lie_algebra R L₁] [lie_algebra R L₂] {f : L₁ →ₗ⁅R L₂} (h₁ : function.surjective f) (h₂ : is_lie_abelian L₁) :
theorem lie_abelian_iff_equiv_lie_abelian {R : Type u} {L₁ : Type v} {L₂ : Type w} [comm_ring R] [lie_ring L₁] [lie_ring L₂] [lie_algebra R L₁] [lie_algebra R L₂] (e : L₁ ≃ₗ⁅R L₂) :
@[protected]
def lie_module.ker (R : Type u) (L : Type v) (M : Type w) [comm_ring R] [lie_ring L] [lie_algebra R L] [add_comm_group M] [module R M] [lie_ring_module L M] [lie_module R L M] :

The kernel of the action of a Lie algebra L on a Lie module M as a Lie ideal in L.

Equations
@[protected, simp]
theorem lie_module.mem_ker (R : Type u) (L : Type v) (M : Type w) [comm_ring R] [lie_ring L] [lie_algebra R L] [add_comm_group M] [module R M] [lie_ring_module L M] [lie_module R L M] (x : L) :
x lie_module.ker R L M (m : M), x, m = 0
def lie_module.max_triv_submodule (R : Type u) (L : Type v) (M : Type w) [comm_ring R] [lie_ring L] [lie_algebra R L] [add_comm_group M] [module R M] [lie_ring_module L M] [lie_module R L M] :

The largest submodule of a Lie module M on which the Lie algebra L acts trivially.

Equations
Instances for lie_module.max_triv_submodule
@[simp]
theorem lie_module.mem_max_triv_submodule (R : Type u) (L : Type v) (M : Type w) [comm_ring R] [lie_ring L] [lie_algebra R L] [add_comm_group M] [module R M] [lie_ring_module L M] [lie_module R L M] (m : M) :

max_triv_submodule is functorial.

Equations
@[simp, norm_cast]
theorem lie_module.coe_max_triv_hom_apply {R : Type u} {L : Type v} {M : Type w} {N : Type w₁} [comm_ring R] [lie_ring L] [lie_algebra R L] [add_comm_group M] [module R M] [lie_ring_module L M] [lie_module R L M] [add_comm_group N] [module R N] [lie_ring_module L N] [lie_module R L N] (f : M →ₗ⁅R,L N) (m : (lie_module.max_triv_submodule R L M)) :

The maximal trivial submodules of Lie-equivalent Lie modules are Lie-equivalent.

Equations
@[simp, norm_cast]

A linear map between two Lie modules is a morphism of Lie modules iff the Lie algebra action on it is trivial.

Equations
@[reducible]
def lie_algebra.center (R : Type u) (L : Type v) [comm_ring R] [lie_ring L] [lie_algebra R L] :

The center of a Lie algebra is the set of elements that commute with everything. It can be viewed as the maximal trivial submodule of the Lie algebra as a Lie module over itself via the adjoint representation.

@[protected, instance]
@[simp]
theorem lie_submodule.trivial_lie_oper_zero {R : Type u} {L : Type v} {M : Type w} [comm_ring R] [lie_ring L] [lie_algebra R L] [add_comm_group M] [module R M] [lie_ring_module L M] [lie_module R L M] (N : lie_submodule R L M) (I : lie_ideal R L) [lie_module.is_trivial L M] :