src/HOL/Power.thy
changeset 15131 c69542757a4d
parent 15066 d2f2b908e0a4
child 15140 322485b816ac
--- a/src/HOL/Power.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Power.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -7,7 +7,9 @@
 
 header{*Exponentiation and Binomial Coefficients*}
 
-theory Power = Divides:
+theory Power
+import Divides
+begin
 
 subsection{*Powers for Arbitrary Semirings*}