src/HOL/ex/Codegenerator.thy
author haftmann
Mon, 13 Aug 2007 21:22:37 +0200
changeset 24249 1f60b45c5f97
parent 24195 7d1a16c77f7c
child 24348 c708ea5b109a
permissions -rw-r--r--
renamed keyword "to" to "module_name"
haftmann@19281
     1
(*  ID:         $Id$
haftmann@19281
     2
    Author:     Florian Haftmann, TU Muenchen
haftmann@19281
     3
*)
haftmann@19281
     4
haftmann@21877
     5
header {* Tests and examples for code generator *}
haftmann@19281
     6
haftmann@19281
     7
theory Codegenerator
haftmann@21911
     8
imports ExecutableContent
haftmann@19281
     9
begin
haftmann@19281
    10
haftmann@24249
    11
code_gen "*" in SML module_name CodegenTest
haftmann@23811
    12
  in OCaml file -
haftmann@23811
    13
  in Haskell file -
haftmann@19281
    14
wenzelm@23266
    15
end