Skip to content

Commit

Permalink
fix "no text on tutorial intro" bug
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Sep 25, 2023
1 parent 0249d2e commit 707f7c4
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 5 deletions.
6 changes: 5 additions & 1 deletion Game/Levels/Addition/L01zero_add.lean
Original file line number Diff line number Diff line change
@@ -1,6 +1,10 @@
import Game.Metadata
import Game.MyNat.Addition
import Game.Levels.Tutorial.L05add_succ
import Game.MyNat.DecidableEq

-- try to fix tutorial world entry page text issue
-- import Game.Levels.Tutorial.L05add_succ

World "Addition"
Level 1
Title "zero_add"
Expand Down
4 changes: 0 additions & 4 deletions Game/Levels/Multiplication/L01mul_one.lean
Original file line number Diff line number Diff line change
Expand Up @@ -35,20 +35,16 @@ NewDefinition Mul

LemmaDoc MyNat.mul_zero as "mul_zero" in "Mul"
"
`mul_zero m` is the proof that `m * 0 = 0`."

LemmaDoc MyNat.mul_succ as "mul_succ" in "Mul"
"
`mul_succ a b` is the proof that `a * succ b = a * b + a`.
"

NewLemma MyNat.mul_zero MyNat.mul_succ

LemmaDoc MyNat.mul_one as "mul_one" in "Mul" "
`mul_one m : m * 1 = m`
`mul_one m` is the proof that `m * 1 = m`.
"

Expand Down
1 change: 1 addition & 0 deletions Game/Levels/Tutorial/L03three_eq_sss0.lean
Original file line number Diff line number Diff line change
Expand Up @@ -78,6 +78,7 @@ LemmaDoc MyNat.four_eq_succ_three as "four_eq_succ_three" in "numerals"

NewLemma MyNat.one_eq_succ_zero MyNat.two_eq_succ_one MyNat.three_eq_succ_two
MyNat.four_eq_succ_three

LemmaTab "numerals"

Conclusion
Expand Down

0 comments on commit 707f7c4

Please sign in to comment.