Skip to content

Commit ec3b006

Browse files
committed
chore(Algebra/Lie/Solvable): add instance IsSolvable R A for LieIdeal R L (#20395)
1 parent 0b74e84 commit ec3b006

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

Mathlib/Algebra/Lie/Solvable.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -229,6 +229,9 @@ theorem Injective.lieAlgebra_isSolvable [h₁ : IsSolvable R L] (h₂ : Injectiv
229229
apply LieIdeal.bot_of_map_eq_bot h₂; rw [eq_bot_iff, ← hk]
230230
apply LieIdeal.derivedSeries_map_le
231231

232+
instance (A : LieIdeal R L) [IsSolvable R L] : IsSolvable R A :=
233+
A.incl_injective.lieAlgebra_isSolvable
234+
232235
theorem Surjective.lieAlgebra_isSolvable [h₁ : IsSolvable R L'] (h₂ : Surjective f) :
233236
IsSolvable R L := by
234237
obtain ⟨k, hk⟩ := id h₁
@@ -238,7 +241,7 @@ theorem Surjective.lieAlgebra_isSolvable [h₁ : IsSolvable R L'] (h₂ : Surjec
238241

239242
end Function
240243

241-
theorem LieHom.isSolvable_range (f : L' →ₗ⁅R⁆ L) [LieAlgebra.IsSolvable R L'] :
244+
instance LieHom.isSolvable_range (f : L' →ₗ⁅R⁆ L) [LieAlgebra.IsSolvable R L'] :
242245
LieAlgebra.IsSolvable R f.range :=
243246
f.surjective_rangeRestrict.lieAlgebra_isSolvable
244247

0 commit comments

Comments
 (0)