| author | wenzelm |
| Wed, 15 Oct 2008 21:45:02 +0200 | |
| changeset 28605 | 12d6087ec18c |
| parent 28335 | 25326092cf9a |
| child 28686 | 5d63184c10c7 |
| permissions | -rw-r--r-- |
(* ID: $Id$ Author: Florian Haftmann, TU Muenchen *) header {* Tests and examples for code generator *} theory Codegenerator imports ExecutableContent begin ML {* (*FIXME get rid of this*) nonfix union; nonfix inter; nonfix upto; *} export_code "RType.*" -- "workaround for cache problem" export_code * in SML module_name CodegenTest in OCaml module_name CodegenTest file - in Haskell file - ML {* infix union; infix inter; infix 4 upto; *} end