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/StatementTest.lean

39 lines
631 B
Plaintext

2 years ago
import TestGame.Metadata
import Mathlib
Game "TestGame"
World "TestWorld"
Level 1
Title "Annahmen"
Introduction "yadaa yadaa"
class MyClass (n : ) where
Statement name
"Beweise dieses Lemma."
(n m : ) : CommSemigroup where
mul := fun i j => 0
mul_comm := sorry
mul_assoc := sorry
--@[exercise]
instance instTest (n m : ) : CommSemigroup where
mul := fun i j => 0
mul_comm := by
sorry
mul_assoc := by
sorry
--@[exercise]
lemma asdf (a b c d : ) (h₁ : c = d) (h₂ : a = b) (h₃ : a = d) : b = c := by
rewrite [h₁]
rw [←h₂]
assumption
Conclusion ""
Tactics assumption