Statement of Fermat's Last Theorem #
This file states Fermat's Last Theorem. We provide a statement over a general semiring with specific exponent, along with the usual statement over the naturals.
Main definitions #
FermatLastTheoremWith R n: The statement that only solutions to the Fermat equationa^n + b^n = c^nin the semiringRhavea = 0,b = 0orc = 0.Note that this statement can certainly be false for certain values of
Randn. For exampleFermatLastTheoremWith ℝ 3is false as1^3 + 1^3 = (2^{1/3})^3, andFermatLastTheoremWith ℕ 2is false, as 3^2 + 4^2 = 5^2.FermatLastTheoremFor n: The statement that the only solutions toa^n + b^n = c^ninℕhavea = 0,b = 0orc = 0. Again, this statement is not always true, for exampleFermatLastTheoremFor 1is false because2^1 + 2^1 = 4^1.FermatLastTheorem: The statement of Fermat's Last Theorem, namely that the only solutions toa^n + b^n = c^ninℕwhenn ≥ 3havea = 0,b = 0orc = 0.
History #
Fermat's Last Theorem was an open problem in number theory for hundreds of years, until it was finally solved by Andrew Wiles, assisted by Richard Taylor, in 1994 (see A. Wiles, Modular elliptic curves and Fermat's last theorem and R. Taylor and A. Wiles, Ring-theoretic properties of certain Hecke algebras). An ongoing Lean formalisation of the proof, using mathlib as a dependency, is taking place at https://github.com/ImperialCollegeLondon/FLT .
Statement of Fermat's Last Theorem over the naturals for a given exponent.
Equations
Instances For
Statement of Fermat's Last Theorem: a ^ n + b ^ n = c ^ n has no nontrivial natural solution
when n ≥ 3.
This is now a theorem of Wiles and Taylor--Wiles; see https://github.com/ImperialCollegeLondon/FLT for an ongoing Lean formalisation of a proof.
Equations
- FermatLastTheorem = ∀ n ≥ 3, FermatLastTheoremFor n
Instances For
A relaxed variant of Fermat's Last Theorem over a given commutative semiring with a specific exponent, allowing nonzero solutions of units and their common multiples.
- The variant
FermatLastTheoremWith' Ris weaker thanFermatLastTheoremWith Rin general. In particular, it holds trivially for[Field R]. - This variant is equivalent to the original
FermatLastTheoremWith RforR = ℕorℤ. In general, they are equivalent if there is no solutions of units to the Fermat equation. - For a polynomial ring
R = k[X], the originalFermatLastTheoremWith Ris false but the weaker variantFermatLastTheoremWith' Ris true. This polynomial variant of Fermat's Last Theorem can be shown elementarily using Mason--Stothers theorem.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of fermatLastTheoremWith'_of_semifield.
To prove Fermat Last Theorem in any semiring that is a NormalizedGCDMonoid one can assume
that the gcd of {a, b, c} is 1.