You cannot select more than 25 topics Topics must start with a letter or number, can include dashes ('-') and can be up to 35 characters long.
lean4game/server/testgame/TestGame/Levels/Prime/L01_Prime.lean

40 lines
570 B
Plaintext

import TestGame.Metadata
import Mathlib.Data.Nat.Prime
import Std.Tactic.RCases
import Mathlib.Tactic.LeftRight
import Mathlib.Tactic.Contrapose
import Mathlib.Tactic.Use
import Mathlib.Tactic.Ring
import TestGame.ToBePorted
Game "TestGame"
World "Prime"
Level 1
Title "Primzahlen"
Introduction
"
"
Statement
"TODO"
(n : ) : ∃! (n : ), Nat.Prime n ∧ Even n := by
use (2 : )
constructor
simp only [true_and]
use 1
intro y
rintro ⟨h₁, h₂⟩
rw [← Nat.Prime.even_iff]
assumption
assumption
Conclusion ""
Tactics
Lemmas