Files
NNG/Game/Levels/Power.lean

33 lines
1.0 KiB
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.Power.L01zero_pow_zero
import Game.Levels.Power.L02zero_pow_succ
import Game.Levels.Power.L03pow_one
import Game.Levels.Power.L04one_pow
import Game.Levels.Power.L05pow_two
import Game.Levels.Power.L06pow_add
import Game.Levels.Power.L07mul_pow
import Game.Levels.Power.L08pow_pow
import Game.Levels.Power.L09add_sq
import Game.Levels.Power.L10FLT
World "Power"
Title "Power World"
Introduction
"
This world introduces exponentiation. If you want to define `37 ^ n`
then, as always, you will need to know what `37 ^ 0` is, and
what `37 ^ (succ d)` is, given only `37 ^ d`.
You can probably guess the names of the general theorems:
* `pow_zero (a : ) : a ^ 0 = 1`
* `pow_succ (a b : ) : a ^ succ b = a ^ b * a`
Using only these, can you get past the final boss level?
The levels in this world were designed by Sian Carey, a UROP student
at Imperial College London, funded by a Mary Lister McCammon Fellowship
in the summer of 2019. Thanks to Sian and also thanks to Imperial
College for funding her.
"