src/HOL/Hyperreal/Poly.thy
changeset 15131 c69542757a4d
parent 14435 9e22eeccf129
child 15140 322485b816ac
--- a/src/HOL/Hyperreal/Poly.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Hyperreal/Poly.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -8,8 +8,9 @@
 
 header{*Univariate Real Polynomials*}
 
-theory Poly = Transcendental:
-
+theory Poly
+import Transcendental
+begin
 
 text{*Application of polynomial as a real function.*}