Force/Delay need to be inlined in Builtins

Otherwise (especially in the case of delay) the argument might be
evaluated prematurely.
This commit is contained in:
Edwin Brady 2020-12-06 20:00:48 +00:00
parent 22a534f400
commit 63a46722ef

View File

@ -186,11 +186,11 @@ export partial
idris_crash : String -> a
idris_crash = prim__crash _
public export
public export %inline
delay : a -> Lazy a
delay x = Delay x
public export
public export %inline
force : Lazy a -> a
force x = Force x