src/HOL/Polynomial.thy
changeset 29664 6146e275e8af
parent 29660 d59918e668b7
parent 29654 24e73987bfe2
child 29668 33ba3faeaa0e
--- a/src/HOL/Polynomial.thy	Tue Jan 27 22:39:41 2009 -0800
+++ b/src/HOL/Polynomial.thy	Wed Jan 28 06:03:46 2009 -0800
@@ -6,7 +6,7 @@
 header {* Univariate Polynomials *}
 
 theory Polynomial
-imports Plain SetInterval
+imports Plain SetInterval Main
 begin
 
 subsection {* Definition of type @{text poly} *}