src/HOL/Groups.thy
changeset 52435 6646bb548c6b
parent 52289 83ce5d2841e7
child 54147 97a8ff4e4ac9
--- a/src/HOL/Groups.thy	Sun Jun 23 21:16:06 2013 +0200
+++ b/src/HOL/Groups.thy	Sun Jun 23 21:16:07 2013 +0200
@@ -1359,14 +1359,8 @@
 by (auto intro: add_strict_right_mono add_strict_left_mono
   add_less_le_mono add_le_less_mono add_strict_mono)
 
-code_modulename SML
-  Groups Arith
-
-code_modulename OCaml
-  Groups Arith
-
-code_modulename Haskell
-  Groups Arith
+code_identifier
+  code_module Groups \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith
 
 
 text {* Legacy *}