Skip to content

Commit

Permalink
Fix missing checks in stdlib test suite
Browse files Browse the repository at this point in the history
  • Loading branch information
SkySkimmer committed Dec 18, 2024
1 parent eafed8f commit 7a62178
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 1 deletion.
1 change: 1 addition & 0 deletions .gitignore
Original file line number Diff line number Diff line change
Expand Up @@ -97,6 +97,7 @@ test-suite/Datatypes.mli
test-suite/bug_10796.ml
test-suite/bug_10796.mli
test-suite/**/*.time
stdlib/test-suite/**/*.time

# `nix build` (through flake) symlink
result
Expand Down
3 changes: 3 additions & 0 deletions stdlib/test-suite/Makefile
Original file line number Diff line number Diff line change
Expand Up @@ -195,9 +195,12 @@ summary:
$(call summary_dir, "Success tests", success); \
$(call summary_dir, "Bugs tests", bugs); \
$(call summary_dir, "Output tests", output); \
$(call summary_dir, "Miscellaneous tests", misc); \
$(call summary_dir, "Complexity tests", complexity); \
$(call summary_dir, "Micromega tests", micromega); \
$(call summary_dir, "Module tests", modules); \
$(call summary_dir, "STM tests", stm); \
$(call summary_dir, "Ltac2 tests", ltac2); \
nb_success=`grep -e $(log_success) -r . -l --include="*.log" --exclude-dir=logs | wc -l`; \
nb_failure=`grep -e $(log_failure) -r . -l --include="*.log" --exclude-dir=logs | wc -l`; \
nb_tests=`expr $$nb_success + $$nb_failure`; \
Expand Down
2 changes: 1 addition & 1 deletion stdlib/test-suite/micromega/bug_14054.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ From Stdlib.Init Require Byte.
From Stdlib.Strings Require Byte.
From Stdlib Require Import ZifyClasses Lia.

Notation byte := Stdlib.Init.Byte.byte.
Notation byte := Corelib.Init.Byte.byte.

Module byte.
Definition unsigned(b: byte): Z := Z.of_N (Byte.to_N b).
Expand Down

0 comments on commit 7a62178

Please sign in to comment.