Skip to content

Commit

Permalink
chore: simplify lakefile (#950)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Sep 28, 2024
1 parent 8311edc commit 51c38e3
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 7 deletions.
2 changes: 1 addition & 1 deletion .github/workflows/build.yml
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,7 @@ jobs:
name: build, test, and lint batteries
uses: leanprover/lean-action@v1
with:
build-args: '-Kwerror'
build-args: '--wfail'

- name: Check that all files are imported
run: lake env lean scripts/check_imports.lean
Expand Down
7 changes: 1 addition & 6 deletions lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,13 +2,8 @@ import Lake

open Lake DSL

macro "opt_arg?" x:ident v:term : term => `(if get_config? $x |>.isSome then $v else default)

package batteries where
moreLeanArgs := opt_arg? werror #["-DwarningAsError=true"]
leanOptions :=
#[⟨`linter.missingDocs, true⟩] ++
opt_arg? disable_new_compiler #[⟨`compiler.enableNew, false⟩]
leanOptions := #[⟨`linter.missingDocs, true⟩]

@[default_target]
lean_lib Batteries
Expand Down

0 comments on commit 51c38e3

Please sign in to comment.