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
Instances For
@[simp]
theorem
AbelRuffini.map_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
{S : Type u_2}
[CommRing S]
(f : R →+* S)
:
Polynomial.map f (AbelRuffini.Φ R a b) = AbelRuffini.Φ S a b
@[simp]
theorem
AbelRuffini.coeff_zero_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
:
(AbelRuffini.Φ R a b).coeff 0 = ↑b
@[simp]
theorem
AbelRuffini.coeff_five_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
:
(AbelRuffini.Φ R a b).coeff 5 = 1
theorem
AbelRuffini.degree_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
[Nontrivial R]
:
(AbelRuffini.Φ R a b).degree = ↑5
theorem
AbelRuffini.natDegree_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
[Nontrivial R]
:
(AbelRuffini.Φ R a b).natDegree = 5
theorem
AbelRuffini.leadingCoeff_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
[Nontrivial R]
:
(AbelRuffini.Φ R a b).leadingCoeff = 1
theorem
AbelRuffini.monic_Phi
{R : Type u_1}
[CommRing R]
(a b : ℕ)
[Nontrivial R]
:
(AbelRuffini.Φ R a b).Monic
theorem
AbelRuffini.irreducible_Phi
(a b p : ℕ)
(hp : Nat.Prime p)
(hpa : p ∣ a)
(hpb : p ∣ b)
(hp2b : ¬p ^ 2 ∣ b)
:
Irreducible (AbelRuffini.Φ ℚ a b)
theorem
AbelRuffini.real_roots_Phi_le
(a b : ℕ)
:
Fintype.card ↑((AbelRuffini.Φ ℚ a b).rootSet ℝ) ≤ 3
theorem
AbelRuffini.real_roots_Phi_ge_aux
(a b : ℕ)
(hab : b < a)
:
∃ (x : ℝ) (y : ℝ),
x ≠ y ∧ (Polynomial.aeval x) (AbelRuffini.Φ ℚ a b) = 0 ∧ (Polynomial.aeval y) (AbelRuffini.Φ ℚ a b) = 0
theorem
AbelRuffini.real_roots_Phi_ge
(a b : ℕ)
(hab : b < a)
:
2 ≤ Fintype.card ↑((AbelRuffini.Φ ℚ a b).rootSet ℝ)
theorem
AbelRuffini.complex_roots_Phi
(a b : ℕ)
(h : (AbelRuffini.Φ ℚ a b).Separable)
:
Fintype.card ↑((AbelRuffini.Φ ℚ a b).rootSet ℂ) = 5
theorem
AbelRuffini.not_solvable_by_rad
(a b p : ℕ)
(x : ℂ)
(hx : (Polynomial.aeval x) (AbelRuffini.Φ ℚ a b) = 0)
(hab : b < a)
(hp : Nat.Prime p)
(hpa : p ∣ a)
(hpb : p ∣ b)
(hp2b : ¬p ^ 2 ∣ b)
:
theorem
AbelRuffini.not_solvable_by_rad'
(x : ℂ)
(hx : (Polynomial.aeval x) (AbelRuffini.Φ ℚ 4 2) = 0)
:
Abel-Ruffini Theorem