Skip to content

Commit

Permalink
chore(lie/semisimple): tweak `lie_algebra.subsingleton_of_semisimple_…
Browse files Browse the repository at this point in the history
…lie_abelian` (#8728)
  • Loading branch information
ocfnash committed Aug 17, 2021
1 parent 31d5549 commit e6e5718
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/algebra/lie/semisimple.lean
Expand Up @@ -84,12 +84,12 @@ begin
exact h₂ hI,
end

-- TODO[gh-6025]: make this an instance once safe to do so
/-- A semisimple Abelian Lie algebra is trivial. -/
lemma subsingleton_of_semisimple_lie_abelian [is_semisimple R L] [h : is_lie_abelian L] :
subsingleton (lie_ideal R L) :=
subsingleton L :=
begin
apply subsingleton_of_bot_eq_top,
rwa [is_lie_abelian_iff_center_eq_top R L, center_eq_bot_of_semisimple] at h,
rw [is_lie_abelian_iff_center_eq_top R L, center_eq_bot_of_semisimple] at h,
exact (lie_submodule.subsingleton_iff R L L).mp (subsingleton_of_bot_eq_top h),
end

lemma abelian_radical_of_semisimple [is_semisimple R L] : is_lie_abelian (radical R L) :=
Expand Down

0 comments on commit e6e5718

Please sign in to comment.