src/HOL/Hyperreal/Lim.thy
changeset 15131 c69542757a4d
parent 15086 e6a2a98d5ef5
child 15140 322485b816ac
--- a/src/HOL/Hyperreal/Lim.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Hyperreal/Lim.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -7,7 +7,9 @@
 
 header{*Limits, Continuity and Differentiation*}
 
-theory Lim = SEQ + RealDef:
+theory Lim
+import SEQ RealDef
+begin
 
 text{*Standard and Nonstandard Definitions*}