Skip to content

Commit

Permalink
chore: build lean4checker with current toolchain (#8669)
Browse files Browse the repository at this point in the history
After leanprover/lean4#2766 lands, the git hash of will be embedded in every olean. `lean4checker` will thus reject oleans unless it was compiled on the same toolchain as they were!

We may want to relax this later, but for now, since we are building `lean4checker` in CI anyway, let's just make sure it is on the same toolchain as mathlib.

Co-authored-by: Scott Morrison <[email protected]>
  • Loading branch information
kim-em and kim-em committed Nov 28, 2023
1 parent 2577ef7 commit 16f64a1
Show file tree
Hide file tree
Showing 4 changed files with 12 additions and 0 deletions.
3 changes: 3 additions & 0 deletions .github/workflows/bors.yml
Original file line number Diff line number Diff line change
Expand Up @@ -261,6 +261,9 @@ jobs:
git clone https://github.com/leanprover/lean4checker
cd lean4checker
git checkout toolchain/v4.3.0-rc2
# Now that the git hash is embedded in each olean,
# we need to compile lean4checker on the same toolchain
cp ../lean-toolchain .
lake build
./test.sh
cd ..
Expand Down
3 changes: 3 additions & 0 deletions .github/workflows/build.yml
Original file line number Diff line number Diff line change
Expand Up @@ -268,6 +268,9 @@ jobs:
git clone https://github.com/leanprover/lean4checker
cd lean4checker
git checkout toolchain/v4.3.0-rc2
# Now that the git hash is embedded in each olean,
# we need to compile lean4checker on the same toolchain
cp ../lean-toolchain .
lake build
./test.sh
cd ..
Expand Down
3 changes: 3 additions & 0 deletions .github/workflows/build.yml.in
Original file line number Diff line number Diff line change
Expand Up @@ -247,6 +247,9 @@ jobs:
git clone https://github.com/leanprover/lean4checker
cd lean4checker
git checkout toolchain/v4.3.0-rc2
# Now that the git hash is embedded in each olean,
# we need to compile lean4checker on the same toolchain
cp ../lean-toolchain .
lake build
./test.sh
cd ..
Expand Down
3 changes: 3 additions & 0 deletions .github/workflows/build_fork.yml
Original file line number Diff line number Diff line change
Expand Up @@ -265,6 +265,9 @@ jobs:
git clone https://github.com/leanprover/lean4checker
cd lean4checker
git checkout toolchain/v4.3.0-rc2
# Now that the git hash is embedded in each olean,
# we need to compile lean4checker on the same toolchain
cp ../lean-toolchain .
lake build
./test.sh
cd ..
Expand Down

0 comments on commit 16f64a1

Please sign in to comment.