src/HOL/Real/RComplete.thy
changeset 15131 c69542757a4d
parent 14641 79b7bd936264
child 15140 322485b816ac
--- a/src/HOL/Real/RComplete.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Real/RComplete.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -8,7 +8,9 @@
 
 header{*Completeness of the Reals; Floor and Ceiling Functions*}
 
-theory RComplete = Lubs + RealDef:
+theory RComplete
+import Lubs RealDef
+begin
 
 lemma real_sum_of_halves: "x/2 + x/2 = (x::real)"
 by simp