File tree 6 files changed +14
-13
lines changed
6 files changed +14
-13
lines changed Original file line number Diff line number Diff line change @@ -10,3 +10,4 @@ sources/
10
10
config.oneshot.json
11
11
config.lean.json
12
12
config.mathlib.json
13
+ lakefile.olean
Original file line number Diff line number Diff line change @@ -34,7 +34,7 @@ def mathport1 (config : Config) (path : Path) : IO Unit := do
34
34
|>.setBool `pp.rawOnError true
35
35
36
36
try
37
- withImportModulesConst imports.toList (opts := opts) (trustLevel := 0 ) $ λ env => do
37
+ withImportModulesConst imports (opts := opts) (trustLevel := 0 ) $ λ env => do
38
38
let env := env.setMainModule path.mod4
39
39
let cmdCtx : Elab.Command.Context := {
40
40
fileName := path.toLean3 pcfg ".lean" |>.toString
Original file line number Diff line number Diff line change @@ -7,4 +7,4 @@ import Lean
7
7
open Lean
8
8
9
9
@[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 α
Original file line number Diff line number Diff line change 2
2
"packagesDir" : " lake-packages" ,
3
3
"packages" :
4
4
[{"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" :
5
13
{"url" : " https://github.com/EdAyers/ProofWidgets4" ,
6
14
"subDir?" : null ,
7
15
"rev" : " 44e6673a20fc0449d003983d1e1f472df40f7107" ,
17
25
"name" : " Cli" ,
18
26
"inputRev?" : " nightly" ,
19
27
"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 }},
28
28
{"git" :
29
29
{"url" : " https://github.com/gebner/quote4" ,
30
30
"subDir?" : null ,
44
44
{"git" :
45
45
{"url" : " https://github.com/leanprover/std4" ,
46
46
"subDir?" : null ,
47
- "rev" : " ba5e5e3af519b4fc5221ad0fa4b2c87276f1d323 " ,
47
+ "rev" : " 67855403d60daf181775fa1ec63b04e70bcc3921 " ,
48
48
"opts" : {},
49
49
"name" : " std" ,
50
50
"inputRev?" : " main" ,
Original file line number Diff line number Diff line change @@ -11,7 +11,7 @@ target ffi.o pkg : FilePath := do
11
11
let oFile := pkg.buildDir / "c" / "ffi.o"
12
12
let srcJob ← inputFile <| pkg.dir / "Mathport" / "FFI.cpp"
13
13
let flags := #["-I" , (← getLeanIncludeDir).toString, "-fPIC" ]
14
- buildO "FFI.c" oFile srcJob flags "c++"
14
+ buildO "FFI.c" oFile srcJob flags (compiler := "c++" )
15
15
16
16
extern_lib libleanffi (pkg : NPackage `mathport) := do
17
17
let name := nameToStaticLib "leanffi"
Original file line number Diff line number Diff line change 1
- leanprover/lean4:v4.0.0
1
+ leanprover/lean4:v4.1.0-rc1
You can’t perform that action at this time.
0 commit comments