Files
NNG/Game/Levels/Tutorial.lean
2023-08-25 02:56:40 +01:00

21 lines
647 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.Tutorial.L01rfl
import Game.Levels.Tutorial.L02rw
import Game.Levels.Tutorial.L03three_eq_sss0
import Game.Levels.Tutorial.L04add_zero
import Game.Levels.Tutorial.L05add_succ
import Game.Levels.Tutorial.L06twoaddone
import Game.Levels.Tutorial.L07twoaddtwo
World "Tutorial"
Title "Tutorial World"
Introduction
"
In this world we introduce two basic tactics (`rfl` and `rw`).
We also introduce several mathematical concepts: the (natural) numbers ``,
explicit examples of numbers such as 0 and 3, and addition of two numbers.
The final boss is to prove that `2 + 2 = 4`. Good luck!
Click on \"Next\" to begin your quest.
"