Skip to content

Commit

Permalink
bench 8.18 vs 8.17
Browse files Browse the repository at this point in the history
  • Loading branch information
SkySkimmer committed Oct 16, 2023
1 parent 49fce3a commit 4b750f6
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions dev/bench/bench.sh
Original file line number Diff line number Diff line change
Expand Up @@ -72,8 +72,8 @@ check_variable () {
: "${coq_opam_packages:=coq-bignums coq-hott coq-performance-tests-lite coq-engine-bench-lite coq-mathcomp-ssreflect coq-mathcomp-fingroup coq-mathcomp-algebra coq-mathcomp-solvable coq-mathcomp-field coq-mathcomp-character coq-mathcomp-odd-order coq-math-classes coq-corn coq-compcert coq-equations coq-metacoq-template coq-metacoq-pcuic coq-metacoq-safechecker coq-metacoq-erasure coq-metacoq-translations coq-color coq-coqprime coq-coqutil coq-bedrock2 coq-rewriter coq-fiat-core coq-fiat-parsers coq-fiat-crypto-with-bedrock coq-unimath coq-coquelicot coq-iris-examples coq-verdi coq-verdi-raft coq-fourcolor coq-rewriter-perf-SuperFast coq-perennial coq-vst coq-category-theory}"
: "${coq_native:=}"

: "${new_coq_commit:=$(git rev-parse HEAD^2)}"
: "${old_coq_commit:=$(git merge-base HEAD^1 $new_coq_commit)}"
: "${new_coq_commit:=$(git rev-parse V8.18.0)}"
: "${old_coq_commit:=336b7fc9bcd7e0a5671a6724c7112d775369ef9f}"

new_ocaml_switch=ocaml-base-compiler.$new_ocaml_version
old_ocaml_switch=ocaml-base-compiler.$old_ocaml_version
Expand Down

0 comments on commit 4b750f6

Please sign in to comment.