Skip to content

Commit

Permalink
chore(algebra/lie): adjoint rep of lie algebra uses lowercase ad (#…
Browse files Browse the repository at this point in the history
…4891)

The uppercase is for Lie groups




Co-authored-by: Oliver Nash <oliver.nash@gmail.com>
  • Loading branch information
jcommelin and Oliver Nash committed Nov 3, 2020
1 parent e88a5bb commit 712a0b7
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/algebra/lie/basic.lean
Expand Up @@ -357,7 +357,7 @@ lemma endo_algebra_bracket (M : Type v) [add_comm_group M] [module R M] (f g : m
⁅f, g⁆ = f.comp g - g.comp f := rfl

/-- The adjoint action of a Lie algebra on itself. -/
def Ad : L →ₗ⁅R⁆ module.End R L :=
def ad : L →ₗ⁅R⁆ module.End R L :=
{ to_fun := λ x,
{ to_fun := has_bracket.bracket x,
map_add' := by { intros, apply lie_add, },
Expand Down Expand Up @@ -556,7 +556,7 @@ def lie_module.of_endo_morphism (α : L →ₗ⁅R⁆ module.End R M) : lie_modu

/-- Every Lie algebra is a module over itself. -/
instance lie_algebra_self_module : lie_module R L L :=
lie_module.of_endo_morphism R L L lie_algebra.Ad
lie_module.of_endo_morphism R L L lie_algebra.ad

/-- A Lie submodule of a Lie module is a submodule that is closed under the Lie bracket.
This is a sufficient condition for the subset itself to form a Lie module. -/
Expand Down

0 comments on commit 712a0b7

Please sign in to comment.