Files
NNG/Game/Levels/AdvAddition/Level_11.lean
Jon Eugster 2604c89284 big refactor
2023-05-15 15:12:35 +02:00

31 lines
511 B
Lean4
Raw Blame History

This file contains ambiguous Unicode characters
This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.
import Game.Levels.AdvAddition.Level_10
Game "NNG"
World "AdvAddition"
Level 11
Title "add_right_eq_zero"
open MyNat
Introduction
"
We just proved `add_left_eq_zero (a b : ) : a + b = 0 → b = 0`.
Hopefully `add_right_eq_zero` shouldn't be too hard now.
"
Statement MyNat.add_right_eq_zero
"If $a$ and $b$ are natural numbers such that
$$ a + b = 0, $$
then $a = 0$."
{a b : } : a + b = 0 a = 0 := by
intro h
rw [add_comm] at h
exact add_left_eq_zero h
LemmaTab "Add"
Conclusion
"
"