Skip to content

Commit

Permalink
Merge pull request #106 from mhuisi/lean-pr-testing-7087
Browse files Browse the repository at this point in the history
chore: adapt for leanprover/lean4#7087
  • Loading branch information
kim-em authored Feb 23, 2025
2 parents 3011328 + 95d1fcf commit 6b234dc
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions ProofWidgets/Cancellable.lean
Original file line number Diff line number Diff line change
Expand Up @@ -34,9 +34,9 @@ def mkCancellable [RpcEncodable β] (handler : α → RequestM (RequestTask β))
α → RequestM (RequestTask RequestId) := fun a => do
RequestM.asTask do
let t ← handler a
let t' := t.map (·.map rpcEncode)
let t' := t.mapCheap (·.map rpcEncode)
runningRequests.modifyGet fun (id, m) =>
(id, (id+1, m.insert id ⟨t', IO.cancel t⟩))
(id, (id+1, m.insert id ⟨t'.task, t.cancel⟩))

/-- Cancel the request with ID `rid`.
Does nothing if `rid` is invalid. -/
Expand Down

0 comments on commit 6b234dc

Please sign in to comment.