Skip to content

Commit 603affe

Browse files
committed
Bump toolchain to 4.12
Signed-off-by: Andrew Wells <andrewmw94@gmail.com>
1 parent adbbfcb commit 603affe

File tree

7 files changed

+27
-15
lines changed

7 files changed

+27
-15
lines changed

REPL/Lean/Environment.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -26,6 +26,6 @@ and then replace the new constants.
2626
def unpickle (path : FilePath) : IO (Environment × CompactedRegion) := unsafe do
2727
let ((imports, map₂), region) ← _root_.unpickle (Array Import × PHashMap Name ConstantInfo) path
2828
let env ← importModules imports {} 0
29-
return (← env.replay (HashMap.ofList map₂.toList), region)
29+
return (← env.replay (Std.HashMap.ofList map₂.toList), region)
3030

3131
end Lean.Environment

REPL/Main.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -205,6 +205,8 @@ def runCommand (s : Command) : M IO (CommandResponse ⊕ Error) := do
205205
let tactics ← match s.allTactics with
206206
| some true => tactics trees
207207
| _ => pure []
208+
-- The list is repeated, so we only keep the second half.
209+
let tactics := tactics.drop (tactics.length / 2)
208210
let cmdSnapshot :=
209211
{ cmdState
210212
cmdContext := (cmdSnapshot?.map fun c => c.cmdContext).getD

REPL/Snapshots.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -83,7 +83,7 @@ def unpickle (path : FilePath) : IO (CommandSnapshot × CompactedRegion) := unsa
8383
let ((imports, map₂, cmdState, cmdContext), region) ←
8484
_root_.unpickle (Array Import × PHashMap Name ConstantInfo × CompactableCommandSnapshot ×
8585
Command.Context) path
86-
let env ← (← importModules imports {} 0).replay (HashMap.ofList map₂.toList)
86+
let env ← (← importModules imports {} 0).replay (Std.HashMap.ofList map₂.toList)
8787
let p' : CommandSnapshot :=
8888
{ cmdState := { cmdState with env }
8989
cmdContext }
@@ -285,9 +285,9 @@ def unpickle (path : FilePath) (cmd? : Option CommandSnapshot) :
285285
let env ← match cmd? with
286286
| none =>
287287
enableInitializersExecution
288-
(← importModules imports {} 0).replay (HashMap.ofList map₂.toList)
288+
(← importModules imports {} 0).replay (Std.HashMap.ofList map₂.toList)
289289
| some cmd =>
290-
cmd.cmdState.env.replay (HashMap.ofList map₂.toList)
290+
cmd.cmdState.env.replay (Std.HashMap.ofList map₂.toList)
291291
let p' : ProofSnapshot :=
292292
{ coreState := { coreState with env }
293293
coreContext

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.11.0
1+
leanprover/lean4:v4.12.0

test/Mathlib/lake-manifest.json

Lines changed: 18 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "leanprover-community",
8-
"rev": "9c6c2d647e57b2b7a0b42dd8080c698bd33a1b6f",
8+
"rev": "4756e0fc48acce0cc808df0ad149de5973240df6",
99
"name": "batteries",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "main",
@@ -15,7 +15,7 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "leanprover-community",
18-
"rev": "9d0bdd07bdfe53383567509348b1fe917fc08de4",
18+
"rev": "2c8ae451ce9ffc83554322b14437159c1a9703f9",
1919
"name": "Qq",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "master",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "deb279eb7be16848d0bc8387f80d6e41bcdbe738",
28+
"rev": "28fa80508edc97d96ed6342c9a771a67189e0baa",
2929
"name": "aesop",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "master",
@@ -35,10 +35,10 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "a96aee5245720f588876021b6a0aa73efee49c76",
38+
"rev": "eb08eee94098fe530ccd6d8751a86fe405473d4c",
3939
"name": "proofwidgets",
4040
"manifestFile": "lake-manifest.json",
41-
"inputRev": "v0.0.41",
41+
"inputRev": "v0.0.42",
4242
"inherited": true,
4343
"configFile": "lakefile.lean"},
4444
{"url": "https://github.com/leanprover/lean4-cli",
@@ -55,20 +55,30 @@
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "1ef0b288623337cb37edd1222b9c26b4b77c6620",
58+
"rev": "e285a7ade149c551c17a4b24f127e1ef782e4bb1",
5959
"name": "importGraph",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "main",
6262
"inherited": true,
6363
"configFile": "lakefile.toml"},
64+
{"url": "https://github.com/leanprover-community/LeanSearchClient",
65+
"type": "git",
66+
"subDir": null,
67+
"scope": "leanprover-community",
68+
"rev": "2ba60fa2c384a94735454db11a2d523612eaabff",
69+
"name": "LeanSearchClient",
70+
"manifestFile": "lake-manifest.json",
71+
"inputRev": "main",
72+
"inherited": true,
73+
"configFile": "lakefile.toml"},
6474
{"url": "https://github.com/leanprover-community/mathlib4",
6575
"type": "git",
6676
"subDir": null,
6777
"scope": "",
68-
"rev": "8edf04f0977c3183d3b633792e03fd570be1777f",
78+
"rev": "809c3fb3b5c8f5d7dace56e200b426187516535a",
6979
"name": "mathlib",
7080
"manifestFile": "lake-manifest.json",
71-
"inputRev": "master",
81+
"inputRev": "v4.12.0",
7282
"inherited": false,
7383
"configFile": "lakefile.lean"}],
7484
"name": "«repl-mathlib-tests»",

test/Mathlib/lakefile.toml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ defaultTargets = ["ReplMathlibTests"]
44
[[require]]
55
name = "mathlib"
66
git = "https://github.com/leanprover-community/mathlib4"
7-
rev = "master"
7+
rev = "v4.12.0"
88

99
[[lean_lib]]
1010
name = "ReplMathlibTests"

test/Mathlib/lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.11.0
1+
leanprover/lean4:v4.12.0

0 commit comments

Comments
 (0)