Zulip Chat Archive
Stream: new members
Topic: Existence proofs
Michael Bucko (Nov 16 2024 at 22:48):
Wrote those 2 proofs from The Mechanics of Proof. In both cases, I used use
. Can I outsource the search to an ATP directly from Lean?
Proof 1
Proof 2
Also, re-wrote the proof from the book like this:
It's a very interesting number
Bjørn Kjos-Hanssen (Nov 17 2024 at 02:06):
At least this works (and is a sufficient search since 13^3 > 1729):
import Mathlib
example : ∃ a b c d : Fin (13),
a ^ 3 + b ^ 3 = 1729 ∧ c ^ 3 + d ^ 3 = 1729 ∧ a ≠ c ∧ a ≠ d := by decide
Last updated: May 02 2025 at 03:31 UTC