Files
NNG/Game/Levels/Power/L08pow_pow.lean
2024-06-12 14:38:20 +02:00

49 lines
1.2 KiB
Lean4
Raw Permalink 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.Power.L07mul_pow
World "Power"
Level 8
Title "pow_pow"
namespace MyNat
Introduction
"
One of the best named levels in the game, a savage `pow_pow`
sub-boss appears as the music reaches a frenzy. What
else could there be to prove about powers after this?
"
/-- `pow_pow a m n` is a proof that $(a^m)^n=a^{mn}.$ -/
TheoremDoc MyNat.pow_pow as "pow_pow" in "^"
/-- For all naturals $a$, $m$, $n$, we have $(a ^ m) ^ n = a ^ {mn}$. -/
Statement pow_pow
(a m n : ) : (a ^ m) ^ n = a ^ (m * n) := by
induction n with t Ht
· rw [mul_zero, pow_zero, pow_zero]
rfl
· rw [pow_succ, Ht, mul_succ, pow_add]
rfl
TheoremTab "^"
-- **TODO** if these are `simp` then they should be `simp`ed at source.
attribute [simp] MyNat.pow_zero
attribute [simp] MyNat.pow_succ
attribute [simp] MyNat.pow_one
attribute [simp] MyNat.one_pow
attribute [simp] MyNat.pow_pow -- yes or no?
Conclusion
"
The music dies down. Is that it?
Course it isn't, you can
clearly see that there are two levels left.
A passing mathematician says that mathematicians don't have a name
for the structure you just constructed. You feel cheated.
Suddenly the music starts up again. This really is the final boss.
"