| author | wenzelm | 
| Fri, 09 Jan 2009 19:41:33 +0100 | |
| changeset 29414 | 747c95f7bb7e | 
| parent 28663 | bd8438543bf2 | 
| child 29933 | 125d513d9e39 | 
| permissions | -rw-r--r-- | 
(* Title: HOL/ex/Codegenerator_Pretty.thy ID: $Id$ Author: Florian Haftmann, TU Muenchen *) header {* Simple examples for pretty numerals and such *} theory Codegenerator_Pretty imports ExecutableContent Code_Char Efficient_Nat begin declare isnorm.simps [code del] ML {* (*FIXME get rid of this*) nonfix union; nonfix inter; nonfix upto; *} 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