Agda-2.5.1: A dependently typed functional programming language and proof assistant

Safe HaskellNone
LanguageHaskell98

Agda.Compiler.MAlonzo.Compiler

Synopsis

Documentation

definition :: Maybe CoinductionKit -> Definition -> TCM [Decl] Source

Note that the INFINITY, SHARP and FLAT builtins are translated as follows (if a CoinductionKit is given):

  type Infinity a b = b

  sharp :: a -> a
  sharp x = x

  flat :: a -> a
  flat x = x

data CCEnv Source

Environment for naming of local variables. Invariant: reverse ccCxt ++ ccNameSupply

Constructors

CCEnv 

Fields

ccNameSupply :: NameSupply

Supply of fresh names

ccCxt :: CCContext

Names currently in scope

initCCEnv :: CCEnv Source

Initial environment for expression generation.

lookupIndex :: Int -> CCContext -> Name Source

Term variables are de Bruijn indices.

freshNames :: Int -> ([Name] -> CC a) -> CC a Source

intros :: Int -> ([Name] -> CC a) -> CC a Source

Introduce n variables into the context.

term :: TTerm -> CC Exp Source

Extract Agda term to Haskell expression. Erased arguments are extracted as (). Types are extracted as ().

alt :: Int -> TAlt -> CC Alt Source

tvaldecl Source

Arguments

:: QName 
-> Induction

Is the type inductive or coinductive?

-> Nat 
-> Nat 
-> [ConDecl] 
-> Maybe Clause 
-> [Decl]