Skip to content

Commit 06352ca

Browse files
algebraic-devTwoFX
andcommitted
Update src/Std/Sync/Broadcast.lean
Co-authored-by: Markus Himmel <[email protected]>
1 parent 18e0fd0 commit 06352ca

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Std/Sync/Broadcast.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -560,8 +560,8 @@ def unsubscribe (ch : Broadcast.Receiver α) : IO Unit := do
560560
Note that if this function is called twice, each message will only arrive at exactly one invocation.
561561
-/
562562
partial def forAsync (f : α → BaseIO Unit) (ch : Broadcast.Receiver α)
563-
(prio : Task.Priority := .default) : BaseIO (Task Unit) := do
564-
ch.inner.forAsync f prio
563+
(prio : Task.Priority := .default) : BaseIO (Task Unit) := do
564+
ch.inner.forAsync f prio
565565

566566
instance [Inhabited α] : AsyncStream (Broadcast.Receiver α) (Option α) where
567567
next channel := channel.recvSelector

0 commit comments

Comments
 (0)