Skip to content

Commit

Permalink
statment of Twin Prime
Browse files Browse the repository at this point in the history
  • Loading branch information
archiebrowne committed Nov 16, 2023
1 parent 67c7253 commit c5d6984
Show file tree
Hide file tree
Showing 2 changed files with 26 additions and 0 deletions.
2 changes: 2 additions & 0 deletions Game/Levels/Hard.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,8 @@ import Game.Levels.Power
import Game.MyNat.Addition
import Game.MyNat.Multiplication



World "Hard"
Title "Hard World"

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


World "Hard"
Level 3
Title "Twin Prime"

LemmaTab "Hard"

namespace MyNat

Introduction
"
A twin prime is a pair of primes (2, 3), (41, 43) etc. that are 2 apart. The conjecture
states that there are infinitley many such pairs.
"

LemmaDoc MyNat.Twin_Prime as "Twin_Prime" in "Hard" "
`Twin_Prime` is the proof of disproof of the Twin Prime conjecture.
"

Statement Twin_Prime :
(∀ M : ℕ), (∃ a b : ℕ), (a ≥ M) ∧ (b ≥ M) ∧ (a + 2 = b) ∧ (Prime a) ∧ (Prime b) := by sorry

0 comments on commit c5d6984

Please sign in to comment.