Skip to content

Commit

Permalink
Golbach Conjecture
Browse files Browse the repository at this point in the history
  • Loading branch information
archiebrowne committed Nov 16, 2023
1 parent 3ee7a21 commit 67c7253
Show file tree
Hide file tree
Showing 2 changed files with 24 additions and 2 deletions.
2 changes: 0 additions & 2 deletions Game/Levels/Hard/level_2.lean
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
import Game.Levels.Hard.level_1
import Game.MyNat.Multiplication




Expand Down
24 changes: 24 additions & 0 deletions Game/Levels/Hard/level_3.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,24 @@
import Game.Levels.Hard.level_2


World "Hard"
Level 3
Title "Golbach"

LemmaTab "Hard"

namespace MyNat

Introduction
"
The Golbach conjecture, first posed in 1792 in a letter to Euler states that every
natural number greater than 2 is the sum of two prime numbers. It remains unproven
to this day, but has been checked for all naturals up to 4 x 10¹⁸.
"

LemmaDoc MyNat.Golbach as "Golbach" in "Hard" "
`Golbach` is the proof of disproof of the Golbach conjecture.
"

Statement Golbach : (∀ n : ℕ), n ≥ 2 → (∃ a b : ℕ), (Prime a) ∧ (Prime b) ∧ (n = a + b) := by
sorry

0 comments on commit 67c7253

Please sign in to comment.