Skip to content

Commit 4f43a7c

Browse files
committed
feat: run tests in CI
1 parent 6853e4c commit 4f43a7c

File tree

3 files changed

+8
-0
lines changed

3 files changed

+8
-0
lines changed

.github/workflows/build.yml

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -56,6 +56,9 @@ jobs:
5656
- name: Build demos
5757
run: lake build ProofWidgets.Demos
5858

59+
- name: Run tests
60+
run: lake test
61+
5962
- name: Create GitHub release for tag (Ubuntu)
6063
if: github.ref_type == 'tag' && matrix.os == 'ubuntu-latest'
6164
uses: softprops/action-gh-release@v2

lakefile.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -101,3 +101,7 @@ lean_lib ProofWidgets where
101101
lean_lib ProofWidgets.Demos where
102102
needs := #[widgetJsAll]
103103
globs := #[.submodules `ProofWidgets.Demos]
104+
105+
@[test_driver]
106+
lean_lib test where
107+
globs := #[.submodules `test]

test/checkh.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -3,6 +3,7 @@ import ProofWidgets.Extra.CheckHighlight
33
/-- info: Decidable.em (p : Prop) : p ∨ ¬p -/
44
#guard_msgs in
55
#checkh Decidable.em
6+
67
/-- info: Decidable.em (p : Prop) [Decidable p] : p ∨ ¬p -/
78
#guard_msgs in
89
#checkh' Decidable.em

0 commit comments

Comments
 (0)