Construction of an algebraic number that is not solvable by radicals. #
The main ingredients are:
solvableByRad.isSolvable'
inMathlib/FieldTheory/AbelRuffini.lean
: an irreducible polynomial with anIsSolvableByRad
root has solvable Galois groupgalActionHom_bijective_of_prime_degree'
inMathlib/FieldTheory/PolynomialGaloisGroup.lean
: an irreducible polynomial of prime degree with 1-3 non-real roots has full Galois groupEquiv.Perm.not_solvable
inMathlib/GroupTheory/Solvable.lean
: the symmetric group is not solvable
Then all that remains is the construction of a specific polynomial satisfying the conditions of
galActionHom_bijective_of_prime_degree'
, which is done in this file.
A quintic polynomial that we will show is irreducible
Equations
- AbelRuffini.Φ R a b = Polynomial.X ^ 5 - Polynomial.C ↑a * Polynomial.X + Polynomial.C ↑b
Instances For
theorem
AbelRuffini.real_roots_Phi_ge
(a b : ℕ)
(hab : b < a)
:
2 ≤ Fintype.card ↑((Φ ℚ a b).rootSet ℝ)
theorem
AbelRuffini.complex_roots_Phi
(a b : ℕ)
(h : (Φ ℚ a b).Separable)
:
Fintype.card ↑((Φ ℚ a b).rootSet ℂ) = 5
theorem
AbelRuffini.gal_Phi
(a b : ℕ)
(hab : b < a)
(h_irred : Irreducible (Φ ℚ a b))
:
Function.Bijective ⇑(Polynomial.Gal.galActionHom (Φ ℚ a b) ℂ)
Abel-Ruffini Theorem