Skip to content

Commit

Permalink
steps towards chinese nng
Browse files Browse the repository at this point in the history
  • Loading branch information
joneugster committed Mar 27, 2024
1 parent fdad0f8 commit 20813a0
Show file tree
Hide file tree
Showing 8 changed files with 1,485 additions and 4,387 deletions.
3,744 changes: 0 additions & 3,744 deletions .i18n/Game.pot

This file was deleted.

3 changes: 2 additions & 1 deletion .i18n/config.json
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
{
"sourceLang": "en",
"translationContactEmail": ""
"translationContactEmail": "",
"useJson": true
}
740 changes: 740 additions & 0 deletions .i18n/en/Game.json

Large diffs are not rendered by default.

1,365 changes: 732 additions & 633 deletions .i18n/zh/Game.json

Large diffs are not rendered by default.

6 changes: 3 additions & 3 deletions .i18n/Game-zh_CN.po → .i18n/zh/Game.po
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ msgstr ""
"Report-Msgid-Bugs-To: \n"
"POT-Creation-Date: Mon Mar 18 16:33:40 2024\n"
"PO-Revision-Date: \n"
"Last-Translator: \n"
"Last-Translator: @JiechengZhao \n"
"Language-Team: none\n"
"Language: zh_CN\n"
"MIME-Version: 1.0\n"
Expand Down Expand Up @@ -639,7 +639,7 @@ msgid ""
"## Details\n"
"\n"
"A mathematician sometimes thinks of `add_zero`\n"
"as \"one thing\", namely a proof of $\forall n ∈ ℕ, n + 0 = n$.\n"
"as \"one thing\", namely a proof of $\\forall n ∈ ℕ, n + 0 = n$.\n"
"This is just another way of saying that it's a function which\n"
"can eat any number n and will return a proof that `n + 0 = n`."
msgstr ""
Expand Down Expand Up @@ -2493,7 +2493,7 @@ msgid ""
"You can think of `succ_inj` itself as a proof; it is the proof\n"
"that `succ` is an injective function. In other words,\n"
"`succ_inj` is a proof of\n"
"$\forall a, b \\in \\mathbb{N}, ( \\operatorname{succ}(a) = \\operatorname{succ}(b)) \\implies a=b$.\n"
"$\\forall a, b \\in \\mathbb{N}, ( \\operatorname{succ}(a) = \\operatorname{succ}(b)) \\implies a=b$.\n"
"\n"
"`succ_inj` was postulated as an axiom by Peano, but\n"
"in Lean it can be proved using `pred`, a mathematically\n"
Expand Down
3 changes: 2 additions & 1 deletion Game.lean
Original file line number Diff line number Diff line change
Expand Up @@ -17,6 +17,7 @@ import Game.Levels.AdvMultiplication
--import Game.Levels.StrongInduction
--import Game.Levels.Hard
import Game.Levels.Algorithm
import I18n

-- Here's what we'll put on the title screen
Title "Natural Number Game"
Expand Down Expand Up @@ -101,7 +102,7 @@ Alternatively, if you experience issues / bugs you can also open github issues:
-- Dependency Implication → Power -- `Power` uses `≠` which is introduced in `Implication`

/-! Information to be displayed on the servers landing page. -/
Languages "English"
Languages "en" "zh"
CaptionShort "The classical introduction game for Lean."
CaptionLong "In this game you recreate the natural numbers $\\mathbb{N}$ from the Peano axioms,
learning the basics about theorem proving in Lean.
Expand Down
8 changes: 4 additions & 4 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -13,19 +13,19 @@
{"url": "https://github.com/hhu-adam/lean-i18n.git",
"type": "git",
"subDir": null,
"rev": "c5b84feffb28dbd5b1ac74b3bf63271296fabfa5",
"rev": "2c5ce050296621fda7f938b270a18d00672d556b",
"name": "i18n",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.6.0",
"inputRev": "main",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/lean4game.git",
"type": "git",
"subDir": "server",
"rev": "68f84a3426684914f834342854bf4963ba2d8d57",
"rev": "1a54edffd49bc49f699de74c868656d1914f00c0",
"name": "GameServer",
"manifestFile": "lake-manifest.json",
"inputRev": "v4.6.0",
"inputRev": "dev",
"inherited": false,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover-community/quote4",
Expand Down
3 changes: 2 additions & 1 deletion lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,7 +11,8 @@ def LocalGameServer : Dependency := {

def RemoteGameServer : Dependency := {
name := `GameServer
src := Source.git "https://github.com/leanprover-community/lean4game.git" leanVersion "server"
-- TODO: change back to stable version
src := Source.git "https://github.com/leanprover-community/lean4game.git" "dev" "server" -- leanVersion "server"
}

/- Choose GameServer dependency depending on the environment variable `LEAN4GAME`. -/
Expand Down

1 comment on commit 20813a0

@zzz6519003
Copy link

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

bravo!

Please sign in to comment.