Documentation

Counterexamples.EulerSumOfPowers

Euler's sum of powers conjecture #

Euler's sum of powers conjecture says that at least n nth powers of positive integers are required to sum to an nth power of a positive integer.

This was an attempt to generalize Fermat's Last Theorem, which is the special case of summing 2 nth powers.

We demonstrate the connection with FLT, prove that it's true for n ≤ 3, and provide counterexamples for n = 4 and n = 5. The status of the conjecture for n ≥ 6 is unknown.

https://en.wikipedia.org/wiki/Euler%27s_sum_of_powers_conjecture http://euler.free.fr/

TODO #

@[reducible, inline]

Euler's sum of powers conjecture over a given semiring with a specific exponent.

Equations
Instances For
    @[reducible, inline]

    Euler's sum of powers conjecture over the naturals for a given exponent.

    Equations
    Instances For
      @[reducible, inline]

      Euler's sum of powers conjecture over the naturals.

      Equations
      Instances For

        Euler's sum of powers conjecture over a given semiring with a specific exponent implies FLT.

        Euler's sum of powers conjecture over the naturals implies FLT.

        For n = 3, Euler's sum of powers conjecture over a given semiring is equivalent to FLT.

        Euler's sum of powers conjecture over the naturals is true for n ≤ 3.

        theorem Counterexample.sumOfPowersConjecture_of_ringHom {R : Type u_1} {S : Type u_2} [Semiring R] [Semiring S] {f : R →+* S} (hf : ∀ (x : R), f x = 0x = 0) {n : } (conj : SumOfPowersConjectureWith S n) :

        Given a ring homomorphism from R to S with no nontrivial zeros, the conjecture over S implies the conjecture over R.

        Given an injective ring homomorphism from R to S, the conjecture over S implies the conjecture over R.

        The first counterexample was found by Leon J. Lander and Thomas R. Parkin in 1966 through a computer search, disproving the conjecture. https://www.ams.org/journals/bull/1966-72-06/S0002-9904-1966-11654-3/S0002-9904-1966-11654-3.pdf This is also the smallest counterexample for n = 5.

        The first counterexample for n = 4 was found by Noam D. Elkies in October 1988: a := [2_682_440, 15_365_639, 18_796_760], b := 20_615_673 https://www.ams.org/journals/mcom/1988-51-184/S0025-5718-1988-0930224-9/S0025-5718-1988-0930224-9.pdf In this paper, Elkies constructs infinitely many solutions to a^4 + b^4 + c^4 = d^4 for coprime a, b, c, d, which provide infinitely many coprime counterexamples for the case n = 4. Here we use the smallest counterexample for n = 4, which was found a month later by Roger E. Frye https://ieeexplore.ieee.org/document/74138

        @[reducible, inline]

        For all (k, m, n) we define the Diophantine equation ∑ x_i ^ k = ∑ y_i ^ k where x and y are disjoint with length m and n respectively. This is a generalization of the diophantine equation of Euler's sum of powers conjecture.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          Euler's sum of powers conjecture for k restricts solutions for (k, m, 1).

          @[reducible, inline]

          After the first counterexample was found, Leon J. Lander, Thomas R. Parkin, and John Selfridge made a similar conjecture that is not amenable to the counterexamples found so far. The status of this conjecture is unknown. https://en.wikipedia.org/wiki/Lander,_Parkin,_and_Selfridge_conjecture https://www.ams.org/journals/mcom/1967-21-099/S0025-5718-1967-0222008-0/S0025-5718-1967-0222008-0.pdf

          Equations
          Instances For

            Euler's sum of powers conjecture for k implies the Lander, Parkin, and Selfridge conjecture for (k, m, 1).