author | huffman |
Mon, 12 Jan 2009 09:04:25 -0800 | |
changeset 29455 | 0139c9a01ca4 |
parent 29454 | b0f586f38dd7 |
child 29456 | 3f8b85444512 |
--- a/src/HOL/Polynomial.thy Mon Jan 12 08:46:07 2009 -0800 +++ b/src/HOL/Polynomial.thy Mon Jan 12 09:04:25 2009 -0800 @@ -100,6 +100,13 @@ where [code del]: "pCons a p = Abs_poly (nat_case a (coeff p))" +syntax + "_poly" :: "args \<Rightarrow> 'a poly" ("[:(_):]") + +translations + "[:x, xs:]" == "CONST pCons x [:xs:]" + "[:x:]" == "CONST pCons x 0" + lemma Poly_nat_case: "f \<in> Poly \<Longrightarrow> nat_case a f \<in> Poly" unfolding Poly_def by (auto split: nat.split)