Epic

How to install latest development version

The latest version of the epic backend needs some patches for epic before it can be merged into the Agda-tree. The following steps are needed to install. Install new Epic

$ git clone https://github.com/ollef/EpiVM.git
$ cd EpiVM
$ cabal install

Our darcs patch is located at http://web.student.chalmers.se/~danig/agda/ so download the latest (we haven't tested to merge yet so some conflict may occur, send an email and we will hopefully fix it).

Small example using the patch to standard library:

 module Test1 where

 open import Data.List hiding (_++_)
 open import Data.Unit
 open import Data.String
 open import Data.Nat
 open import Function
 open import IO.Epic.Strict

 stuff : String
 stuff = unlines
   $ "line 1"
   ∷ "line 2"
   ∷ "line 3"
   ∷ "line 4"
   ∷ [] -- cons for list

 main : IO ⊤ -- Unit
 main =
   getContents            >>= \ c    ->
   putStr c               >>= \ _    ->
   writeFile "temp" stuff >>= \ _    ->
   readFile  "temp"       >>= \ file ->
   putStr (fromList (toList file))

Epic compiler backend.

A new backend for Agda to compile to Epic has been created. Epic is a language used by Idris and Epigram made by Edwin Brady. Almost all of Agda should work when using this backend, but it needs more testing. It should be noted that this is very much experimental code.

There is a new pragma for giving the Epic code for postulated definitions. The Epic code given can then contain the definition itself, or use a foreign call to call a C function. The pragma is {-# COMPILED_EPIC def code #-} and works similar to the COMPILED pragma but instead of expecting Haskell code, it expects Epic code. The code includes function arguments, return type and the function body. Note that def is the name of an Agda definition, which will be translated to a valid Epic name automatically.

The Epic backend supports Agda's primitive pragma for primitive functions that are defined (with the same name) in the AgdaPrelude.e (Agda/src/data/EpicInclude/) file.

Usage: > agda --epic --epic-flag=<EPIC-FLAG> --compile-dir=<DIR> <FILE>.agda

A new directory, Epic, will be created in the compile-dir (default: the project root), containing the file main.e with the Epic source code. The compiler will also do a system call running the Epic compiler on that file, passing any epic-flags to Epic in the order of their appearance.

The compilation requires a definition of main, which should be of type IO Unit. Currently IO A actions are represented in Epic as functions from Unit to A. Because of this the main function is applied a single unit.

Here follows how to define the IO monad:

 
  postulate
    IO      : Set -> Set
    return  : {A : Set} -> A -> IO A
    _>>=_   : {A B : Set} -> IO A -> (A -> IO B) -> IO B

  {-# COMPILED_EPIC return (u1 : Unit, a : Any) -> Any = ioreturn(a) #-}
  {-# COMPILED_EPIC _>>=_ (u1 : Unit, u2 : Unit, x : Any, f : Any) -> Any = iobind(x,f) #-}

ioreturn and iobind are Epic functions defined in AgdaPrelude.e which is always included. This is how IO is defined in the standard library (IO.Primitive). We only need to add the new COMPILED_EPIC pragmas.

The backend supports the {-# BUILTIN #-} pragma, which can be used e.g. to get Natural numbers and their operations to be represented more efficiently as BigInts and operations on them in Epic.

By default the backend will remove forced constructor arguments. Pattern matching on forced variables will be rewritten so that it doesn't use the forced variable. This optmization can be disabled by using the flag --no-forcing.

All types that looks like Nats after forced constructor arguments have been removed - i.e. if they have two constructors: one with no arguments and one with a recursive argument - will be represented as BigInts. This applies to the standard Fin type for example.

Compilation using Epic requires a few libraries. Particularly gcc, the Boehm garbage collector and the GNU MP library. For more information, check out Epic's homepage: http://www.cs.st-andrews.ac.uk/~eb/epic.php

Link to report: http://web.student.chalmers.se/~danig/report.pdf

Page last modified on April 27, 2011, at 02:15 pm
Powered by PmWiki