Agda
Safe HaskellNone
LanguageHaskell2010

Agda.Compiler.Backend

Description

Interface for compiler backend writers.

Synopsis

Documentation

data Recompile menv mod Source #

Constructors

Recompile menv 
Skip mod 

data IsMain Source #

Constructors

IsMain 
NotMain 

Instances

Instances details
Monoid IsMain Source # 
Instance details

Defined in Agda.Syntax.Common

Semigroup IsMain Source #

Conjunctive semigroup (NotMain is absorbing).

Instance details

Defined in Agda.Syntax.Common

Show IsMain Source # 
Instance details

Defined in Agda.Syntax.Common

Eq IsMain Source # 
Instance details

Defined in Agda.Syntax.Common

Methods

(==) :: IsMain -> IsMain -> Bool #

(/=) :: IsMain -> IsMain -> Bool #

type Flag opts = opts -> OptM opts Source #

f :: Flag opts is an action on the option record that results from parsing an option. f opts produces either an error message or an updated options record

data CheckResult where Source #

The result and associated parameters of a type-checked file, when invoked directly via interaction or a backend. Note that the constructor is not exported.

Bundled Patterns

pattern CheckResult :: Interface -> Set TCWarning -> ModuleCheckMode -> Source -> CheckResult

Flattened unidirectional pattern for CheckResult for destructuring inside the ModuleInfo field.

callBackend :: BackendName -> IsMain -> CheckResult -> TCM () Source #

Call the compilerMain function of the given backend.

callBackendInteractTop :: BackendName -> String -> CommandM () Source #

Call the backendInteractTop function of the given backend.

callBackendInteractHole :: BackendName -> String -> InteractionId -> Range -> String -> CommandM () Source #

Call the backendInteractHole function of the given backend.