src/HOL/Int.thy
changeset 52435 6646bb548c6b
parent 51994 82cc2aeb7d13
child 53065 de1816a7293e
--- a/src/HOL/Int.thy	Sun Jun 23 21:16:06 2013 +0200
+++ b/src/HOL/Int.thy	Sun Jun 23 21:16:07 2013 +0200
@@ -1614,14 +1614,8 @@
 
 text {* Serializer setup *}
 
-code_modulename SML
-  Int Arith
-
-code_modulename OCaml
-  Int Arith
-
-code_modulename Haskell
-  Int Arith
+code_identifier
+  code_module Int \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith
 
 quickcheck_params [default_type = int]