Skip to content

Commit 3165c97

Browse files
committed
chore: update lean
1 parent ec8b427 commit 3165c97

File tree

6 files changed

+14
-13
lines changed

6 files changed

+14
-13
lines changed

.gitignore

+1
Original file line numberDiff line numberDiff line change
@@ -10,3 +10,4 @@ sources/
1010
config.oneshot.json
1111
config.lean.json
1212
config.mathlib.json
13+
lakefile.olean

Mathport.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -34,7 +34,7 @@ def mathport1 (config : Config) (path : Path) : IO Unit := do
3434
|>.setBool `pp.rawOnError true
3535

3636
try
37-
withImportModulesConst imports.toList (opts := opts) (trustLevel := 0) $ λ env => do
37+
withImportModulesConst imports (opts := opts) (trustLevel := 0) $ λ env => do
3838
let env := env.setMainModule path.mod4
3939
let cmdCtx : Elab.Command.Context := {
4040
fileName := path.toLean3 pcfg ".lean" |>.toString

Mathport/Util/Import.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -7,4 +7,4 @@ import Lean
77
open Lean
88

99
@[implemented_by withImportModules]
10-
opaque withImportModulesConst (imports : List Import) (opts : Options) (trustLevel : UInt32 := 0) (x : Environment → IO α) : IO α
10+
opaque withImportModulesConst (imports : Array Import) (opts : Options) (trustLevel : UInt32 := 0) (x : Environment → IO α) : IO α

lake-manifest.json

+9-9
Original file line numberDiff line numberDiff line change
@@ -2,6 +2,14 @@
22
"packagesDir": "lake-packages",
33
"packages":
44
[{"git":
5+
{"url": "https://github.com/leanprover-community/mathlib4",
6+
"subDir?": null,
7+
"rev": "8da7f369150d3ab5cb843226b2d91d84c55c0e7e",
8+
"opts": {},
9+
"name": "mathlib",
10+
"inputRev?": "master",
11+
"inherited": false}},
12+
{"git":
513
{"url": "https://github.com/EdAyers/ProofWidgets4",
614
"subDir?": null,
715
"rev": "44e6673a20fc0449d003983d1e1f472df40f7107",
@@ -17,14 +25,6 @@
1725
"name": "Cli",
1826
"inputRev?": "nightly",
1927
"inherited": true}},
20-
{"git":
21-
{"url": "https://github.com/leanprover-community/mathlib4",
22-
"subDir?": null,
23-
"rev": "193761250a9869327056b499a7f49d676ed5e3a9",
24-
"opts": {},
25-
"name": "mathlib",
26-
"inputRev?": "master",
27-
"inherited": false}},
2828
{"git":
2929
{"url": "https://github.com/gebner/quote4",
3030
"subDir?": null,
@@ -44,7 +44,7 @@
4444
{"git":
4545
{"url": "https://github.com/leanprover/std4",
4646
"subDir?": null,
47-
"rev": "ba5e5e3af519b4fc5221ad0fa4b2c87276f1d323",
47+
"rev": "67855403d60daf181775fa1ec63b04e70bcc3921",
4848
"opts": {},
4949
"name": "std",
5050
"inputRev?": "main",

lakefile.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@ target ffi.o pkg : FilePath := do
1111
let oFile := pkg.buildDir / "c" / "ffi.o"
1212
let srcJob ← inputFile <| pkg.dir / "Mathport" / "FFI.cpp"
1313
let flags := #["-I", (← getLeanIncludeDir).toString, "-fPIC"]
14-
buildO "FFI.c" oFile srcJob flags "c++"
14+
buildO "FFI.c" oFile srcJob flags (compiler := "c++")
1515

1616
extern_lib libleanffi (pkg : NPackage `mathport) := do
1717
let name := nameToStaticLib "leanffi"

lean-toolchain

+1-1
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.0.0
1+
leanprover/lean4:v4.1.0-rc1

0 commit comments

Comments
 (0)