src/HOL/Word/WordDefinition.thy
changeset 30968 10fef94f40fc
parent 30952 7ab2716dd93b
child 30971 7fbebf75b3ef
--- a/src/HOL/Word/WordDefinition.thy	Thu Apr 23 12:17:51 2009 +0200
+++ b/src/HOL/Word/WordDefinition.thy	Thu Apr 23 12:17:51 2009 +0200
@@ -99,7 +99,7 @@
 
 subsection  "Arithmetic operations"
 
-instantiation word :: (len0) "{number, uminus, minus, plus, one, zero, times, Divides.div, power, ord, bit}"
+instantiation word :: (len0) "{number, uminus, minus, plus, one, zero, times, Divides.div, ord, bit}"
 begin
 
 definition
@@ -126,10 +126,6 @@
 definition
   word_mod_def: "a mod b = word_of_int (uint a mod uint b)"
 
-primrec power_word where
-  "(a\<Colon>'a word) ^ 0 = 1"
-  | "(a\<Colon>'a word) ^ Suc n = a * a ^ n"
-
 definition
   word_number_of_def: "number_of w = word_of_int w"
 
@@ -157,7 +153,7 @@
 
 instance ..
 
-end 
+end
 
 definition
   word_succ :: "'a :: len0 word => 'a word"