src/HOL/ex/Codegenerator.thy
author krauss
Thu, 17 May 2007 22:33:41 +0200
changeset 22999 c1ce129e6f9c
parent 22845 5f9138bcb3d7
child 23266 50f0a4f12ed3
permissions -rw-r--r--
Added unification case study (using new function package)

(*  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