We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 18e0fd0 commit 06352caCopy full SHA for 06352ca
src/Std/Sync/Broadcast.lean
@@ -560,8 +560,8 @@ def unsubscribe (ch : Broadcast.Receiver α) : IO Unit := do
560
Note that if this function is called twice, each message will only arrive at exactly one invocation.
561
-/
562
partial def forAsync (f : α → BaseIO Unit) (ch : Broadcast.Receiver α)
563
- (prio : Task.Priority := .default) : BaseIO (Task Unit) := do
564
- ch.inner.forAsync f prio
+ (prio : Task.Priority := .default) : BaseIO (Task Unit) := do
+ ch.inner.forAsync f prio
565
566
instance [Inhabited α] : AsyncStream (Broadcast.Receiver α) (Option α) where
567
next channel := channel.recvSelector
0 commit comments