Skip to content

Commit ca0bfca

Browse files
committed
Merge branch 'main' of github.com:ImperialCollegeLondon/FLT
2 parents 338fe38 + 220f2ae commit ca0bfca

File tree

13 files changed

+34
-210
lines changed

13 files changed

+34
-210
lines changed

.gitignore

+3
Original file line numberDiff line numberDiff line change
@@ -15,4 +15,7 @@ blueprint/lean_decls
1515
*.log
1616
*.out
1717
*.pdf
18+
*.fls
19+
*.fdb_latexmk
20+
*.synctex.gz
1821

FLT/Basic/Reductions.lean

+3-3
Original file line numberDiff line numberDiff line change
@@ -51,9 +51,9 @@ theorem PNat.pow_add_pow_ne_pow_of_FermatLastTheorem :
5151

5252
/-- Fermat's Last Theorem is true when n = 3. -/
5353
lemma fermatLastTheoremThree : FermatLastTheoremFor 3 := sorry
54-
-- This is proved in the FLT-regular project: see
55-
-- https://github.com/leanprover-community/flt-regular/blob/861b7df057140b45b8bb7d30d33426ffbbdda52b/FltRegular/FltThree/FltThree.lean#L698
56-
-- The way to turn this node green is to port that work to mathlib so we can use it here.
54+
-- This is proved in the FLT-regular project (https://github.com/leanprover-community/flt-regular/blob/861b7df057140b45b8bb7d30d33426ffbbdda52b/FltRegular/FltThree/FltThree.lean#L698)
55+
-- and the FLT3 project (https://github.com/riccardobrasca/flt3).
56+
-- The way to turn this node green is to port this latter one to mathlib so we can use it here.
5757

5858
namespace FLT
5959

-187 KB
Binary file not shown.

FLT/GlobalLanglandsConjectures/notes.tex

-182
This file was deleted.

FLT/for_mathlib/Coalgebra/Monoid.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -131,9 +131,9 @@ end Coalgebra
131131
section Bialgebra
132132

133133
/--
134-
An algebra homomorphism point is an algebra homorphism from `A` to `L` where `A` is an `R`-biagebra
134+
An algebra homomorphism point is an algebra homomorphism from `A` to `L` where `A` is an `R`-biagebra
135135
and `L` an `R`-algebra. We introduce this abbreviation is to prevent instance clashing when we put a
136-
monnoid structure on these algebra homomorphism points with convolution product.
136+
monoid structure on these algebra homomorphism points with convolution product.
137137
138138
This confusion happens when `A` and `L` are the same where default multiplication is composition.
139139
-/

FLT/for_mathlib/HopfAlgebra/Basic.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -14,10 +14,10 @@ import FLT.for_mathlib.Coalgebra.TensorProduct
1414
For an `R`-hopf algebra `A`, we prove in this file the following basic properties:
1515
- the antipodal map is anticommutative;
1616
- the antipodal map is unique linear map whose convolution inverse is the identity `𝟙 A`.
17-
(Note that, confusingly, the indeity linear map `x ↦ x` is not acutally the unit in the monoid
17+
(Note that, confusingly, the identity linear map `x ↦ x` is not actually the unit in the monoid
1818
structure of linear maps. See `for_mathlib/Coalgebra/Monoid.lean`)
1919
if we further assume `A` is commutative then
20-
- the `R`-algebra homorphisms from `A` to `L` has a group structure where multiplication is
20+
- the `R`-algebra homomorphisms from `A` to `L` has a group structure where multiplication is
2121
convolution, and inverse of `f `is `f ∘ antipode`
2222
- in particular, `antipode ∘ antipode = 1`
2323
-/

blueprint/src/chapter/ch02reductions.tex

+15-12
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
1-
\chapter{First reductions of the problem.}
1+
\chapter{First reductions of the problem}
22

33
\section{Overview}
4-
The proof of Fermat's Last Theorem is by contradiction. We assume that we have a counterexample $a^n+b^n=c^n$, and manipulate it until it satsfies the axioms of a ``Frey package''. From the Frey package we build a Frey curve -- an elliptic curve defined over the rationals. We then look at a certain representation of a Galois group coming from this elliptic curve, and finally using two very deep and independent theorems (one due to Mazur, the other due to Wiles) we show that this representation is neither reducible or irreducible, a contradiction.
4+
The proof of Fermat's Last Theorem is by contradiction. We assume that we have a counterexample $a^n+b^n=c^n$, and manipulate it until it satisfies the axioms of a ``Frey package''. From the Frey package we build a Frey curve -- an elliptic curve defined over the rationals. We then look at a certain representation of a Galois group coming from this elliptic curve, and finally using two very deep and independent theorems (one due to Mazur, the other due to Wiles) we show that this representation is neither reducible or irreducible, a contradiction.
55

66
\section{Reduction to \texorpdfstring{$n\geq5$}{ngeq5} and prime}
77

@@ -28,7 +28,10 @@ \section{Reduction to \texorpdfstring{$n\geq5$}{ngeq5} and prime}
2828
There are no solutions in positive integers to $a^3+b^3=c^3$.
2929
\end{lemma}
3030
\begin{proof}
31-
The proof has been formalised in Lean in the FLT-regular project \href{https://github.com/leanprover-community/flt-regular/blob/861b7df057140b45b8bb7d30d33426ffbbdda52b/FltRegular/FltThree/FltThree.lean#L698}{\underline{here}}. To get this node green, the proof (or another proof) needs to be upstreamed to mathlib. This is currently work in progress by a team from the Lean For the Curious Mathematician conference held in Luminy in March 2024.
31+
A proof has been formalised in Lean in the FLT-regular project \href{https://github.com/leanprover-community/flt-regular/blob/861b7df057140b45b8bb7d30d33426ffbbdda52b/FltRegular/FltThree/FltThree.lean#L698}{\underline{here}}.
32+
Another proof has been formalised in Lean in the FLT3 project \href{https://github.com/riccardobrasca/flt3}{\underline{here}} by a team from the Lean For the Curious Mathematician conference held in Luminy in March 2024
33+
(its dependency graph can be visualised \href{https://pitmonticone.github.io/FLT3/blueprint/dep_graph_document.html}{\underline{here}}).
34+
To get this node green, this latter proof needs to be upstreamed to mathlib. This is currently work in progress by the same team.
3235
\end{proof}
3336

3437
\begin{corollary}\label{FLT.p_ge_5_counterexample_of_not_FermatLastTheorem}\lean{FLT.p_ge_5_counterexample_of_not_FermatLastTheorem}\leanok If there is a counterexample to Fermat's Last Theorem, then there is a counterexample $a^p+b^p=c^p$ with $p$ prime and $p\geq 5$.
@@ -47,9 +50,9 @@ \section{Frey packages}
4750
If Fermat's Last Theorem is false, then there exists a Frey package.
4851
\end{lemma}
4952
\begin{proof}\uses{FLT.FreyPackage, FLT.p_ge_5_counterexample_of_not_FermatLastTheorem} By Corollary \ref{FLT.p_ge_5_counterexample_of_not_FermatLastTheorem} we may assume that there is a counterexample $a^p+b^p=c^p$ with $p\geq 5$ and prime; we now build a Frey package from this data.
50-
51-
If the greatest common divisor of $a,b,c$ is $d$ then $a^p+b^p=c^p$ implies $(a/d)^p+(b/d)^p=(c/d)^p$. Dividing through, we can thus assume that no prime divides all of $a,b,c$. Under this assumption we must have that $a,b,c$ are pairwise coprime, as if some prime divides two of the integers $a,b,c$ then by $a^p+b^p=c^p$ and unique factorization it must divide all three of them. In particular we may assume that not all of $a,b,c$ are even, and now reducing modulo~2 shows that precisely one of them must be even.
52-
53+
54+
If the greatest common divisor of $a,b,c$ is $d$ then $a^p+b^p=c^p$ implies $(a/d)^p+(b/d)^p=(c/d)^p$. Dividing through, we can thus assume that no prime divides all of $a,b,c$. Under this assumption we must have that $a,b,c$ are pairwise coprime, as if some prime divides two of the integers $a,b,c$ then by $a^p+b^p=c^p$ and unique factorization it must divide all three of them. In particular we may assume that not all of $a,b,c$ are even, and now reducing modulo~2 shows that precisely one of them must be even.
55+
5356
Next we show that we can find a counterexample with $b$ even. If $a$ is the even one then we can just switch $a$ and $b$. If $c$ is the even one then we can replace $c$ by $-b$ and $b$ by $-c$ (using that $p$ is odd).
5457

5558
The last thing to ensure is that $a$ is 3 mod~4. Because $b$ is even, we know that $a$ is odd, so it is either~1 or~3 mod~4. If $a$ is 3 mod~4 then we are home; if however $a$ is 1 mod~4 we replace $a,b,c$ by their negatives and this is the Frey package we seek.
@@ -63,7 +66,7 @@ \section{Galois representations and elliptic curves}\label{twopointfour}
6366

6467
The group structure behaves well under change of field.
6568

66-
\begin{lemma}\label{EllipticCurve.Points.map}\lean{EllipticCurve.Points.map}\leanok If $E$ is an elliptic curve over a field $k$, and if $K$ and $L$ are two fields which are $k$-algebras, and if $f:K\to L$ is a $k$-algebra homomorphism, the map from $E(K)$ to $E(L)$ induced by $f$ is an additive group homomorphism.
69+
\begin{lemma}\label{EllipticCurve.Points.map}\lean{EllipticCurve.Points.map}\leanok If $E$ is an elliptic curve over a field $k$, and if $K$ and $L$ are two fields which are $k$-algebras, and if $f:K\to L$ is a $k$-algebra homomorphism, the map from $E(K)$ to $E(L)$ induced by $f$ is an additive group homomorphism.
6770
\end{lemma}
6871
\begin{proof} The equations defining the group law are ratios of polynomials with coefficients in $k$, and such things behave well under $k$-algebra homomorphisms.
6972
\end{proof}
@@ -85,22 +88,22 @@ \section{Galois representations and elliptic curves}\label{twopointfour}
8588
\begin{proof} Another easy calculation.
8689
\end{proof}
8790

88-
Thus if $f K\to L$ is an isomorphism of fields, the induced map $E(K)\to E(L)$ is an isomorphism of groups, with the inverse isomorphism being the map $E(L)\to E(K)$ induced by $f^{-1}$. This construction thus gives us an action of the multiplicative group $\Aut_k(K)$ of automorphisms of the field $K$ on the additive abelian group $E(K)$.
89-
91+
Thus if $f:K\to L$ is an isomorphism of fields, the induced map $E(K)\to E(L)$ is an isomorphism of groups, with the inverse isomorphism being the map $E(L)\to E(K)$ induced by $f^{-1}$. This construction thus gives us an action of the multiplicative group $\Aut_k(K)$ of automorphisms of the field $K$ on the additive abelian group $E(K)$.
92+
9093
\begin{definition}\label{EllipticCurve.galoisRepresentation}\lean{EllipticCurve.galoisRepresentation}\uses{EllipticCurve.Points.map_id,EllipticCurve.Points.map_comp}
9194
If $E$ is an elliptic curve over a field $k$ and $K$ is a field and a $k$-algebra,
9295
then the group of $k$-automorphisms of $K$ acts on the additive abelian group $E(K)$.
9396
\end{definition}
9497
In particular, if $\Qbar$ denotes an algebraic closure of the rationals (for example, the algebraic numbers in $\bbC$) and if $\GQ$ denotes the group of field isomorphisms $\Qbar\to\Qbar$, then for any elliptic curve $E$ over $\Q$ we have an action of $\GQ$ on the additive abelian group $E(\Qbar)$.
9598

96-
We need a variant of this construction where we only consider the $n$-torsion of the curve, for $n$ a positive integer. Recall that if $A$ is any additive abelian group, and if $n$ is a positive integer, then we can consider the subgroup $A[n]$ of elements $a$ such that $na=0$. If a group~$G$ acts on $A$ via additive group isomorphisms, then there will be an induced action of~$G$ on $A[n]$.
99+
We need a variant of this construction where we only consider the $n$-torsion of the curve, for $n$ a positive integer. Recall that if $A$ is any additive abelian group, and if $n$ is a positive integer, then we can consider the subgroup $A[n]$ of elements $a$ such that $na=0$. If a group~$G$ acts on $A$ via additive group isomorphisms, then there will be an induced action of~$G$ on $A[n]$.
97100

98101
\begin{definition}\label{EllipticCurve.torsionGaloisRepresentation}\lean{EllipticCurve.torsionGaloisRepresentation}\uses{EllipticCurve.galoisRepresentation}
99102
If $E$ is an elliptic curve over a field $k$ and $K$ is a field and a $k$-algebra,
100103
and if $n$ is a natural number, hen the group of $k$-automorphisms of $K$ acts on the additive abelian group $E(K)[n]$ of $n$-torsion points on the curve.
101104
\end{definition}
102105

103-
If furthermore $n=p$ is prime, then $A[p]$ is naturally a vector space over the field $\Z/p\Z$, and thus it inherits the stucture of a mod $p$ representation of $G$. Applying this to the above situation, we deduce that if $E$ is an elliptic curve over $\Q$ then $\GQ$ acts on $E(\Qbar)[p]$ and this is the \emph{mod $p$ Galois representation} attached to the curve $E$.
106+
If furthermore $n=p$ is prime, then $A[p]$ is naturally a vector space over the field $\Z/p\Z$, and thus it inherits the structure of a mod $p$ representation of $G$. Applying this to the above situation, we deduce that if $E$ is an elliptic curve over $\Q$ then $\GQ$ acts on $E(\Qbar)[p]$ and this is the \emph{mod $p$ Galois representation} attached to the curve $E$.
104107

105108
In the next section we apply this theory to an elliptic curve coming from a counterexample to Fermat's Last theorem.
106109

@@ -114,7 +117,7 @@ \section{The Frey curve}
114117
Given a Frey package $(a,b,c,p)$ with corresponding Frey curve $E$, the mod $p$ Galois representation associated to this package is the representation of $\GQ$ on $E(\Qbar)[p].$ Frey's observation is that this mod $p$ Galois representation has some very surprising properties. We will make this remark more explicit in the next chapter. Here we shall show how these properties can be used to finish the job.
115118

116119
\section{Reduction to two big theorems.}
117-
120+
118121
Recall that a representation of a group $G$ on a vector space $W$ is said to be \emph{irreducible} if there are precisely two $G$-stable subspaces of $W$, namely $0$ and $W$. The representation is said to be \emph{reducible} otherwise.
119122

120123
Now say Fermat's Last Theorem is false, and hence by Lemma~\ref{FLT.FreyPackage.of_not_FermatLastTheorem} a Frey package $(a,b,c,p)$ exists. Consider the mod $p$ representation of $\GQ$ coming from the $p$-torsion in the Frey curve $Y^2=X(x-a^p)(X+b^p)$ associated to the package. Let's call this representation $\rho$. Is it reducible or irreducible?

blueprint/src/chapter/ch03frey.tex

+1-1
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,7 @@ \section{Overview}
88
\section{The arithmetic of elliptic curves}
99

1010
We give an overview of the results we need, citing the literature for proofs. Everything here is
11-
standard, and mostof it dates back to the 1970s or before.
11+
standard, and most of it dates back to the 1970s or before.
1212

1313
\begin{theorem}\label{EllipticCurve.n_torsion_card}\lean{EllipticCurve.n_torsion_card}\notready
1414
Let $n$ be a positive integer, let $F$ be a separably closed

blueprint/src/chapter/ch04overview.tex

+2-2
Original file line numberDiff line numberDiff line change
@@ -31,7 +31,7 @@ \section{Potential modularity.}
3131
\item A modularity lifting theorem.
3232
\end{itemize}
3333

34-
Almost verything here dates back to the the 1980s or before.
34+
Almost everything here dates back to the the 1980s or before.
3535
The exception is the modularity lifting theorem, which we now state explicitly.
3636

3737
\section{A modularity lifting theorem}
@@ -82,7 +82,7 @@ \section{A modularity lifting theorem}
8282
In the minimal case, the argument is the usual Taylor--Wiles trick, using refinements due to Kisin and others.
8383
\end{proof}
8484

85-
Given this modularity lifting theorem, the strategy to show potential modularity of $\rho$ is to use Moret--Bailly to find an appropriate totally real field $F$, an auxilary prime $p$, and an auxiliary elliptic curve over $F$ whose mod $\ell$ Galois representation is $\rho$ and whose
85+
Given this modularity lifting theorem, the strategy to show potential modularity of $\rho$ is to use Moret--Bailly to find an appropriate totally real field $F$, an auxiliary prime $p$, and an auxiliary elliptic curve over $F$ whose mod $\ell$ Galois representation is $\rho$ and whose
8686
mod $p$ Galois representation is induced from a character. By converse theorems (for example)
8787
the mod $p$ Galois representation is associated to an automorphic representation of
8888
$\GL_2/F$ and hence by Jacquet--Langlands it is modular. Now we use the

blueprint/src/chapter/chtopbestiary.tex

+3-3
Original file line numberDiff line numberDiff line change
@@ -9,7 +9,7 @@ \section{Results from class field theory}
99
Let $K$ be a finite extension of $\Q_p$. We write $\widehat{\Z}$ for the profinite completion of $\Z$; it is isomorphic to $\prod_p\Z_p$ where $\Z_p$ is the $p$-adic integers and the product is over all primes.
1010

1111
\begin{theorem}\label{maximal_unramified_extension_of_p-adic_field}\notready The maximal unramified extension $K^{un}$ in a given algebraic closure of $K$
12-
is Galois over $K$ with Galois group ``canonically'' isomorphic to $\widehat{\Z}$ in two ways; one of these two isomorphisms identifies $1\in\widehat{\Z}$ with an arithmetic Frobenius (the endomorphism inducing $x\mapsto x^q$ on the residue field of $K^{un}$, where $q$ is the size of the residue field of $K$). The other identifies 1 with geometric Frobenius (defined to be the inverse of arithematic Frobenius).
12+
is Galois over $K$ with Galois group ``canonically'' isomorphic to $\widehat{\Z}$ in two ways; one of these two isomorphisms identifies $1\in\widehat{\Z}$ with an arithmetic Frobenius (the endomorphism inducing $x\mapsto x^q$ on the residue field of $K^{un}$, where $q$ is the size of the residue field of $K$). The other identifies 1 with geometric Frobenius (defined to be the inverse of arithmetic Frobenius).
1313
\end{theorem}
1414

1515
It is impossible to say which of the two canonical isomorphisms is ``the most canonical''; people working in different areas make different choices in order to locally minimise the number of minus signs in their results.
@@ -158,7 +158,7 @@ \section{Automorphic forms and representations}
158158
\item $\phi$ is locally constant on $G(\A_N^f)$ and $C^\infty$ on $G(N_\infty)$. In other words, for every $g_\infty$, $\phi(-,g_\infty)$ is locally constant, and for every $g_f$, $\phi(g_f,-)$ is smooth.
159159
\item $\phi$ is left-invariant under $G(N)$;
160160
\item $\phi$ is right-$U_\infty$-finite (that is, the space spanned by $x\mapsto \phi(xu)$ as $u$ varies over $U_\infty$ is finite-dimensional);
161-
\item $\phi$ is right $K_f$-finite, where $K_f$ is one (or equivalentally all) compact open subgroups of $G(\A_N^f)$;
161+
\item $\phi$ is right $K_f$-finite, where $K_f$ is one (or equivalently all) compact open subgroups of $G(\A_N^f)$;
162162
\item $\phi$ is $\mathcal{z}$-finite, where $\mathcal{z}$ is the centre of the universal enveloping algebra of the Lie algebra of $G(N_\infty)$, acting via differential operators. Equivalently $\phi$ is annihiliated by a finite index ideal of this centre, so morally $\phi$ satisfies lots of differential equations of a certain type;
163163
\item For all $g_f$, the function $g_\infty\mapsto \phi(g_f g\infty)$ is slowly-increasing in the sense above.
164164
\end{itemize}
@@ -217,7 +217,7 @@ \section{Galois representations}
217217
\section{Algebraic geometry}
218218

219219
We have already mentioned Mazur's Theorem on torsion subgroups of elliptic curves (theorem~\cite{mazur}).
220-
The proof of this is 100 pages of a subtle analysis of the bad reduction of modular curves and the consquences of this on their Jacobians.
220+
The proof of this is 100 pages of a subtle analysis of the bad reduction of modular curves and the consequences of this on their Jacobians.
221221

222222
Talking of modular curves, we also need the existence of Shimura curves and surfaces over totally real fields~$F$ (of degree greater than~2, so always compact). The curves are "modeles \'etranges" in the sense of Deligne, so we also need moduli spaces of unitary Shimura varieties over CM extensions. We need to decompose the first and second etale cohomology groups of these varieties into Galois representations, by understanding them
223223
in terms of automorphic representations.

blueprint/src/chapter/global_langlands.tex

+1-1
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ \section{Statement of the conjecture}
1212

1313
An \emph{affine group scheme over $R$} is a group object in the category of affine schemes over $R$.
1414

15-
\begin{definition}\label{Hopf_algebra}\lean{TODO}% we have Hopf alegbras in mathlib
15+
\begin{definition}\label{Hopf_algebra}\lean{TODO}% we have Hopf algebras in mathlib
1616

1717
%%%%%%%%%%%%%%%%%%%
1818

blueprint/src/web.tex

+1-1
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@
77
\usepackage{graphicx}
88
\DeclareGraphicsExtensions{.svg,.png,.jpg}
99
\usepackage[capitalize]{cleveref}
10-
\usepackage[dep_graph, project=../../]{blueprint}
10+
\usepackage[showmore,dep_graph, project=../../]{blueprint}
1111

1212
\usepackage{tikz-cd}
1313
\usepackage{tikz}

docs/_config.yml

+1-1
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,7 @@
1818
# You can create any custom variable you would like, and they will be accessible
1919
# in the templates via {{ site.myvariable }}.
2020

21-
title: Fermat's Last Theorems
21+
title: Fermat's Last Theorem
2222
2323
description: An ongoing multi-author open source project to formalise a proof of Fermat's Last Theorem in the Lean theorem prover.
2424
baseurl: "" # the subpath of your site, e.g. /blog

0 commit comments

Comments
 (0)