src/HOL/Power.thy
changeset 52435 6646bb548c6b
parent 51263 31e786e0e6a7
child 53015 a1119cf551e8
--- a/src/HOL/Power.thy	Sun Jun 23 21:16:06 2013 +0200
+++ b/src/HOL/Power.thy	Sun Jun 23 21:16:07 2013 +0200
@@ -742,14 +742,8 @@
 
 declare power.power.simps [code]
 
-code_modulename SML
-  Power Arith
-
-code_modulename OCaml
-  Power Arith
-
-code_modulename Haskell
-  Power Arith
+code_identifier
+  code_module Power \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith
 
 end