diff -r 5b466efedd2c -r 63beb38e9258 src/HOL/Library/Polynomial.thy --- a/src/HOL/Library/Polynomial.thy Fri Feb 21 00:09:55 2014 +0100 +++ b/src/HOL/Library/Polynomial.thy Fri Feb 21 00:09:56 2014 +0100 @@ -406,7 +406,7 @@ { fix ms :: "nat list" and f :: "nat \ 'a" and x :: "'a" assume "\m\set ms. m > 0" then have "map (case_nat x f) ms = map f (map (\n. n - 1) ms)" - by (induct ms) (auto, metis Suc_pred' nat.cases(2)) } + by (induct ms) (auto, metis Suc_pred' nat.case(2)) } note * = this show ?thesis by (simp add: coeffs_def * upt_conv_Cons coeff_pCons map_decr_upt One_nat_def del: upt_Suc) @@ -452,7 +452,7 @@ lemma coeff_Poly_eq: "coeff (Poly xs) n = nth_default 0 xs n" apply (induct xs arbitrary: n) apply simp_all - by (metis nat.cases not0_implies_Suc nth_default_Cons_0 nth_default_Cons_Suc pCons.rep_eq) + by (metis nat.case not0_implies_Suc nth_default_Cons_0 nth_default_Cons_Suc pCons.rep_eq) lemma nth_default_coeffs_eq: "nth_default 0 (coeffs p) = coeff p"