-
Notifications
You must be signed in to change notification settings - Fork 90
/
lakefile.lean
32 lines (27 loc) · 1020 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
import Lake
open Lake DSL
package math2001 where
moreServerArgs := #[
"-Dlinter.unusedVariables=false", -- ignores unused variables
"-DquotPrecheck=false",
"-DwarningAsError=false",
"-Dpp.unicode.fun=true" -- pretty-prints `fun a ↦ b`
]
lean_lib Library
@[default_target]
lean_lib Math2001 where
globs := #[.submodules `Math2001]
moreLeanArgs := #[
"-Dlinter.unusedVariables=false", -- ignores unused variables
"-DquotPrecheck=false",
"-DwarningAsError=false",
"-Dpp.unicode.fun=true" -- pretty-prints `fun a ↦ b`
]
/-
want also
"-Dpush_neg.use_distrib=true", -- negates ¬(P ∧ Q) to (¬ P ∨ ¬ Q)
but currently only Lean core options can be set in lakefile
-/
require mathlib from git "https://github.com/leanprover-community/mathlib4" @ s!"v{Lean.versionString}"
require Duper from git "https://github.com/hrmacbeth/duper" @ "main"
require autograder from git "https://github.com/robertylewis/lean4-autograder-main" @ "864b34ce06d8536aec0c38e57448c17d1f83572a"