Skip to content

Commit ec62338

Browse files
committed
Merge remote-tracking branch 'origin/master' into nightly-testing
2 parents 983ad45 + 05be7e6 commit ec62338

File tree

1 file changed

+1
-4
lines changed

1 file changed

+1
-4
lines changed

Cache/Hashing.lean

Lines changed: 1 addition & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -91,9 +91,6 @@ Computes the root hash, which mixes the hashes of the content of:
9191
* `lake-manifest.json`
9292
9393
and the hash of `Lean.githash`.
94-
95-
(We hash `Lean.githash` in case the toolchain changes even though `lean-toolchain` hasn't.
96-
This happens with the `lean-pr-testing-NNNN` toolchains when Lean 4 PRs are updated.)
9794
-/
9895
def getRootHash : CacheM UInt64 := do
9996
let mathlibDepPath := (← read).mathlibDepPath
@@ -103,7 +100,7 @@ def getRootHash : CacheM UInt64 := do
103100
mathlibDepPath / "lake-manifest.json"]
104101
let hashes ← rootFiles.mapM fun path =>
105102
hashFileContents <$> IO.FS.readFile path
106-
return hash (rootHashGeneration :: hash Lean.githash :: hashes)
103+
return hash (rootHashGeneration :: hashes)
107104

108105
/--
109106
Computes the hash of a file, which mixes:

0 commit comments

Comments
 (0)