tuned declaration
authorhaftmann
Thu, 29 Dec 2011 10:47:56 +0100
changeset 46031 ac6bae9fdc2f
parent 46030 51b2f3412a03
child 46032 0da934e135b0
tuned declaration
src/HOL/Library/Polynomial.thy
--- a/src/HOL/Library/Polynomial.thy	Thu Dec 29 10:47:55 2011 +0100
+++ b/src/HOL/Library/Polynomial.thy	Thu Dec 29 10:47:56 2011 +0100
@@ -147,7 +147,7 @@
 apply (rule le_degree, simp)
 done
 
-lemma pCons_0_0 [simp]: "pCons 0 0 = 0"
+lemma pCons_0_0 [simp, code_post]: "pCons 0 0 = 0"
 by (rule poly_ext, simp add: coeff_pCons split: nat.split)
 
 lemma pCons_eq_iff [simp]:
@@ -1505,8 +1505,6 @@
 
 quickcheck_generator poly constructors: "0::'a::zero poly", pCons
 
-declare pCons_0_0 [code_post]
-
 instantiation poly :: ("{zero, equal}") equal
 begin