src/HOL/Library/Univ_Poly.thy
changeset 28562 4e74209f113e
parent 27487 c8a6ce181805
child 28823 dcbef866c9e2
--- a/src/HOL/Library/Univ_Poly.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/Library/Univ_Poly.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -72,7 +72,7 @@
 
 definition (in semiring_0)
   divides :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool"  (infixl "divides" 70) where
-  [code func del]: "p1 divides p2 = (\<exists>q. poly p2 = poly(p1 *** q))"
+  [code del]: "p1 divides p2 = (\<exists>q. poly p2 = poly(p1 *** q))"
 
     --{*order of a polynomial*}
 definition (in ring_1) order :: "'a => 'a list => nat" where