Skip to content

Commit

Permalink
Apply suggestions from code review
Browse files Browse the repository at this point in the history
Co-authored-by: Markus Himmel <[email protected]>
  • Loading branch information
hargoniX and TwoFX authored Jan 13, 2025
1 parent f1e506a commit aa17466
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion src/Std/Internal/Async/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -32,7 +32,7 @@ instance : Pure AsyncTask where
/--
Create a new `AsyncTask` that will run after `x` has finished.
If `x`:
- errors, return an `AsyncTask` that reolves to the error.
- errors, return an `AsyncTask` that resolves to the error.
- succeeds, run `f` on the result of `x` and return the `AsyncTask` produced by `f`.
-/
@[inline]
Expand Down
2 changes: 1 addition & 1 deletion src/Std/Internal/Async/Timer.lean
Original file line number Diff line number Diff line change
Expand Up @@ -56,7 +56,7 @@ def reset (s : Sleep) : IO Unit :=

/--
If:
- `s` is still running this stops `s` without resolving any remaing `AsyncTask` that were created
- `s` is still running this stops `s` without resolving any remaining `AsyncTask`s that were created
through `wait`. Note that if another `AsyncTask` is binding on any of these it is going hang
forever without further intervention.
- `s` is not yet or not anymore running this is a no-op.
Expand Down

0 comments on commit aa17466

Please sign in to comment.