src/HOL/Library/Formal_Power_Series.thy
changeset 59667 651ea265d568
parent 58881 b9556a055632
child 59730 b7c394c7a619
--- a/src/HOL/Library/Formal_Power_Series.thy	Tue Mar 10 11:56:32 2015 +0100
+++ b/src/HOL/Library/Formal_Power_Series.thy	Tue Mar 10 15:20:40 2015 +0000
@@ -5,7 +5,7 @@
 section{* A formalization of formal power series *}
 
 theory Formal_Power_Series
-imports "~~/src/HOL/Number_Theory/Binomial"
+imports Complex_Main
 begin