Skip to content

Commit

Permalink
Merge pull request #2956 from FStarLang/guido_build
Browse files Browse the repository at this point in the history
Some build+test system tweaks
  • Loading branch information
mtzguido committed Jun 6, 2023
2 parents 211b0cc + e707a56 commit 17f2353
Show file tree
Hide file tree
Showing 12 changed files with 1,327 additions and 1,292 deletions.
19 changes: 16 additions & 3 deletions Makefile
Original file line number Diff line number Diff line change
Expand Up @@ -132,24 +132,37 @@ output:
+$(Q)$(MAKE) -C tests/ide/emacs accept
+$(Q)$(MAKE) -C tests/bug-reports output-accept

# This rule is meant to mimic what the docker based CI does, but it
# is not perfect. In particular it will not look for a diff on the
# snapshot, nor run the build-standalone script.
.PHONY: ci
ci:
+$(Q)FSTAR_HOME=$(CURDIR) $(MAKE) ci-pre
+$(Q)FSTAR_HOME=$(CURDIR) $(MAKE) ci-post

# This rule runs a CI job in a local container, exactly like is done for
# CI.
.PHONY: docker-ci
docker-ci:
docker build -f .docker/standalone.Dockerfile --build-arg CI_THREADS=$(shell nproc) .

.PHONY: ci-pre
ci-pre:
ci-pre: ci-rebootstrap ci-ocaml-test ci-ulib-in-fsharp

.PHONY: ci-rebootstrap
ci-rebootstrap:
+$(Q)$(MAKE) full-bootstrap FSTAR_BUILD_PROFILE=test

.PHONY: ci-ocaml-test
ci-ocaml-test: ci-rebootstrap
+$(Q)$(MAKE) -C src ocaml-unit-tests
+$(Q)$(MAKE) -C ulib ulib-in-fsharp #build ulibfs

.PHONY: ci-ulib-in-fsharp
ci-ulib-in-fsharp: ci-rebootstrap
+$(Q)$(MAKE) -C ulib ulib-in-fsharp

.PHONY: ci-post
ci-post: ci-uregressions
+if [ -n "${FSTAR_CI_UREGRESSIONS_ULONG}" ]; then $(MAKE) ci-uregressions-ulong; fi

.PHONY: ci-uregressions
ci-uregressions:
Expand Down
8 changes: 5 additions & 3 deletions examples/Makefile
Original file line number Diff line number Diff line change
Expand Up @@ -5,16 +5,18 @@ include Makefile.include
# These examples are excluded since the binary package can't verify
# them.

# Scheduling these first as some files take very long.
ALL_EXAMPLE_DIRS += layeredeffects
ALL_EXAMPLE_DIRS += dsls
ALL_EXAMPLE_DIRS += data_structures

ALL_EXAMPLE_DIRS += algorithms
ALL_EXAMPLE_DIRS += calc
ALL_EXAMPLE_DIRS += crypto
ALL_EXAMPLE_DIRS += data_structures
ALL_EXAMPLE_DIRS += demos
ALL_EXAMPLE_DIRS += doublylinkedlist
ALL_EXAMPLE_DIRS += dsls
ALL_EXAMPLE_DIRS += generic
ALL_EXAMPLE_DIRS += indexed_effects
ALL_EXAMPLE_DIRS += layeredeffects
ALL_EXAMPLE_DIRS += low-mitls-experiments
ALL_EXAMPLE_DIRS += maths
ALL_EXAMPLE_DIRS += metatheory
Expand Down
38 changes: 19 additions & 19 deletions examples/tactics/Canon.fst
Original file line number Diff line number Diff line change
Expand Up @@ -60,25 +60,25 @@ let lem4 (a b c : int) =
(* The following tests should pass, but it's too slow to run them on every regression build, *)
(* and the previous ones are probably enough *)

let lem5 (a b c d e : int) =
assert
((a+b+c+d+e)*(a+b+c+d+e) ==
a * a + a * b + a * c + a * d + a * e
+ b * a + b * b + b * c + b * d + b * e
+ c * a + c * b + c * c + c * d + c * e
+ d * a + d * b + d * c + d * d + d * e
+ e * a + e * b + e * c + e * d + e * e)
by check_canon ()

let lem6 (a b c d e : int) =
assert
((a+b+c+d+e)*(e+d+c+b+a) ==
a * a + a * b + a * c + a * d + a * e
+ b * a + b * b + b * c + b * d + b * e
+ c * a + c * b + c * c + c * d + c * e
+ d * a + d * b + d * c + d * d + d * e
+ e * a + e * b + e * c + e * d + e * e)
by check_canon ()
// let lem5 (a b c d e : int) =
// assert
// ((a+b+c+d+e)*(a+b+c+d+e) ==
// a * a + a * b + a * c + a * d + a * e
// + b * a + b * b + b * c + b * d + b * e
// + c * a + c * b + c * c + c * d + c * e
// + d * a + d * b + d * c + d * d + d * e
// + e * a + e * b + e * c + e * d + e * e)
// by check_canon ()
//
// let lem6 (a b c d e : int) =
// assert
// ((a+b+c+d+e)*(e+d+c+b+a) ==
// a * a + a * b + a * c + a * d + a * e
// + b * a + b * b + b * c + b * d + b * e
// + c * a + c * b + c * c + c * d + c * e
// + d * a + d * b + d * c + d * d + d * e
// + e * a + e * b + e * c + e * d + e * e)
// by check_canon ()

let lem7 (a b c d : int) =
assert
Expand Down
1,974 changes: 987 additions & 987 deletions ocaml/fstar-lib/generated/FStar_InteractiveHelpers_PostProcess.ml

Large diffs are not rendered by default.

33 changes: 19 additions & 14 deletions ocaml/fstar-lib/generated/FStar_Tactics_Derived.ml

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

Loading

0 comments on commit 17f2353

Please sign in to comment.