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/Predicate/L01_Ring.lean

31 lines
704 B
Plaintext

import Adam.Metadata
2 years ago
import Mathlib.Tactic.Ring
--set_option tactic.hygienic false
Game "Adam"
World "Predicate"
2 years ago
Level 1
Title "Natürliche Zahlen"
Introduction
""
2 years ago
Statement (x y : ) : (x + y) ^ 2 = x ^ 2 + 2 * x * y + y ^ 2 := by
Hint "**Du**: Das ist doch Schulmathematik! Man rechnet das einfach aus,
indem man die Terme umsortiert.
**Robo**: Wenn die Gleichung stimmt, kannst Du auf Leansch sogar einfach mit `ring` beweisen, dass das so ist.
**Du**: Aber `` ist doch gar kein Ring?
2 years ago
**Robo**: `ring` funktioniert sogar für sogenannte Halbringe. Ich glaube, man sagt `ring`, weil es in (kommutativen) Ringen am besten funktioniert.
"
2 years ago
ring
Conclusion
""
2 years ago
NewTactic ring