Skip to content

Commit e6a94e7

Browse files
committed
fix: coehead o coedep
1 parent 228fa2b commit e6a94e7

File tree

2 files changed

+5
-5
lines changed

2 files changed

+5
-5
lines changed

src/Std/Sync/StreamMap.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -35,8 +35,8 @@ inductive AnyAsyncStream (α : Type) where
3535
def 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
/--
4242
A map container that associates string keys with async streams.

tests/lean/run/async_streammap.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff 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)

0 commit comments

Comments
 (0)