[ fix ] custom backend doc

The type Codegen was changed in #2594.
This commit is contained in:
Guillaume Allais 2022-07-25 20:55:42 +01:00 committed by G. Allais
parent 572a4c74d6
commit 4a465ac21e

View File

@ -27,14 +27,20 @@ Now create a file containing
import Core.Context
import Compiler.Common
import Idris.Driver
import Idris.Syntax
compile : Ref Ctxt Defs -> (tmpDir : String) -> (execDir : String) ->
ClosedTerm -> (outfile : String) -> Core (Maybe String)
compile defs tmp dir term file = do coreLift $ putStrLn "I'd rather not."
pure $ Nothing
compile :
Ref Ctxt Defs -> Ref Syn SyntaxInfo ->
(tmpDir : String) -> (execDir : String) ->
ClosedTerm -> (outfile : String) -> Core (Maybe String)
compile syn defs tmp dir term file
= do coreLift $ putStrLn "I'd rather not."
pure Nothing
execute : Ref Ctxt Defs -> (execDir : String) -> ClosedTerm -> Core ()
execute defs dir term = do coreLift $ putStrLn "Maybe in an hour."
execute :
Ref Ctxt Defs -> Ref Syn SyntaxInfo ->
(execDir : String) -> ClosedTerm -> Core ()
execute defs syn dir term = do coreLift $ putStrLn "Maybe in an hour."
lazyCodegen : Codegen
lazyCodegen = MkCG compile execute Nothing Nothing