src/HOL/Power.thy
changeset 33364 2bd12592c5e8
parent 33274 b6ff7db522b5
child 35028 108662d50512
--- a/src/HOL/Power.thy	Fri Oct 30 14:02:42 2009 +0100
+++ b/src/HOL/Power.thy	Fri Oct 30 18:32:40 2009 +0100
@@ -467,4 +467,13 @@
 
 declare power.power.simps [code]
 
+code_modulename SML
+  Power Arith
+
+code_modulename OCaml
+  Power Arith
+
+code_modulename Haskell
+  Power Arith
+
 end