-
Notifications
You must be signed in to change notification settings - Fork 6
/
lakefile.lean
39 lines (31 loc) · 935 Bytes
/
lakefile.lean
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
import Lake
open Lake DSL
package Formal2024 {
leanOptions := #[
⟨`pp.unicode.fun, true⟩,
-- ⟨`pp.proofs.withType, false⟩,
⟨`autoImplicit, false⟩,
⟨`relaxedAutoImplicit, false⟩
]
}
lean_lib Library {
srcDir:= "Tactics"
}
-- lean_lib «TruthTable» {
-- srcDir:= "Tactics"
-- }
lean_lib «MIL» {
srcDir:= "References"
}
lean_lib «Tutorials» {
srcDir:= "References"
}
require mathlib from git "https://github.com/leanprover-community/mathlib4.git"
-- require Paperproof from git "https://github.com/Paper-Proof/paperproof.git"@"main"/"lean"
-- require autograder from git "https://github.com/robertylewis/lean4-autograder-main" @ "master"
-- require proofwidgets from git "https://github.com/EdAyers/ProofWidgets4"@"v0.0.28"
-- require std from git "https://github.com/leanprover/std4.git"
@[default_target]
lean_lib Formal2024 where -- {
-- globs := #[.submodules `Formal2024]
-- }