src/HOL/ex/Codegenerator.thy
changeset 22845 5f9138bcb3d7
parent 22297 757ace95c4a0
child 23266 50f0a4f12ed3
--- a/src/HOL/ex/Codegenerator.thy	Sun May 06 21:49:44 2007 +0200
+++ b/src/HOL/ex/Codegenerator.thy	Sun May 06 21:50:17 2007 +0200
@@ -8,7 +8,7 @@
 imports ExecutableContent
 begin
 
-code_gen "*" (SML) (Haskell) (OCaml)
-code_gen (SML #) (Haskell -) (OCaml -)
+code_gen "*" in SML in OCaml file - in OCaml file -
+code_gen in SML in OCaml file - in OCaml file -
 
 end
\ No newline at end of file