Zulip Chat Archive

Stream: maths

Topic: Fermat's last theorem for n=3


Riccardo Brasca (May 11 2022 at 12:29):

@Ruben Van de Velde If I remember correctly you were working on the case n=3 of Fermat's last theorem. What is the status of your project? I think this case has to be treated by hand, even if 3 is a regular prime.

Riccardo Brasca (May 11 2022 at 12:34):

I found you repository, and

lemma flt_three
  {a b c : }
  (ha : a  0)
  (hb : b  0)
  (hc : c  0) :
  a ^ 3 + b ^ 3  c ^ 3

is sorry free! Congratulations! Are you interested in PRing this to mathlib?

Ruben Van de Velde (May 11 2022 at 13:01):

Yeah, next step is probably figuring out if there's anything I can split out or if I should just make a 2500 line PR. I haven't had much time for it recently

Yaël Dillies (May 11 2022 at 13:03):

Oh are you actually using docs#zsqrtd? It seems that this is a quite dated construct that either needs to be replaced by the more general machinery we now have or be substantially reworked to bring it up to today's standards.

Riccardo Brasca (May 11 2022 at 13:11):

docs#zsqrt is unfortunately mathematically wrong, in the sense that we should consider the ring of integers of Q(d)\mathbb{Q}(\sqrt{d}).

Riccardo Brasca (May 11 2022 at 13:12):

It's surprisingly that it is enough for d=-3, but of course a proof is a proof

Yaël Dillies (May 11 2022 at 13:12):

Yeah so a first step would be to get rid of the use of zsqrtd in the proof.

Riccardo Brasca (May 11 2022 at 13:14):

We really need a number_theory/quadratic_field folder...

Eric Rodriguez (May 11 2022 at 13:23):

Imagine telling people that we have the discriminant of the p^nth cyclotomic field and not the rth quadratic field :D

Ruben Van de Velde (May 11 2022 at 13:27):

I have no particular interest in reworking the proof I have using the the ring of integers of Q(3)\mathbb{Q}(\sqrt{-3}); if people think that's the way to go, we might need to find another volunteer :)

Eric Wieser (May 11 2022 at 18:39):

Sorry, docs#zsqrtd is wrong as in doesn't accurately model what it claims to, or just isn't what's needed here?

Kevin Buzzard (May 11 2022 at 18:42):

I think the issue is that mathematically the integers of Q(3)\mathbb{Q}(\sqrt{-3}) is strictly bigger than Z[3]\mathbb{Z}[\sqrt{-3}] as it also contains (1+3)/2(1+\sqrt{-3})/2.

Eric Wieser (May 11 2022 at 19:19):

Should we just change zsqrtd to sqrtd ℤ, making ℤ an argument?

Riccardo Brasca (May 11 2022 at 19:20):

It's "wrong" in the sense it's not mathematically interesting (at least, not always). For example what one wants is Z[1+32]\mathbb{Z}[\frac{1+\sqrt{-3}}{2}] as Kevin said

Riccardo Brasca (May 11 2022 at 19:22):

In any case what we probably want is a characteristic predicate saying that a field is a quadratic extension of Q\mathbb{Q} associated to dd, and then we abstractly have its ring of integers.

Riccardo Brasca (May 11 2022 at 19:31):

Something like "the dimension over Q\mathbb{Q} is 2 and there is an element whose square is d, where d is a squarefree integer".

Kevin Buzzard (May 11 2022 at 20:39):

The ring zsqrt d is relevant for eg solutions to Pell's equation when d isn't squarefree; IIRC this is why Mario made that structure in the first place. I think it plays a useful role; we number theorists can develop the theory of integers of number fields elsewhere.

Kevin Buzzard (May 11 2022 at 20:41):

There's a theory of orders in number fields, they relate to ring class fields (or is it ray class fields, I can never remember which is which) and a theorem saying that most ideals factor uniquely into primes etc.

Anne Baanen (May 12 2022 at 09:22):

Eric Wieser said:

Should we just change zsqrtd to sqrtd ℤ, making ℤ an argument?

Alex, Nirvana, Sander and I are working on defining a "generic quadratic ring", i.e. R[X] / X^2 - aX - b for arbitrary rings R and a, b : R.

Kevin Buzzard (May 12 2022 at 14:53):

Oh that's a nice approach!


Last updated: Dec 20 2023 at 11:08 UTC