mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-01 09:49:24 +03:00
Update API test for new Codegen fields
This commit is contained in:
parent
94088bea80
commit
6c319dbcaf
@ -13,7 +13,7 @@ execute : Ref Ctxt Defs -> (execDir : String) -> ClosedTerm -> Core ()
|
||||
execute defs dir term = do coreLift $ putStrLn "Maybe in an hour."
|
||||
|
||||
lazyCodegen : Codegen
|
||||
lazyCodegen = MkCG compile execute
|
||||
lazyCodegen = MkCG compile execute Nothing Nothing
|
||||
|
||||
main : IO ()
|
||||
main = mainWithCodegens [("lazy", lazyCodegen)]
|
||||
|
Loading…
Reference in New Issue
Block a user