src/HOL/Algebra/UnivPoly.thy
changeset 14553 4740fc2da7bb
parent 14399 dc677b35e54f
child 14577 dbb95b825244
--- a/src/HOL/Algebra/UnivPoly.thy	Tue Apr 13 10:45:35 2004 +0200
+++ b/src/HOL/Algebra/UnivPoly.thy	Tue Apr 13 13:53:54 2004 +0200
@@ -9,6 +9,19 @@
 
 section {* Univariate Polynomials *}
 
+text {*
+  Polynomials are formalised as modules with additional operations for 
+  extracting coefficients from polynomials and for obtaining monomials 
+  from coefficients and exponents (record @{text "up_ring"}).
+  The carrier set is 
+  a set of bounded functions from Nat to the coefficient domain.  
+  Bounded means that these functions return zero above a certain bound 
+  (the degree).  There is a chapter on the formalisation of polynomials 
+  in my PhD thesis (http://www4.in.tum.de/\~{}ballarin/publications/), 
+  which was implemented with axiomatic type classes.  This was later
+  ported to Locales.
+*}
+
 subsection {* The Constructor for Univariate Polynomials *}
 
 (* Could alternatively use locale ...