src/HOL/Complex_Main.thy
changeset 63571 aee0d92995b6
parent 63570 1826a90b9cbc
child 73411 1f1366966296
--- a/src/HOL/Complex_Main.thy	Sun Jul 31 18:05:20 2016 +0200
+++ b/src/HOL/Complex_Main.thy	Sun Jul 31 19:09:21 2016 +0200
@@ -2,12 +2,8 @@
 
 theory Complex_Main
 imports
-  Main
-  Real
   Complex
-  Transcendental
   MacLaurin
-  Deriv
 begin
 
 end