src/HOL/Real/RealPow.thy
changeset 14269 502a7c95de73
parent 14268 5cf13e80be0e
child 14288 d149e3cbdb39
--- a/src/HOL/Real/RealPow.thy	Thu Nov 27 10:47:55 2003 +0100
+++ b/src/HOL/Real/RealPow.thy	Fri Nov 28 12:09:37 2003 +0100
@@ -6,10 +6,7 @@
 
 *)
 
-theory RealPow = RealAbs:
-
-(*belongs to theory RealAbs*)
-lemmas [arith_split] = abs_split
+theory RealPow = RealArith:
 
 instance real :: power ..