src/HOL/Complex/Complex_Main.thy
changeset 15131 c69542757a4d
parent 13984 e055ba9020eb
child 15140 322485b816ac
--- a/src/HOL/Complex/Complex_Main.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Complex/Complex_Main.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -6,6 +6,8 @@
 
 header{*Comprehensive Complex Theory*}
 
-theory Complex_Main = CLim:
+theory Complex_Main
+import CLim
+begin
 
 end