Import fgetc and listen from libc (where they actually reside) rather than the support libs

This commit is contained in:
Matthew Baulch 2020-06-21 15:24:45 +10:00
parent 6505be6c06
commit 916c3e7090
2 changed files with 2 additions and 2 deletions

View File

@ -31,7 +31,7 @@ prim_fileErrno : PrimIO Int
prim__readLine : FilePtr -> PrimIO (Ptr String)
%foreign support "idris2_readChars"
prim__readChars : Int -> FilePtr -> PrimIO (Ptr String)
%foreign support "fgetc"
%foreign "C:fgetc,libc 6"
prim__readChar : FilePtr -> PrimIO Int
%foreign support "idris2_writeLine"
prim__writeLine : FilePtr -> String -> PrimIO Int

View File

@ -11,7 +11,7 @@ import Network.Socket.Data
export
socket_close : (sockdes : SocketDescriptor) -> PrimIO Int
%foreign "C:listen,libidris2_support"
%foreign "C:listen,libc 6"
export
socket_listen : (sockfd : SocketDescriptor) -> (backlog : Int) -> PrimIO Int