src/HOL/ex/Classpackage.thy
changeset 19888 2b4c09941e04
parent 19363 667b5ea637dd
child 19928 cb8472f4c5fd
--- a/src/HOL/ex/Classpackage.thy	Wed Jun 14 12:12:37 2006 +0200
+++ b/src/HOL/ex/Classpackage.thy	Wed Jun 14 12:13:12 2006 +0200
@@ -314,9 +314,9 @@
   "x = ((2::nat) \<otimes> \<one> \<otimes> 3, (2::int) \<otimes> \<one> \<otimes> \<div> 3, [1::nat, 2] \<otimes> \<one> \<otimes> [1, 2, 3])"
   "y = (2 :: int, \<div> 2 :: int) \<otimes> \<one> \<otimes> (3, \<div> 3)"
 
-code_generate "op \<otimes>" "\<one>" "inv"
-code_generate x
-code_generate y
+code_generate (ml, haskell) "op \<otimes>" "\<one>" "inv"
+code_generate (ml, haskell) x
+code_generate (ml, haskell) y
 
 code_serialize ml (-)