author | huffman |
Fri, 27 Feb 2009 15:37:56 -0800 | |
changeset 30155 | f65dc19cd5f0 |
parent 30143 | 98a986b02022 |
child 30156 | c621f8b6f4e6 |
--- a/src/HOL/Library/Polynomial.thy Fri Feb 27 16:05:40 2009 +0100 +++ b/src/HOL/Library/Polynomial.thy Fri Feb 27 15:37:56 2009 -0800 @@ -106,6 +106,7 @@ translations "[:x, xs:]" == "CONST pCons x [:xs:]" "[:x:]" == "CONST pCons x 0" + "[:x:]" <= "CONST pCons x (_constrain 0 t)" lemma Poly_nat_case: "f \<in> Poly \<Longrightarrow> nat_case a f \<in> Poly" unfolding Poly_def by (auto split: nat.split)