File tree Expand file tree Collapse file tree 1 file changed +4
-1
lines changed Expand file tree Collapse file tree 1 file changed +4
-1
lines changed Original file line number Diff line number Diff line change @@ -229,6 +229,9 @@ theorem Injective.lieAlgebra_isSolvable [h₁ : IsSolvable R L] (h₂ : Injectiv
229
229
apply LieIdeal.bot_of_map_eq_bot h₂; rw [eq_bot_iff, ← hk]
230
230
apply LieIdeal.derivedSeries_map_le
231
231
232
+ instance (A : LieIdeal R L) [IsSolvable R L] : IsSolvable R A :=
233
+ A.incl_injective.lieAlgebra_isSolvable
234
+
232
235
theorem Surjective.lieAlgebra_isSolvable [h₁ : IsSolvable R L'] (h₂ : Surjective f) :
233
236
IsSolvable R L := by
234
237
obtain ⟨k, hk⟩ := id h₁
@@ -238,7 +241,7 @@ theorem Surjective.lieAlgebra_isSolvable [h₁ : IsSolvable R L'] (h₂ : Surjec
238
241
239
242
end Function
240
243
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'] :
242
245
LieAlgebra.IsSolvable R f.range :=
243
246
f.surjective_rangeRestrict.lieAlgebra_isSolvable
244
247
You can’t perform that action at this time.
0 commit comments