src/HOL/Library/Univ_Poly.thy
changeset 37765 26bdfb7b680b
parent 37598 893dcabf0c04
child 37860 2ae085b07f2f
     1.1 --- a/src/HOL/Library/Univ_Poly.thy	Mon Jul 12 08:58:12 2010 +0200
     1.2 +++ b/src/HOL/Library/Univ_Poly.thy	Mon Jul 12 08:58:13 2010 +0200
     1.3 @@ -71,7 +71,7 @@
     1.4  
     1.5  definition (in semiring_0)
     1.6    divides :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool"  (infixl "divides" 70) where
     1.7 -  [code del]: "p1 divides p2 = (\<exists>q. poly p2 = poly(p1 *** q))"
     1.8 +  "p1 divides p2 = (\<exists>q. poly p2 = poly(p1 *** q))"
     1.9  
    1.10      --{*order of a polynomial*}
    1.11  definition (in ring_1) order :: "'a => 'a list => nat" where