Skip to content

Commit

Permalink
.
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Oct 2, 2024
1 parent 23c24c3 commit cd20dae
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -80,7 +80,7 @@ def widgetJsAllTarget (pkg : Package) (isDev : Bool) : FetchM (BuildJob (Array F
We must instead ensure that the cloud release is fetched first
so that this target does not build from scratch unnecessarily.
`afterReleaseAsync` guarantees this. -/
pkg.afterReleaseAsync $ deps.bindSync fun depInfo depTrace => do
pkg.afterBuildCacheAsync $ deps.bindSync fun depInfo depTrace => do
let traceFile := buildDir / "js" / "lake.trace"
let _ ← buildUnlessUpToDate? traceFile depTrace traceFile do
/- HACK: Ensure that NPM modules are installed before building TypeScript,
Expand Down
2 changes: 1 addition & 1 deletion lean-toolchain
Original file line number Diff line number Diff line change
@@ -1 +1 @@
leanprover/lean4:v4.12.0
leanprover/lean4:nightly-2024-10-02

0 comments on commit cd20dae

Please sign in to comment.