File tree Expand file tree Collapse file tree 1 file changed +6
-6
lines changed
Expand file tree Collapse file tree 1 file changed +6
-6
lines changed Original file line number Diff line number Diff line change @@ -22,15 +22,15 @@ This module provides buffered asynchronous I/O operations for efficient reading
2222-/
2323
2424/--
25- Interface for asynchronous reading operations
25+ Interface for asynchronous reading operations.
2626-/
27- class AsyncRead (α : Type ) (β : outParam Type ) where
27+ class AsyncRead (α : Type ) (β : Type ) where
2828 read : α → Async β
2929
3030/--
31- Interface for asynchronous writing operations
31+ Interface for asynchronous writing operations.
3232-/
33- class AsyncWrite (α : Type ) (β : outParam Type ) where
33+ class AsyncWrite (α : Type ) (β : Type ) where
3434 write : α → β → Async Unit
3535
3636 writeAll : α → Array β → Async Unit :=
@@ -40,9 +40,9 @@ class AsyncWrite (α : Type) (β : outParam Type) where
4040 fun _ => pure ()
4141
4242/--
43- Interface for asynchronous streaming with selector-based iteration
43+ Interface for asynchronous streaming with selector-based iteration.
4444-/
45- class AsyncStream (α : Type ) (β : outParam Type ) where
45+ class AsyncStream (α : Type ) (β : Type ) where
4646 next : α → Selector β
4747
4848 stop : α → IO Unit :=
You can’t perform that action at this time.
0 commit comments