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/LeftOvers/xx_Functions.lean

26 lines
471 B
Plaintext

import TestGame.Metadata
import Mathlib.Tactic.Ring
Game "TestGame"
World "Function"
Level 1
Title "Funktionen"
Introduction
"
Funktionen werden in Lean als `(f : )` geschrieben (`\\to`), also mit dem gleichen
Pfeil wie Implikationen. Entsprechend kann man Implikationen und Funktionen genau
gleich behandeln.
"
Statement : ∃ (f : ), ∀ (x : ), f x = 0 := by
let g := fun (x : ) ↦ 0
use g
simp
Conclusion ""
Tactics use simp