mirror of
https://github.com/idris-lang/Idris2.git
synced 2025-01-03 00:55:00 +03:00
Import fgetc and listen from libc (where they actually reside) rather than the support libs
This commit is contained in:
parent
6505be6c06
commit
916c3e7090
@ -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
|
||||
|
@ -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
|
||||
|
||||
|
Loading…
Reference in New Issue
Block a user