Skip to content

Commit

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




Expand Down
3 changes: 1 addition & 2 deletions Game/Levels/Hard/level_2.lean
Original file line number Diff line number Diff line change
@@ -1,7 +1,6 @@
import Game.Levels.Hard.level_1



World "Hard"
Level 2
Title "Collatz"
Expand All @@ -20,7 +19,7 @@ Introduction
"

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

-- halving used for the sequence
Expand Down
4 changes: 2 additions & 2 deletions Game/Levels/Hard/level_3.lean
Original file line number Diff line number Diff line change
Expand Up @@ -17,8 +17,8 @@ Introduction
"

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

Statement Golbach : (∀ n : ℕ), n ≥ 2(∃ a b : ℕ), (Prime a) ∧ (Prime b) ∧ (n = a + b) := by
Statement Golbach : ∀ (n : ℕ), n ≥ 2∃ (a b : ℕ), (Prime a) ∧ (Prime b) ∧ (n = a + b) := by
sorry
3 changes: 1 addition & 2 deletions Game/Levels/Hard/level_4.lean
Original file line number Diff line number Diff line change
Expand Up @@ -16,9 +16,8 @@ Introduction
"

LemmaDoc MyNat.Twin_Prime as "Twin_Prime" in "Hard" "
`Twin_Prime` is the proof of disproof of the Twin Prime conjecture.
`Twin_Prime` is the proof 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 e73913e

Please sign in to comment.