File tree Expand file tree Collapse file tree 1 file changed +1
-4
lines changed Expand file tree Collapse file tree 1 file changed +1
-4
lines changed Original file line number Diff line number Diff line change @@ -91,9 +91,6 @@ Computes the root hash, which mixes the hashes of the content of:
91
91
* `lake-manifest.json`
92
92
93
93
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.)
97
94
-/
98
95
def getRootHash : CacheM UInt64 := do
99
96
let mathlibDepPath := (← read).mathlibDepPath
@@ -103,7 +100,7 @@ def getRootHash : CacheM UInt64 := do
103
100
mathlibDepPath / "lake-manifest.json" ]
104
101
let hashes ← rootFiles.mapM fun path =>
105
102
hashFileContents <$> IO.FS.readFile path
106
- return hash (rootHashGeneration :: hash Lean.githash :: hashes)
103
+ return hash (rootHashGeneration :: hashes)
107
104
108
105
/--
109
106
Computes the hash of a file, which mixes:
You can’t perform that action at this time.
0 commit comments