File tree Expand file tree Collapse file tree 2 files changed +5
-5
lines changed
Expand file tree Collapse file tree 2 files changed +5
-5
lines changed Original file line number Diff line number Diff line change @@ -35,8 +35,8 @@ inductive AnyAsyncStream (α : Type) where
3535def AnyAsyncStream.getSelector : AnyAsyncStream α → Selector α × IO Unit
3636 | AnyAsyncStream.mk stream => (AsyncStream.next stream, AsyncStream.stop stream)
3737
38- instance [AsyncStream t α] : CoeHead t (AnyAsyncStream α) where
39- coe := AnyAsyncStream.mk
38+ instance [AsyncStream t α] : CoeDep t x (AnyAsyncStream α) where
39+ coe := AnyAsyncStream.mk x
4040
4141/--
4242A map container that associates string keys with async streams.
Original file line number Diff line number Diff line change @@ -10,9 +10,9 @@ def testSimpleMessages : Async Unit := do
1010 let channelC ← Std.Channel.new (α := Nat)
1111
1212 let channel := Std.StreamMap.ofArray #[
13- ("a" , .mk channelA),
14- ("b" , .mk channelB),
15- ("c" , .mk channelC),
13+ ("a" , channelA),
14+ ("b" , channelB),
15+ ("c" , channelC),
1616 ]
1717
1818 await (← channelC.send 1 )
You can’t perform that action at this time.
0 commit comments