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/adam/Adam/Levels/Prime/L06_ExistsUnique.lean

35 lines
630 B
Plaintext

import Adam.Metadata
2 years ago
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 Adam.ToBePorted
2 years ago
Game "Adam"
2 years ago
World "Prime"
2 years ago
Level 4
2 years ago
Title "Existiert eindeutig"
Introduction
"
Hier lässt sich noch eine neue Notation einführen: `∃!` bedeutet
\"es existiert ein eindeutiges\" und ist definiert als
"
Statement
"Zeige dass die einzige gerade Primzahl $2$ ist."
: ∃! p, Nat.Prime p ∧ Even p := by
use 2
constructor
simp
rintro y ⟨hy, hy'⟩
rw [←Nat.Prime.even_iff hy]
assumption