src/HOL/Real/RComplete.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15234 ec91a90c604e
--- a/src/HOL/Real/RComplete.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Real/RComplete.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -9,7 +9,7 @@
 header{*Completeness of the Reals; Floor and Ceiling Functions*}
 
 theory RComplete
-import Lubs RealDef
+imports Lubs RealDef
 begin
 
 lemma real_sum_of_halves: "x/2 + x/2 = (x::real)"