src/HOL/Power.thy
changeset 33364 2bd12592c5e8
parent 33274 b6ff7db522b5
child 35028 108662d50512
     1.1 --- a/src/HOL/Power.thy	Fri Oct 30 14:02:42 2009 +0100
     1.2 +++ b/src/HOL/Power.thy	Fri Oct 30 18:32:40 2009 +0100
     1.3 @@ -467,4 +467,13 @@
     1.4  
     1.5  declare power.power.simps [code]
     1.6  
     1.7 +code_modulename SML
     1.8 +  Power Arith
     1.9 +
    1.10 +code_modulename OCaml
    1.11 +  Power Arith
    1.12 +
    1.13 +code_modulename Haskell
    1.14 +  Power Arith
    1.15 +
    1.16  end