mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-28 11:05:17 +03:00
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:
parent
22a534f400
commit
63a46722ef
@ -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
|
||||
|
||||
|
Loading…
Reference in New Issue
Block a user