src/HOL/ex/Codegenerator.thy
author wenzelm
Tue, 10 Jul 2007 23:29:43 +0200
changeset 23719 ccd9cb15c062
parent 23266 50f0a4f12ed3
child 23811 b18557301bf9
permissions -rw-r--r--
more markup for inner and outer syntax; added enclose;

(*  ID:         $Id$
    Author:     Florian Haftmann, TU Muenchen
*)

header {* Tests and examples for code generator *}

theory Codegenerator
imports ExecutableContent
begin

code_gen "*" in SML in OCaml file - in OCaml file -
code_gen in SML in OCaml file - in OCaml file -

end