Skip to content

Commit

Permalink
Changing Nat to Int for FFI type on prim__channelGetWithTimeout.
Browse files Browse the repository at this point in the history
  • Loading branch information
Matthew-Mosior committed Jan 7, 2025
1 parent ef41d27 commit eddaf30
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions libs/base/System/Concurrency.idr
Original file line number Diff line number Diff line change
Expand Up @@ -186,7 +186,7 @@ prim__channelGet : Channel a -> PrimIO a
%foreign "scheme,chez:blodwen-channel-get-non-blocking"
prim__channelGetNonBlocking : Channel a -> PrimIO (Maybe a)
%foreign "scheme,chez:blodwen-channel-get-with-timeout"
prim__channelGetWithTimeout : Channel a -> Nat -> PrimIO (Maybe a)
prim__channelGetWithTimeout : Channel a -> Int -> PrimIO (Maybe a)
%foreign "scheme:blodwen-channel-put"
prim__channelPut : Channel a -> a -> PrimIO ()

Expand Down Expand Up @@ -223,7 +223,7 @@ channelGetNonBlocking chan = primIO (prim__channelGetNonBlocking chan)
partial
export
channelGetWithTimeout : HasIO io => (chan : Channel a) -> (milliseconds : Nat) -> io (Maybe a)
channelGetWithTimeout chan milliseconds = primIO (prim__channelGetWithTimeout chan milliseconds)
channelGetWithTimeout chan milliseconds = primIO (prim__channelGetWithTimeout chan (cast milliseconds))

||| Puts a value on the given channel.
|||
Expand Down

0 comments on commit eddaf30

Please sign in to comment.