src/HOL/Power.thy
changeset 29608 564ea783ace8
parent 28131 3130d7b3149d
child 29978 33df3c4eb629
child 30240 5b25fee0362c
--- a/src/HOL/Power.thy	Wed Jan 21 18:37:44 2009 +0100
+++ b/src/HOL/Power.thy	Wed Jan 21 23:40:23 2009 +0100
@@ -11,7 +11,7 @@
 imports Nat
 begin
 
-class power = type +
+class power =
   fixes power :: "'a \<Rightarrow> nat \<Rightarrow> 'a"            (infixr "^" 80)
 
 subsection{*Powers for Arbitrary Monoids*}