Documentation

Mathlib.FieldTheory.AbelRuffini

The Abel-Ruffini Theorem #

This file proves one direction of the Abel-Ruffini theorem, namely that if an element is solvable by radicals, then its minimal polynomial has solvable Galois group.

Main definitions #

Main results #

theorem gal_C_isSolvable {F : Type u_1} [Field F] (x : F) :
theorem gal_mul_isSolvable {F : Type u_1} [Field F] {p q : Polynomial F} :
theorem gal_prod_isSolvable {F : Type u_1} [Field F] {s : Multiset (Polynomial F)} (hs : ps, IsSolvable p.Gal) :
theorem splits_X_pow_sub_one_of_X_pow_sub_C {F : Type u_3} [Field F] {E : Type u_4} [Field E] (i : F →+* E) (n : ) {a : F} (ha : a 0) (h : Polynomial.Splits i (Polynomial.X ^ n - Polynomial.C a)) :
inductive IsSolvableByRad (F : Type u_1) [Field F] {E : Type u_2} [Field E] [Algebra F E] :
EProp

Inductive definition of solvable by radicals

def solvableByRad (F : Type u_1) [Field F] (E : Type u_2) [Field E] [Algebra F E] :

The intermediate field of solvable-by-radicals elements

Equations
  • solvableByRad F E = { carrier := IsSolvableByRad F, mul_mem' := , one_mem' := , add_mem' := , zero_mem' := , algebraMap_mem' := , inv_mem' := }
theorem solvableByRad.induction {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (P : (solvableByRad F E)Prop) (base : ∀ (α : F), P ((algebraMap F (solvableByRad F E)) α)) (add : ∀ (α β : (solvableByRad F E)), P αP βP (α + β)) (neg : ∀ (α : (solvableByRad F E)), P αP (-α)) (mul : ∀ (α β : (solvableByRad F E)), P αP βP (α * β)) (inv : ∀ (α : (solvableByRad F E)), P αP α⁻¹) (rad : ∀ (α : (solvableByRad F E)) (n : ), n 0P (α ^ n)P α) (α : (solvableByRad F E)) :
P α
theorem solvableByRad.isIntegral {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (α : (solvableByRad F E)) :
def solvableByRad.P {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (α : (solvableByRad F E)) :

The statement to be proved inductively

Equations
theorem solvableByRad.induction3 {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] {α : (solvableByRad F E)} {n : } (hn : n 0) ( : P (α ^ n)) :
P α

An auxiliary induction lemma, which is generalized by solvableByRad.isSolvable.

theorem solvableByRad.induction2 {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] {α β γ : (solvableByRad F E)} ( : γ Fα, β) ( : P α) ( : P β) :
P γ

An auxiliary induction lemma, which is generalized by solvableByRad.isSolvable.

theorem solvableByRad.induction1 {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] {α β : (solvableByRad F E)} ( : β Fα) ( : P α) :
P β

An auxiliary induction lemma, which is generalized by solvableByRad.isSolvable.

theorem solvableByRad.isSolvable {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] (α : (solvableByRad F E)) :
theorem solvableByRad.isSolvable' {F : Type u_1} [Field F] {E : Type u_2} [Field E] [Algebra F E] {α : E} {q : Polynomial F} (q_irred : Irreducible q) (q_aeval : (Polynomial.aeval α) q = 0) ( : IsSolvableByRad F α) :

Abel-Ruffini Theorem (one direction): An irreducible polynomial with an IsSolvableByRad root has solvable Galois group