Skip to content

Commit 14f2585

Browse files
authored
feat: use 'lake test' (#787)
* feat: use 'lake test' * add lake build step
1 parent 9e1609d commit 14f2585

File tree

4 files changed

+55
-13
lines changed

4 files changed

+55
-13
lines changed

.github/workflows/build.yml

+1-1
Original file line numberDiff line numberDiff line change
@@ -29,7 +29,7 @@ jobs:
2929

3030
- name: test batteries
3131
if: steps.build.outcome == 'success'
32-
run: make test
32+
run: lake test
3333

3434
- name: lint batteries
3535
if: steps.build.outcome == 'success'

GNUmakefile

+2-12
Original file line numberDiff line numberDiff line change
@@ -1,22 +1,12 @@
1-
TESTS = $(wildcard test/*.lean)
2-
3-
# Ensure that panics actually cause the tests to fail
4-
export LEAN_ABORT_ON_PANIC=1
5-
61
.PHONY: all build test lint
72

83
all: build test
94

105
build:
116
lake build
127

13-
# Find all .lean files in test and subdirectories, replace .lean with .run
14-
TESTS := $(shell find test -type f -name '*.lean' | sed 's/\.lean$$/.run/')
15-
16-
test: $(TESTS)
17-
18-
%.run: build
19-
lake env lean $(@:.run=.lean)
8+
test:
9+
lake test
2010

2111
lint:
2212
lake exe runLinter

lakefile.lean

+4
Original file line numberDiff line numberDiff line change
@@ -20,3 +20,7 @@ lean_exe runLinter where
2020

2121
meta if get_config? doc |>.isSome then
2222
require «doc-gen4» from git "https://github.com/leanprover/doc-gen4" @ "main"
23+
24+
@[test_runner]
25+
lean_exe test where
26+
srcDir := "scripts"

scripts/test.lean

+48
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,48 @@
1+
/-
2+
Copyright (c) 2024 Kim Morrison. All rights reserved.
3+
Released under Apache 2.0 license as described in the file LICENSE.
4+
Authors: Kim Morrison
5+
-/
6+
open IO.Process
7+
open System
8+
9+
/--
10+
Run tests.
11+
12+
If no arguments are provided, run everything in the `test/` directory.
13+
14+
If arguments are provided, assume they are names of files in the `test/` directory,
15+
and just run those.
16+
-/
17+
def main (args : List String) : IO Unit := do
18+
-- We first run `lake build`, to ensure oleans are available.
19+
-- Alternatively, we could use `lake lean` below instead of `lake env lean`,
20+
-- but currently with parallelism this results in build jobs interfering with each other.
21+
_ ← (← IO.Process.spawn { cmd := "lake", args := #["build"] }).wait
22+
-- Collect test targets, either from the command line or by walking the `test/` directory.
23+
let targets ← match args with
24+
| [] => System.FilePath.walkDir "./test"
25+
| _ => pure <| (args.map fun t => mkFilePath [".", "test", t] |>.withExtension "lean") |>.toArray
26+
let existing ← targets.filterM fun t => do pure <| (← t.pathExists) && !(← t.isDir)
27+
-- Generate a `lake env lean` task for each test target.
28+
let tasks ← existing.mapM fun t => do
29+
IO.asTask do
30+
let out ← IO.Process.output
31+
{ cmd := "lake",
32+
args := #["env", "lean", t.toString],
33+
env := #[("LEAN_ABORT_ON_PANIC", "1")] }
34+
if out.exitCode = 0 then
35+
IO.println s!"Test succeeded: {t}"
36+
else
37+
IO.eprintln s!"Test failed: `lake env lean {t}` produced:"
38+
unless out.stdout.isEmpty do IO.eprintln out.stdout
39+
unless out.stderr.isEmpty do IO.eprintln out.stderr
40+
pure out.exitCode
41+
-- Wait on all the jobs and exit with 1 if any failed.
42+
let mut exitCode : UInt8 := 0
43+
for t in tasks do
44+
let e ← IO.wait t
45+
match e with
46+
| .ok 0 => pure ()
47+
| _ => exitCode := 1
48+
exit exitCode

0 commit comments

Comments
 (0)