Documentation

Mathlib.Algebra.Lie.Derivation.Killing

Derivations of finite dimensional Killing Lie algebras #

This file establishes that all derivations of finite-dimensional Killing Lie algebras are inner.

Main statements #

noncomputable def LieDerivation.IsKilling.rangeAdOrthogonal (R : Type u_1) (L : Type u_2) [Field R] [LieRing L] [LieAlgebra R L] :

The orthogonal complement of the inner derivations is a Lie submodule of all derivations.

Equations
Instances For
    @[simp]
    theorem LieDerivation.IsKilling.rangeAdOrthogonal_carrier (R : Type u_1) (L : Type u_2) [Field R] [LieRing L] [LieAlgebra R L] :
    (rangeAdOrthogonal R L) = {m : LieDerivation R L L | ∀ (a : L), (killingForm R (LieDerivation R L L)).IsOrtho ((ad R L) a) m}

    If a derivation D is in the Killing orthogonal of the range of the adjoint action, then, for any x : L, ad (D x) is also in this orthogonal.

    @[simp]
    theorem LieDerivation.IsKilling.ad_apply_eq_zero_iff (R : Type u_1) (L : Type u_2) [Field R] [LieRing L] [LieAlgebra R L] [Module.Finite R L] [LieAlgebra.IsKilling R L] (x : L) :
    (ad R L) x = 0 x = 0

    The restriction of the Killing form of a finite-dimensional Killing Lie algebra to the range of the adjoint action is nondegenerate.

    @[simp]

    The range of the adjoint action on a finite-dimensional Killing Lie algebra is full.

    theorem LieDerivation.IsKilling.exists_eq_ad {R : Type u_1} {L : Type u_2} [Field R] [LieRing L] [LieAlgebra R L] [Module.Finite R L] [LieAlgebra.IsKilling R L] (D : LieDerivation R L L) :
    ∃ (x : L), (ad R L) x = D

    Every derivation of a finite-dimensional Killing Lie algebra is an inner derivation.