| author | blanchet | 
| Sun, 01 May 2011 18:37:24 +0200 | |
| changeset 42535 | 3c1f302b3ee6 | 
| parent 41959 | b460124855b8 | 
| child 44890 | 22f665a2e91c | 
| permissions | -rw-r--r-- | 
| 41959 | 1 | (* Title: HOL/Library/Polynomial.thy | 
| 29451 | 2 | Author: Brian Huffman | 
| 41959 | 3 | Author: Clemens Ballarin | 
| 29451 | 4 | *) | 
| 5 | ||
| 6 | header {* Univariate Polynomials *}
 | |
| 7 | ||
| 8 | theory Polynomial | |
| 30738 | 9 | imports Main | 
| 29451 | 10 | begin | 
| 11 | ||
| 12 | subsection {* Definition of type @{text poly} *}
 | |
| 13 | ||
| 14 | typedef (Poly) 'a poly = "{f::nat \<Rightarrow> 'a::zero. \<exists>n. \<forall>i>n. f i = 0}"
 | |
| 15 | morphisms coeff Abs_poly | |
| 16 | by auto | |
| 17 | ||
| 18 | lemma expand_poly_eq: "p = q \<longleftrightarrow> (\<forall>n. coeff p n = coeff q n)" | |
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 19 | by (simp add: coeff_inject [symmetric] fun_eq_iff) | 
| 29451 | 20 | |
| 21 | lemma poly_ext: "(\<And>n. coeff p n = coeff q n) \<Longrightarrow> p = q" | |
| 22 | by (simp add: expand_poly_eq) | |
| 23 | ||
| 24 | ||
| 25 | subsection {* Degree of a polynomial *}
 | |
| 26 | ||
| 27 | definition | |
| 28 | degree :: "'a::zero poly \<Rightarrow> nat" where | |
| 29 | "degree p = (LEAST n. \<forall>i>n. coeff p i = 0)" | |
| 30 | ||
| 31 | lemma coeff_eq_0: "degree p < n \<Longrightarrow> coeff p n = 0" | |
| 32 | proof - | |
| 33 | have "coeff p \<in> Poly" | |
| 34 | by (rule coeff) | |
| 35 | hence "\<exists>n. \<forall>i>n. coeff p i = 0" | |
| 36 | unfolding Poly_def by simp | |
| 37 | hence "\<forall>i>degree p. coeff p i = 0" | |
| 38 | unfolding degree_def by (rule LeastI_ex) | |
| 39 | moreover assume "degree p < n" | |
| 40 | ultimately show ?thesis by simp | |
| 41 | qed | |
| 42 | ||
| 43 | lemma le_degree: "coeff p n \<noteq> 0 \<Longrightarrow> n \<le> degree p" | |
| 44 | by (erule contrapos_np, rule coeff_eq_0, simp) | |
| 45 | ||
| 46 | lemma degree_le: "\<forall>i>n. coeff p i = 0 \<Longrightarrow> degree p \<le> n" | |
| 47 | unfolding degree_def by (erule Least_le) | |
| 48 | ||
| 49 | lemma less_degree_imp: "n < degree p \<Longrightarrow> \<exists>i>n. coeff p i \<noteq> 0" | |
| 50 | unfolding degree_def by (drule not_less_Least, simp) | |
| 51 | ||
| 52 | ||
| 53 | subsection {* The zero polynomial *}
 | |
| 54 | ||
| 55 | instantiation poly :: (zero) zero | |
| 56 | begin | |
| 57 | ||
| 58 | definition | |
| 59 | zero_poly_def: "0 = Abs_poly (\<lambda>n. 0)" | |
| 60 | ||
| 61 | instance .. | |
| 62 | end | |
| 63 | ||
| 64 | lemma coeff_0 [simp]: "coeff 0 n = 0" | |
| 65 | unfolding zero_poly_def | |
| 66 | by (simp add: Abs_poly_inverse Poly_def) | |
| 67 | ||
| 68 | lemma degree_0 [simp]: "degree 0 = 0" | |
| 69 | by (rule order_antisym [OF degree_le le0]) simp | |
| 70 | ||
| 71 | lemma leading_coeff_neq_0: | |
| 72 | assumes "p \<noteq> 0" shows "coeff p (degree p) \<noteq> 0" | |
| 73 | proof (cases "degree p") | |
| 74 | case 0 | |
| 75 | from `p \<noteq> 0` have "\<exists>n. coeff p n \<noteq> 0" | |
| 76 | by (simp add: expand_poly_eq) | |
| 77 | then obtain n where "coeff p n \<noteq> 0" .. | |
| 78 | hence "n \<le> degree p" by (rule le_degree) | |
| 79 | with `coeff p n \<noteq> 0` and `degree p = 0` | |
| 80 | show "coeff p (degree p) \<noteq> 0" by simp | |
| 81 | next | |
| 82 | case (Suc n) | |
| 83 | from `degree p = Suc n` have "n < degree p" by simp | |
| 84 | hence "\<exists>i>n. coeff p i \<noteq> 0" by (rule less_degree_imp) | |
| 85 | then obtain i where "n < i" and "coeff p i \<noteq> 0" by fast | |
| 86 | from `degree p = Suc n` and `n < i` have "degree p \<le> i" by simp | |
| 87 | also from `coeff p i \<noteq> 0` have "i \<le> degree p" by (rule le_degree) | |
| 88 | finally have "degree p = i" . | |
| 89 | with `coeff p i \<noteq> 0` show "coeff p (degree p) \<noteq> 0" by simp | |
| 90 | qed | |
| 91 | ||
| 92 | lemma leading_coeff_0_iff [simp]: "coeff p (degree p) = 0 \<longleftrightarrow> p = 0" | |
| 93 | by (cases "p = 0", simp, simp add: leading_coeff_neq_0) | |
| 94 | ||
| 95 | ||
| 96 | subsection {* List-style constructor for polynomials *}
 | |
| 97 | ||
| 98 | definition | |
| 99 | pCons :: "'a::zero \<Rightarrow> 'a poly \<Rightarrow> 'a poly" | |
| 100 | where | |
| 37765 | 101 | "pCons a p = Abs_poly (nat_case a (coeff p))" | 
| 29451 | 102 | |
| 29455 | 103 | syntax | 
| 104 |   "_poly" :: "args \<Rightarrow> 'a poly"  ("[:(_):]")
 | |
| 105 | ||
| 106 | translations | |
| 107 | "[:x, xs:]" == "CONST pCons x [:xs:]" | |
| 108 | "[:x:]" == "CONST pCons x 0" | |
| 30155 
f65dc19cd5f0
make list-style polynomial syntax work when show_sorts is on
 huffman parents: 
30072diff
changeset | 109 | "[:x:]" <= "CONST pCons x (_constrain 0 t)" | 
| 29455 | 110 | |
| 29451 | 111 | lemma Poly_nat_case: "f \<in> Poly \<Longrightarrow> nat_case a f \<in> Poly" | 
| 112 | unfolding Poly_def by (auto split: nat.split) | |
| 113 | ||
| 114 | lemma coeff_pCons: | |
| 115 | "coeff (pCons a p) = nat_case a (coeff p)" | |
| 116 | unfolding pCons_def | |
| 117 | by (simp add: Abs_poly_inverse Poly_nat_case coeff) | |
| 118 | ||
| 119 | lemma coeff_pCons_0 [simp]: "coeff (pCons a p) 0 = a" | |
| 120 | by (simp add: coeff_pCons) | |
| 121 | ||
| 122 | lemma coeff_pCons_Suc [simp]: "coeff (pCons a p) (Suc n) = coeff p n" | |
| 123 | by (simp add: coeff_pCons) | |
| 124 | ||
| 125 | lemma degree_pCons_le: "degree (pCons a p) \<le> Suc (degree p)" | |
| 126 | by (rule degree_le, simp add: coeff_eq_0 coeff_pCons split: nat.split) | |
| 127 | ||
| 128 | lemma degree_pCons_eq: | |
| 129 | "p \<noteq> 0 \<Longrightarrow> degree (pCons a p) = Suc (degree p)" | |
| 130 | apply (rule order_antisym [OF degree_pCons_le]) | |
| 131 | apply (rule le_degree, simp) | |
| 132 | done | |
| 133 | ||
| 134 | lemma degree_pCons_0: "degree (pCons a 0) = 0" | |
| 135 | apply (rule order_antisym [OF _ le0]) | |
| 136 | apply (rule degree_le, simp add: coeff_pCons split: nat.split) | |
| 137 | done | |
| 138 | ||
| 29460 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 139 | lemma degree_pCons_eq_if [simp]: | 
| 29451 | 140 | "degree (pCons a p) = (if p = 0 then 0 else Suc (degree p))" | 
| 141 | apply (cases "p = 0", simp_all) | |
| 142 | apply (rule order_antisym [OF _ le0]) | |
| 143 | apply (rule degree_le, simp add: coeff_pCons split: nat.split) | |
| 144 | apply (rule order_antisym [OF degree_pCons_le]) | |
| 145 | apply (rule le_degree, simp) | |
| 146 | done | |
| 147 | ||
| 148 | lemma pCons_0_0 [simp]: "pCons 0 0 = 0" | |
| 149 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 150 | ||
| 151 | lemma pCons_eq_iff [simp]: | |
| 152 | "pCons a p = pCons b q \<longleftrightarrow> a = b \<and> p = q" | |
| 153 | proof (safe) | |
| 154 | assume "pCons a p = pCons b q" | |
| 155 | then have "coeff (pCons a p) 0 = coeff (pCons b q) 0" by simp | |
| 156 | then show "a = b" by simp | |
| 157 | next | |
| 158 | assume "pCons a p = pCons b q" | |
| 159 | then have "\<forall>n. coeff (pCons a p) (Suc n) = | |
| 160 | coeff (pCons b q) (Suc n)" by simp | |
| 161 | then show "p = q" by (simp add: expand_poly_eq) | |
| 162 | qed | |
| 163 | ||
| 164 | lemma pCons_eq_0_iff [simp]: "pCons a p = 0 \<longleftrightarrow> a = 0 \<and> p = 0" | |
| 165 | using pCons_eq_iff [of a p 0 0] by simp | |
| 166 | ||
| 167 | lemma Poly_Suc: "f \<in> Poly \<Longrightarrow> (\<lambda>n. f (Suc n)) \<in> Poly" | |
| 168 | unfolding Poly_def | |
| 169 | by (clarify, rule_tac x=n in exI, simp) | |
| 170 | ||
| 171 | lemma pCons_cases [cases type: poly]: | |
| 172 | obtains (pCons) a q where "p = pCons a q" | |
| 173 | proof | |
| 174 | show "p = pCons (coeff p 0) (Abs_poly (\<lambda>n. coeff p (Suc n)))" | |
| 175 | by (rule poly_ext) | |
| 176 | (simp add: Abs_poly_inverse Poly_Suc coeff coeff_pCons | |
| 177 | split: nat.split) | |
| 178 | qed | |
| 179 | ||
| 180 | lemma pCons_induct [case_names 0 pCons, induct type: poly]: | |
| 181 | assumes zero: "P 0" | |
| 182 | assumes pCons: "\<And>a p. P p \<Longrightarrow> P (pCons a p)" | |
| 183 | shows "P p" | |
| 184 | proof (induct p rule: measure_induct_rule [where f=degree]) | |
| 185 | case (less p) | |
| 186 | obtain a q where "p = pCons a q" by (rule pCons_cases) | |
| 187 | have "P q" | |
| 188 | proof (cases "q = 0") | |
| 189 | case True | |
| 190 | then show "P q" by (simp add: zero) | |
| 191 | next | |
| 192 | case False | |
| 193 | then have "degree (pCons a q) = Suc (degree q)" | |
| 194 | by (rule degree_pCons_eq) | |
| 195 | then have "degree q < degree p" | |
| 196 | using `p = pCons a q` by simp | |
| 197 | then show "P q" | |
| 198 | by (rule less.hyps) | |
| 199 | qed | |
| 200 | then have "P (pCons a q)" | |
| 201 | by (rule pCons) | |
| 202 | then show ?case | |
| 203 | using `p = pCons a q` by simp | |
| 204 | qed | |
| 205 | ||
| 206 | ||
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 207 | subsection {* Recursion combinator for polynomials *}
 | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 208 | |
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 209 | function | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 210 |   poly_rec :: "'b \<Rightarrow> ('a::zero \<Rightarrow> 'a poly \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'a poly \<Rightarrow> 'b"
 | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 211 | where | 
| 37765 | 212 | poly_rec_pCons_eq_if [simp del]: | 
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 213 | "poly_rec z f (pCons a p) = f a p (if p = 0 then z else poly_rec z f p)" | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 214 | by (case_tac x, rename_tac q, case_tac q, auto) | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 215 | |
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 216 | termination poly_rec | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 217 | by (relation "measure (degree \<circ> snd \<circ> snd)", simp) | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 218 | (simp add: degree_pCons_eq) | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 219 | |
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 220 | lemma poly_rec_0: | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 221 | "f 0 0 z = z \<Longrightarrow> poly_rec z f 0 = z" | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 222 | using poly_rec_pCons_eq_if [of z f 0 0] by simp | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 223 | |
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 224 | lemma poly_rec_pCons: | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 225 | "f 0 0 z = z \<Longrightarrow> poly_rec z f (pCons a p) = f a p (poly_rec z f p)" | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 226 | by (simp add: poly_rec_pCons_eq_if poly_rec_0) | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 227 | |
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 228 | |
| 29451 | 229 | subsection {* Monomials *}
 | 
| 230 | ||
| 231 | definition | |
| 232 | monom :: "'a \<Rightarrow> nat \<Rightarrow> 'a::zero poly" where | |
| 233 | "monom a m = Abs_poly (\<lambda>n. if m = n then a else 0)" | |
| 234 | ||
| 235 | lemma coeff_monom [simp]: "coeff (monom a m) n = (if m=n then a else 0)" | |
| 236 | unfolding monom_def | |
| 237 | by (subst Abs_poly_inverse, auto simp add: Poly_def) | |
| 238 | ||
| 239 | lemma monom_0: "monom a 0 = pCons a 0" | |
| 240 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 241 | ||
| 242 | lemma monom_Suc: "monom a (Suc n) = pCons 0 (monom a n)" | |
| 243 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 244 | ||
| 245 | lemma monom_eq_0 [simp]: "monom 0 n = 0" | |
| 246 | by (rule poly_ext) simp | |
| 247 | ||
| 248 | lemma monom_eq_0_iff [simp]: "monom a n = 0 \<longleftrightarrow> a = 0" | |
| 249 | by (simp add: expand_poly_eq) | |
| 250 | ||
| 251 | lemma monom_eq_iff [simp]: "monom a n = monom b n \<longleftrightarrow> a = b" | |
| 252 | by (simp add: expand_poly_eq) | |
| 253 | ||
| 254 | lemma degree_monom_le: "degree (monom a n) \<le> n" | |
| 255 | by (rule degree_le, simp) | |
| 256 | ||
| 257 | lemma degree_monom_eq: "a \<noteq> 0 \<Longrightarrow> degree (monom a n) = n" | |
| 258 | apply (rule order_antisym [OF degree_monom_le]) | |
| 259 | apply (rule le_degree, simp) | |
| 260 | done | |
| 261 | ||
| 262 | ||
| 263 | subsection {* Addition and subtraction *}
 | |
| 264 | ||
| 265 | instantiation poly :: (comm_monoid_add) comm_monoid_add | |
| 266 | begin | |
| 267 | ||
| 268 | definition | |
| 37765 | 269 | plus_poly_def: | 
| 29451 | 270 | "p + q = Abs_poly (\<lambda>n. coeff p n + coeff q n)" | 
| 271 | ||
| 272 | lemma Poly_add: | |
| 273 | fixes f g :: "nat \<Rightarrow> 'a" | |
| 274 | shows "\<lbrakk>f \<in> Poly; g \<in> Poly\<rbrakk> \<Longrightarrow> (\<lambda>n. f n + g n) \<in> Poly" | |
| 275 | unfolding Poly_def | |
| 276 | apply (clarify, rename_tac m n) | |
| 277 | apply (rule_tac x="max m n" in exI, simp) | |
| 278 | done | |
| 279 | ||
| 280 | lemma coeff_add [simp]: | |
| 281 | "coeff (p + q) n = coeff p n + coeff q n" | |
| 282 | unfolding plus_poly_def | |
| 283 | by (simp add: Abs_poly_inverse coeff Poly_add) | |
| 284 | ||
| 285 | instance proof | |
| 286 | fix p q r :: "'a poly" | |
| 287 | show "(p + q) + r = p + (q + r)" | |
| 288 | by (simp add: expand_poly_eq add_assoc) | |
| 289 | show "p + q = q + p" | |
| 290 | by (simp add: expand_poly_eq add_commute) | |
| 291 | show "0 + p = p" | |
| 292 | by (simp add: expand_poly_eq) | |
| 293 | qed | |
| 294 | ||
| 295 | end | |
| 296 | ||
| 29904 | 297 | instance poly :: (cancel_comm_monoid_add) cancel_comm_monoid_add | 
| 29540 | 298 | proof | 
| 299 | fix p q r :: "'a poly" | |
| 300 | assume "p + q = p + r" thus "q = r" | |
| 301 | by (simp add: expand_poly_eq) | |
| 302 | qed | |
| 303 | ||
| 29451 | 304 | instantiation poly :: (ab_group_add) ab_group_add | 
| 305 | begin | |
| 306 | ||
| 307 | definition | |
| 37765 | 308 | uminus_poly_def: | 
| 29451 | 309 | "- p = Abs_poly (\<lambda>n. - coeff p n)" | 
| 310 | ||
| 311 | definition | |
| 37765 | 312 | minus_poly_def: | 
| 29451 | 313 | "p - q = Abs_poly (\<lambda>n. coeff p n - coeff q n)" | 
| 314 | ||
| 315 | lemma Poly_minus: | |
| 316 | fixes f :: "nat \<Rightarrow> 'a" | |
| 317 | shows "f \<in> Poly \<Longrightarrow> (\<lambda>n. - f n) \<in> Poly" | |
| 318 | unfolding Poly_def by simp | |
| 319 | ||
| 320 | lemma Poly_diff: | |
| 321 | fixes f g :: "nat \<Rightarrow> 'a" | |
| 322 | shows "\<lbrakk>f \<in> Poly; g \<in> Poly\<rbrakk> \<Longrightarrow> (\<lambda>n. f n - g n) \<in> Poly" | |
| 323 | unfolding diff_minus by (simp add: Poly_add Poly_minus) | |
| 324 | ||
| 325 | lemma coeff_minus [simp]: "coeff (- p) n = - coeff p n" | |
| 326 | unfolding uminus_poly_def | |
| 327 | by (simp add: Abs_poly_inverse coeff Poly_minus) | |
| 328 | ||
| 329 | lemma coeff_diff [simp]: | |
| 330 | "coeff (p - q) n = coeff p n - coeff q n" | |
| 331 | unfolding minus_poly_def | |
| 332 | by (simp add: Abs_poly_inverse coeff Poly_diff) | |
| 333 | ||
| 334 | instance proof | |
| 335 | fix p q :: "'a poly" | |
| 336 | show "- p + p = 0" | |
| 337 | by (simp add: expand_poly_eq) | |
| 338 | show "p - q = p + - q" | |
| 339 | by (simp add: expand_poly_eq diff_minus) | |
| 340 | qed | |
| 341 | ||
| 342 | end | |
| 343 | ||
| 344 | lemma add_pCons [simp]: | |
| 345 | "pCons a p + pCons b q = pCons (a + b) (p + q)" | |
| 346 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 347 | ||
| 348 | lemma minus_pCons [simp]: | |
| 349 | "- pCons a p = pCons (- a) (- p)" | |
| 350 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 351 | ||
| 352 | lemma diff_pCons [simp]: | |
| 353 | "pCons a p - pCons b q = pCons (a - b) (p - q)" | |
| 354 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 355 | ||
| 29539 | 356 | lemma degree_add_le_max: "degree (p + q) \<le> max (degree p) (degree q)" | 
| 29451 | 357 | by (rule degree_le, auto simp add: coeff_eq_0) | 
| 358 | ||
| 29539 | 359 | lemma degree_add_le: | 
| 360 | "\<lbrakk>degree p \<le> n; degree q \<le> n\<rbrakk> \<Longrightarrow> degree (p + q) \<le> n" | |
| 361 | by (auto intro: order_trans degree_add_le_max) | |
| 362 | ||
| 29453 | 363 | lemma degree_add_less: | 
| 364 | "\<lbrakk>degree p < n; degree q < n\<rbrakk> \<Longrightarrow> degree (p + q) < n" | |
| 29539 | 365 | by (auto intro: le_less_trans degree_add_le_max) | 
| 29453 | 366 | |
| 29451 | 367 | lemma degree_add_eq_right: | 
| 368 | "degree p < degree q \<Longrightarrow> degree (p + q) = degree q" | |
| 369 | apply (cases "q = 0", simp) | |
| 370 | apply (rule order_antisym) | |
| 29539 | 371 | apply (simp add: degree_add_le) | 
| 29451 | 372 | apply (rule le_degree) | 
| 373 | apply (simp add: coeff_eq_0) | |
| 374 | done | |
| 375 | ||
| 376 | lemma degree_add_eq_left: | |
| 377 | "degree q < degree p \<Longrightarrow> degree (p + q) = degree p" | |
| 378 | using degree_add_eq_right [of q p] | |
| 379 | by (simp add: add_commute) | |
| 380 | ||
| 381 | lemma degree_minus [simp]: "degree (- p) = degree p" | |
| 382 | unfolding degree_def by simp | |
| 383 | ||
| 29539 | 384 | lemma degree_diff_le_max: "degree (p - q) \<le> max (degree p) (degree q)" | 
| 29451 | 385 | using degree_add_le [where p=p and q="-q"] | 
| 386 | by (simp add: diff_minus) | |
| 387 | ||
| 29539 | 388 | lemma degree_diff_le: | 
| 389 | "\<lbrakk>degree p \<le> n; degree q \<le> n\<rbrakk> \<Longrightarrow> degree (p - q) \<le> n" | |
| 390 | by (simp add: diff_minus degree_add_le) | |
| 391 | ||
| 29453 | 392 | lemma degree_diff_less: | 
| 393 | "\<lbrakk>degree p < n; degree q < n\<rbrakk> \<Longrightarrow> degree (p - q) < n" | |
| 29539 | 394 | by (simp add: diff_minus degree_add_less) | 
| 29453 | 395 | |
| 29451 | 396 | lemma add_monom: "monom a n + monom b n = monom (a + b) n" | 
| 397 | by (rule poly_ext) simp | |
| 398 | ||
| 399 | lemma diff_monom: "monom a n - monom b n = monom (a - b) n" | |
| 400 | by (rule poly_ext) simp | |
| 401 | ||
| 402 | lemma minus_monom: "- monom a n = monom (-a) n" | |
| 403 | by (rule poly_ext) simp | |
| 404 | ||
| 405 | lemma coeff_setsum: "coeff (\<Sum>x\<in>A. p x) i = (\<Sum>x\<in>A. coeff (p x) i)" | |
| 406 | by (cases "finite A", induct set: finite, simp_all) | |
| 407 | ||
| 408 | lemma monom_setsum: "monom (\<Sum>x\<in>A. a x) n = (\<Sum>x\<in>A. monom (a x) n)" | |
| 409 | by (rule poly_ext) (simp add: coeff_setsum) | |
| 410 | ||
| 411 | ||
| 412 | subsection {* Multiplication by a constant *}
 | |
| 413 | ||
| 414 | definition | |
| 415 | smult :: "'a::comm_semiring_0 \<Rightarrow> 'a poly \<Rightarrow> 'a poly" where | |
| 416 | "smult a p = Abs_poly (\<lambda>n. a * coeff p n)" | |
| 417 | ||
| 418 | lemma Poly_smult: | |
| 419 | fixes f :: "nat \<Rightarrow> 'a::comm_semiring_0" | |
| 420 | shows "f \<in> Poly \<Longrightarrow> (\<lambda>n. a * f n) \<in> Poly" | |
| 421 | unfolding Poly_def | |
| 422 | by (clarify, rule_tac x=n in exI, simp) | |
| 423 | ||
| 424 | lemma coeff_smult [simp]: "coeff (smult a p) n = a * coeff p n" | |
| 425 | unfolding smult_def | |
| 426 | by (simp add: Abs_poly_inverse Poly_smult coeff) | |
| 427 | ||
| 428 | lemma degree_smult_le: "degree (smult a p) \<le> degree p" | |
| 429 | by (rule degree_le, simp add: coeff_eq_0) | |
| 430 | ||
| 29472 | 431 | lemma smult_smult [simp]: "smult a (smult b p) = smult (a * b) p" | 
| 29451 | 432 | by (rule poly_ext, simp add: mult_assoc) | 
| 433 | ||
| 434 | lemma smult_0_right [simp]: "smult a 0 = 0" | |
| 435 | by (rule poly_ext, simp) | |
| 436 | ||
| 437 | lemma smult_0_left [simp]: "smult 0 p = 0" | |
| 438 | by (rule poly_ext, simp) | |
| 439 | ||
| 440 | lemma smult_1_left [simp]: "smult (1::'a::comm_semiring_1) p = p" | |
| 441 | by (rule poly_ext, simp) | |
| 442 | ||
| 443 | lemma smult_add_right: | |
| 444 | "smult a (p + q) = smult a p + smult a q" | |
| 29667 | 445 | by (rule poly_ext, simp add: algebra_simps) | 
| 29451 | 446 | |
| 447 | lemma smult_add_left: | |
| 448 | "smult (a + b) p = smult a p + smult b p" | |
| 29667 | 449 | by (rule poly_ext, simp add: algebra_simps) | 
| 29451 | 450 | |
| 29457 | 451 | lemma smult_minus_right [simp]: | 
| 29451 | 452 | "smult (a::'a::comm_ring) (- p) = - smult a p" | 
| 453 | by (rule poly_ext, simp) | |
| 454 | ||
| 29457 | 455 | lemma smult_minus_left [simp]: | 
| 29451 | 456 | "smult (- a::'a::comm_ring) p = - smult a p" | 
| 457 | by (rule poly_ext, simp) | |
| 458 | ||
| 459 | lemma smult_diff_right: | |
| 460 | "smult (a::'a::comm_ring) (p - q) = smult a p - smult a q" | |
| 29667 | 461 | by (rule poly_ext, simp add: algebra_simps) | 
| 29451 | 462 | |
| 463 | lemma smult_diff_left: | |
| 464 | "smult (a - b::'a::comm_ring) p = smult a p - smult b p" | |
| 29667 | 465 | by (rule poly_ext, simp add: algebra_simps) | 
| 29451 | 466 | |
| 29472 | 467 | lemmas smult_distribs = | 
| 468 | smult_add_left smult_add_right | |
| 469 | smult_diff_left smult_diff_right | |
| 470 | ||
| 29451 | 471 | lemma smult_pCons [simp]: | 
| 472 | "smult a (pCons b p) = pCons (a * b) (smult a p)" | |
| 473 | by (rule poly_ext, simp add: coeff_pCons split: nat.split) | |
| 474 | ||
| 475 | lemma smult_monom: "smult a (monom b n) = monom (a * b) n" | |
| 476 | by (induct n, simp add: monom_0, simp add: monom_Suc) | |
| 477 | ||
| 29659 | 478 | lemma degree_smult_eq [simp]: | 
| 479 | fixes a :: "'a::idom" | |
| 480 | shows "degree (smult a p) = (if a = 0 then 0 else degree p)" | |
| 481 | by (cases "a = 0", simp, simp add: degree_def) | |
| 482 | ||
| 483 | lemma smult_eq_0_iff [simp]: | |
| 484 | fixes a :: "'a::idom" | |
| 485 | shows "smult a p = 0 \<longleftrightarrow> a = 0 \<or> p = 0" | |
| 486 | by (simp add: expand_poly_eq) | |
| 487 | ||
| 29451 | 488 | |
| 489 | subsection {* Multiplication of polynomials *}
 | |
| 490 | ||
| 29474 | 491 | text {* TODO: move to SetInterval.thy *}
 | 
| 29451 | 492 | lemma setsum_atMost_Suc_shift: | 
| 493 | fixes f :: "nat \<Rightarrow> 'a::comm_monoid_add" | |
| 494 | shows "(\<Sum>i\<le>Suc n. f i) = f 0 + (\<Sum>i\<le>n. f (Suc i))" | |
| 495 | proof (induct n) | |
| 496 | case 0 show ?case by simp | |
| 497 | next | |
| 498 | case (Suc n) note IH = this | |
| 499 | have "(\<Sum>i\<le>Suc (Suc n). f i) = (\<Sum>i\<le>Suc n. f i) + f (Suc (Suc n))" | |
| 500 | by (rule setsum_atMost_Suc) | |
| 501 | also have "(\<Sum>i\<le>Suc n. f i) = f 0 + (\<Sum>i\<le>n. f (Suc i))" | |
| 502 | by (rule IH) | |
| 503 | also have "f 0 + (\<Sum>i\<le>n. f (Suc i)) + f (Suc (Suc n)) = | |
| 504 | f 0 + ((\<Sum>i\<le>n. f (Suc i)) + f (Suc (Suc n)))" | |
| 505 | by (rule add_assoc) | |
| 506 | also have "(\<Sum>i\<le>n. f (Suc i)) + f (Suc (Suc n)) = (\<Sum>i\<le>Suc n. f (Suc i))" | |
| 507 | by (rule setsum_atMost_Suc [symmetric]) | |
| 508 | finally show ?case . | |
| 509 | qed | |
| 510 | ||
| 511 | instantiation poly :: (comm_semiring_0) comm_semiring_0 | |
| 512 | begin | |
| 513 | ||
| 514 | definition | |
| 37765 | 515 | times_poly_def: | 
| 29474 | 516 | "p * q = poly_rec 0 (\<lambda>a p pq. smult a q + pCons 0 pq) p" | 
| 517 | ||
| 518 | lemma mult_poly_0_left: "(0::'a poly) * q = 0" | |
| 519 | unfolding times_poly_def by (simp add: poly_rec_0) | |
| 520 | ||
| 521 | lemma mult_pCons_left [simp]: | |
| 522 | "pCons a p * q = smult a q + pCons 0 (p * q)" | |
| 523 | unfolding times_poly_def by (simp add: poly_rec_pCons) | |
| 524 | ||
| 525 | lemma mult_poly_0_right: "p * (0::'a poly) = 0" | |
| 526 | by (induct p, simp add: mult_poly_0_left, simp) | |
| 29451 | 527 | |
| 29474 | 528 | lemma mult_pCons_right [simp]: | 
| 529 | "p * pCons a q = smult a p + pCons 0 (p * q)" | |
| 29667 | 530 | by (induct p, simp add: mult_poly_0_left, simp add: algebra_simps) | 
| 29474 | 531 | |
| 532 | lemmas mult_poly_0 = mult_poly_0_left mult_poly_0_right | |
| 533 | ||
| 534 | lemma mult_smult_left [simp]: "smult a p * q = smult a (p * q)" | |
| 535 | by (induct p, simp add: mult_poly_0, simp add: smult_add_right) | |
| 536 | ||
| 537 | lemma mult_smult_right [simp]: "p * smult a q = smult a (p * q)" | |
| 538 | by (induct q, simp add: mult_poly_0, simp add: smult_add_right) | |
| 539 | ||
| 540 | lemma mult_poly_add_left: | |
| 541 | fixes p q r :: "'a poly" | |
| 542 | shows "(p + q) * r = p * r + q * r" | |
| 543 | by (induct r, simp add: mult_poly_0, | |
| 29667 | 544 | simp add: smult_distribs algebra_simps) | 
| 29451 | 545 | |
| 546 | instance proof | |
| 547 | fix p q r :: "'a poly" | |
| 548 | show 0: "0 * p = 0" | |
| 29474 | 549 | by (rule mult_poly_0_left) | 
| 29451 | 550 | show "p * 0 = 0" | 
| 29474 | 551 | by (rule mult_poly_0_right) | 
| 29451 | 552 | show "(p + q) * r = p * r + q * r" | 
| 29474 | 553 | by (rule mult_poly_add_left) | 
| 29451 | 554 | show "(p * q) * r = p * (q * r)" | 
| 29474 | 555 | by (induct p, simp add: mult_poly_0, simp add: mult_poly_add_left) | 
| 29451 | 556 | show "p * q = q * p" | 
| 29474 | 557 | by (induct p, simp add: mult_poly_0, simp) | 
| 29451 | 558 | qed | 
| 559 | ||
| 560 | end | |
| 561 | ||
| 29540 | 562 | instance poly :: (comm_semiring_0_cancel) comm_semiring_0_cancel .. | 
| 563 | ||
| 29474 | 564 | lemma coeff_mult: | 
| 565 | "coeff (p * q) n = (\<Sum>i\<le>n. coeff p i * coeff q (n-i))" | |
| 566 | proof (induct p arbitrary: n) | |
| 567 | case 0 show ?case by simp | |
| 568 | next | |
| 569 | case (pCons a p n) thus ?case | |
| 570 | by (cases n, simp, simp add: setsum_atMost_Suc_shift | |
| 571 | del: setsum_atMost_Suc) | |
| 572 | qed | |
| 29451 | 573 | |
| 29474 | 574 | lemma degree_mult_le: "degree (p * q) \<le> degree p + degree q" | 
| 575 | apply (rule degree_le) | |
| 576 | apply (induct p) | |
| 577 | apply simp | |
| 578 | apply (simp add: coeff_eq_0 coeff_pCons split: nat.split) | |
| 29451 | 579 | done | 
| 580 | ||
| 581 | lemma mult_monom: "monom a m * monom b n = monom (a * b) (m + n)" | |
| 582 | by (induct m, simp add: monom_0 smult_monom, simp add: monom_Suc) | |
| 583 | ||
| 584 | ||
| 585 | subsection {* The unit polynomial and exponentiation *}
 | |
| 586 | ||
| 587 | instantiation poly :: (comm_semiring_1) comm_semiring_1 | |
| 588 | begin | |
| 589 | ||
| 590 | definition | |
| 591 | one_poly_def: | |
| 592 | "1 = pCons 1 0" | |
| 593 | ||
| 594 | instance proof | |
| 595 | fix p :: "'a poly" show "1 * p = p" | |
| 596 | unfolding one_poly_def | |
| 597 | by simp | |
| 598 | next | |
| 599 | show "0 \<noteq> (1::'a poly)" | |
| 600 | unfolding one_poly_def by simp | |
| 601 | qed | |
| 602 | ||
| 603 | end | |
| 604 | ||
| 29540 | 605 | instance poly :: (comm_semiring_1_cancel) comm_semiring_1_cancel .. | 
| 606 | ||
| 29451 | 607 | lemma coeff_1 [simp]: "coeff 1 n = (if n = 0 then 1 else 0)" | 
| 608 | unfolding one_poly_def | |
| 609 | by (simp add: coeff_pCons split: nat.split) | |
| 610 | ||
| 611 | lemma degree_1 [simp]: "degree 1 = 0" | |
| 612 | unfolding one_poly_def | |
| 613 | by (rule degree_pCons_0) | |
| 614 | ||
| 29979 | 615 | text {* Lemmas about divisibility *}
 | 
| 616 | ||
| 617 | lemma dvd_smult: "p dvd q \<Longrightarrow> p dvd smult a q" | |
| 618 | proof - | |
| 619 | assume "p dvd q" | |
| 620 | then obtain k where "q = p * k" .. | |
| 621 | then have "smult a q = p * smult a k" by simp | |
| 622 | then show "p dvd smult a q" .. | |
| 623 | qed | |
| 624 | ||
| 625 | lemma dvd_smult_cancel: | |
| 626 | fixes a :: "'a::field" | |
| 627 | shows "p dvd smult a q \<Longrightarrow> a \<noteq> 0 \<Longrightarrow> p dvd q" | |
| 628 | by (drule dvd_smult [where a="inverse a"]) simp | |
| 629 | ||
| 630 | lemma dvd_smult_iff: | |
| 631 | fixes a :: "'a::field" | |
| 632 | shows "a \<noteq> 0 \<Longrightarrow> p dvd smult a q \<longleftrightarrow> p dvd q" | |
| 633 | by (safe elim!: dvd_smult dvd_smult_cancel) | |
| 634 | ||
| 31663 | 635 | lemma smult_dvd_cancel: | 
| 636 | "smult a p dvd q \<Longrightarrow> p dvd q" | |
| 637 | proof - | |
| 638 | assume "smult a p dvd q" | |
| 639 | then obtain k where "q = smult a p * k" .. | |
| 640 | then have "q = p * smult a k" by simp | |
| 641 | then show "p dvd q" .. | |
| 642 | qed | |
| 643 | ||
| 644 | lemma smult_dvd: | |
| 645 | fixes a :: "'a::field" | |
| 646 | shows "p dvd q \<Longrightarrow> a \<noteq> 0 \<Longrightarrow> smult a p dvd q" | |
| 647 | by (rule smult_dvd_cancel [where a="inverse a"]) simp | |
| 648 | ||
| 649 | lemma smult_dvd_iff: | |
| 650 | fixes a :: "'a::field" | |
| 651 | shows "smult a p dvd q \<longleftrightarrow> (if a = 0 then q = 0 else p dvd q)" | |
| 652 | by (auto elim: smult_dvd smult_dvd_cancel) | |
| 653 | ||
| 29979 | 654 | lemma degree_power_le: "degree (p ^ n) \<le> degree p * n" | 
| 655 | by (induct n, simp, auto intro: order_trans degree_mult_le) | |
| 656 | ||
| 29451 | 657 | instance poly :: (comm_ring) comm_ring .. | 
| 658 | ||
| 659 | instance poly :: (comm_ring_1) comm_ring_1 .. | |
| 660 | ||
| 661 | instantiation poly :: (comm_ring_1) number_ring | |
| 662 | begin | |
| 663 | ||
| 664 | definition | |
| 665 | "number_of k = (of_int k :: 'a poly)" | |
| 666 | ||
| 667 | instance | |
| 668 | by default (rule number_of_poly_def) | |
| 669 | ||
| 670 | end | |
| 671 | ||
| 672 | ||
| 673 | subsection {* Polynomials form an integral domain *}
 | |
| 674 | ||
| 675 | lemma coeff_mult_degree_sum: | |
| 676 | "coeff (p * q) (degree p + degree q) = | |
| 677 | coeff p (degree p) * coeff q (degree q)" | |
| 29471 | 678 | by (induct p, simp, simp add: coeff_eq_0) | 
| 29451 | 679 | |
| 680 | instance poly :: (idom) idom | |
| 681 | proof | |
| 682 | fix p q :: "'a poly" | |
| 683 | assume "p \<noteq> 0" and "q \<noteq> 0" | |
| 684 | have "coeff (p * q) (degree p + degree q) = | |
| 685 | coeff p (degree p) * coeff q (degree q)" | |
| 686 | by (rule coeff_mult_degree_sum) | |
| 687 | also have "coeff p (degree p) * coeff q (degree q) \<noteq> 0" | |
| 688 | using `p \<noteq> 0` and `q \<noteq> 0` by simp | |
| 689 | finally have "\<exists>n. coeff (p * q) n \<noteq> 0" .. | |
| 690 | thus "p * q \<noteq> 0" by (simp add: expand_poly_eq) | |
| 691 | qed | |
| 692 | ||
| 693 | lemma degree_mult_eq: | |
| 694 | fixes p q :: "'a::idom poly" | |
| 695 | shows "\<lbrakk>p \<noteq> 0; q \<noteq> 0\<rbrakk> \<Longrightarrow> degree (p * q) = degree p + degree q" | |
| 696 | apply (rule order_antisym [OF degree_mult_le le_degree]) | |
| 697 | apply (simp add: coeff_mult_degree_sum) | |
| 698 | done | |
| 699 | ||
| 700 | lemma dvd_imp_degree_le: | |
| 701 | fixes p q :: "'a::idom poly" | |
| 702 | shows "\<lbrakk>p dvd q; q \<noteq> 0\<rbrakk> \<Longrightarrow> degree p \<le> degree q" | |
| 703 | by (erule dvdE, simp add: degree_mult_eq) | |
| 704 | ||
| 705 | ||
| 29878 | 706 | subsection {* Polynomials form an ordered integral domain *}
 | 
| 707 | ||
| 708 | definition | |
| 35028 
108662d50512
more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
 haftmann parents: 
34973diff
changeset | 709 | pos_poly :: "'a::linordered_idom poly \<Rightarrow> bool" | 
| 29878 | 710 | where | 
| 711 | "pos_poly p \<longleftrightarrow> 0 < coeff p (degree p)" | |
| 712 | ||
| 713 | lemma pos_poly_pCons: | |
| 714 | "pos_poly (pCons a p) \<longleftrightarrow> pos_poly p \<or> (p = 0 \<and> 0 < a)" | |
| 715 | unfolding pos_poly_def by simp | |
| 716 | ||
| 717 | lemma not_pos_poly_0 [simp]: "\<not> pos_poly 0" | |
| 718 | unfolding pos_poly_def by simp | |
| 719 | ||
| 720 | lemma pos_poly_add: "\<lbrakk>pos_poly p; pos_poly q\<rbrakk> \<Longrightarrow> pos_poly (p + q)" | |
| 721 | apply (induct p arbitrary: q, simp) | |
| 722 | apply (case_tac q, force simp add: pos_poly_pCons add_pos_pos) | |
| 723 | done | |
| 724 | ||
| 725 | lemma pos_poly_mult: "\<lbrakk>pos_poly p; pos_poly q\<rbrakk> \<Longrightarrow> pos_poly (p * q)" | |
| 726 | unfolding pos_poly_def | |
| 727 | apply (subgoal_tac "p \<noteq> 0 \<and> q \<noteq> 0") | |
| 728 | apply (simp add: degree_mult_eq coeff_mult_degree_sum mult_pos_pos) | |
| 729 | apply auto | |
| 730 | done | |
| 731 | ||
| 732 | lemma pos_poly_total: "p = 0 \<or> pos_poly p \<or> pos_poly (- p)" | |
| 733 | by (induct p) (auto simp add: pos_poly_pCons) | |
| 734 | ||
| 35028 
108662d50512
more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
 haftmann parents: 
34973diff
changeset | 735 | instantiation poly :: (linordered_idom) linordered_idom | 
| 29878 | 736 | begin | 
| 737 | ||
| 738 | definition | |
| 37765 | 739 | "x < y \<longleftrightarrow> pos_poly (y - x)" | 
| 29878 | 740 | |
| 741 | definition | |
| 37765 | 742 | "x \<le> y \<longleftrightarrow> x = y \<or> pos_poly (y - x)" | 
| 29878 | 743 | |
| 744 | definition | |
| 37765 | 745 | "abs (x::'a poly) = (if x < 0 then - x else x)" | 
| 29878 | 746 | |
| 747 | definition | |
| 37765 | 748 | "sgn (x::'a poly) = (if x = 0 then 0 else if 0 < x then 1 else - 1)" | 
| 29878 | 749 | |
| 750 | instance proof | |
| 751 | fix x y :: "'a poly" | |
| 752 | show "x < y \<longleftrightarrow> x \<le> y \<and> \<not> y \<le> x" | |
| 753 | unfolding less_eq_poly_def less_poly_def | |
| 754 | apply safe | |
| 755 | apply simp | |
| 756 | apply (drule (1) pos_poly_add) | |
| 757 | apply simp | |
| 758 | done | |
| 759 | next | |
| 760 | fix x :: "'a poly" show "x \<le> x" | |
| 761 | unfolding less_eq_poly_def by simp | |
| 762 | next | |
| 763 | fix x y z :: "'a poly" | |
| 764 | assume "x \<le> y" and "y \<le> z" thus "x \<le> z" | |
| 765 | unfolding less_eq_poly_def | |
| 766 | apply safe | |
| 767 | apply (drule (1) pos_poly_add) | |
| 768 | apply (simp add: algebra_simps) | |
| 769 | done | |
| 770 | next | |
| 771 | fix x y :: "'a poly" | |
| 772 | assume "x \<le> y" and "y \<le> x" thus "x = y" | |
| 773 | unfolding less_eq_poly_def | |
| 774 | apply safe | |
| 775 | apply (drule (1) pos_poly_add) | |
| 776 | apply simp | |
| 777 | done | |
| 778 | next | |
| 779 | fix x y z :: "'a poly" | |
| 780 | assume "x \<le> y" thus "z + x \<le> z + y" | |
| 781 | unfolding less_eq_poly_def | |
| 782 | apply safe | |
| 783 | apply (simp add: algebra_simps) | |
| 784 | done | |
| 785 | next | |
| 786 | fix x y :: "'a poly" | |
| 787 | show "x \<le> y \<or> y \<le> x" | |
| 788 | unfolding less_eq_poly_def | |
| 789 | using pos_poly_total [of "x - y"] | |
| 790 | by auto | |
| 791 | next | |
| 792 | fix x y z :: "'a poly" | |
| 793 | assume "x < y" and "0 < z" | |
| 794 | thus "z * x < z * y" | |
| 795 | unfolding less_poly_def | |
| 796 | by (simp add: right_diff_distrib [symmetric] pos_poly_mult) | |
| 797 | next | |
| 798 | fix x :: "'a poly" | |
| 799 | show "\<bar>x\<bar> = (if x < 0 then - x else x)" | |
| 800 | by (rule abs_poly_def) | |
| 801 | next | |
| 802 | fix x :: "'a poly" | |
| 803 | show "sgn x = (if x = 0 then 0 else if 0 < x then 1 else - 1)" | |
| 804 | by (rule sgn_poly_def) | |
| 805 | qed | |
| 806 | ||
| 807 | end | |
| 808 | ||
| 809 | text {* TODO: Simplification rules for comparisons *}
 | |
| 810 | ||
| 811 | ||
| 29451 | 812 | subsection {* Long division of polynomials *}
 | 
| 813 | ||
| 814 | definition | |
| 29537 | 815 | pdivmod_rel :: "'a::field poly \<Rightarrow> 'a poly \<Rightarrow> 'a poly \<Rightarrow> 'a poly \<Rightarrow> bool" | 
| 29451 | 816 | where | 
| 29537 | 817 | "pdivmod_rel x y q r \<longleftrightarrow> | 
| 29451 | 818 | x = q * y + r \<and> (if y = 0 then q = 0 else r = 0 \<or> degree r < degree y)" | 
| 819 | ||
| 29537 | 820 | lemma pdivmod_rel_0: | 
| 821 | "pdivmod_rel 0 y 0 0" | |
| 822 | unfolding pdivmod_rel_def by simp | |
| 29451 | 823 | |
| 29537 | 824 | lemma pdivmod_rel_by_0: | 
| 825 | "pdivmod_rel x 0 0 x" | |
| 826 | unfolding pdivmod_rel_def by simp | |
| 29451 | 827 | |
| 828 | lemma eq_zero_or_degree_less: | |
| 829 | assumes "degree p \<le> n" and "coeff p n = 0" | |
| 830 | shows "p = 0 \<or> degree p < n" | |
| 831 | proof (cases n) | |
| 832 | case 0 | |
| 833 | with `degree p \<le> n` and `coeff p n = 0` | |
| 834 | have "coeff p (degree p) = 0" by simp | |
| 835 | then have "p = 0" by simp | |
| 836 | then show ?thesis .. | |
| 837 | next | |
| 838 | case (Suc m) | |
| 839 | have "\<forall>i>n. coeff p i = 0" | |
| 840 | using `degree p \<le> n` by (simp add: coeff_eq_0) | |
| 841 | then have "\<forall>i\<ge>n. coeff p i = 0" | |
| 842 | using `coeff p n = 0` by (simp add: le_less) | |
| 843 | then have "\<forall>i>m. coeff p i = 0" | |
| 844 | using `n = Suc m` by (simp add: less_eq_Suc_le) | |
| 845 | then have "degree p \<le> m" | |
| 846 | by (rule degree_le) | |
| 847 | then have "degree p < n" | |
| 848 | using `n = Suc m` by (simp add: less_Suc_eq_le) | |
| 849 | then show ?thesis .. | |
| 850 | qed | |
| 851 | ||
| 29537 | 852 | lemma pdivmod_rel_pCons: | 
| 853 | assumes rel: "pdivmod_rel x y q r" | |
| 29451 | 854 | assumes y: "y \<noteq> 0" | 
| 855 | assumes b: "b = coeff (pCons a r) (degree y) / coeff y (degree y)" | |
| 29537 | 856 | shows "pdivmod_rel (pCons a x) y (pCons b q) (pCons a r - smult b y)" | 
| 857 | (is "pdivmod_rel ?x y ?q ?r") | |
| 29451 | 858 | proof - | 
| 859 | have x: "x = q * y + r" and r: "r = 0 \<or> degree r < degree y" | |
| 29537 | 860 | using assms unfolding pdivmod_rel_def by simp_all | 
| 29451 | 861 | |
| 862 | have 1: "?x = ?q * y + ?r" | |
| 863 | using b x by simp | |
| 864 | ||
| 865 | have 2: "?r = 0 \<or> degree ?r < degree y" | |
| 866 | proof (rule eq_zero_or_degree_less) | |
| 29539 | 867 | show "degree ?r \<le> degree y" | 
| 868 | proof (rule degree_diff_le) | |
| 29451 | 869 | show "degree (pCons a r) \<le> degree y" | 
| 29460 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 870 | using r by auto | 
| 29451 | 871 | show "degree (smult b y) \<le> degree y" | 
| 872 | by (rule degree_smult_le) | |
| 873 | qed | |
| 874 | next | |
| 875 | show "coeff ?r (degree y) = 0" | |
| 876 | using `y \<noteq> 0` unfolding b by simp | |
| 877 | qed | |
| 878 | ||
| 879 | from 1 2 show ?thesis | |
| 29537 | 880 | unfolding pdivmod_rel_def | 
| 29451 | 881 | using `y \<noteq> 0` by simp | 
| 882 | qed | |
| 883 | ||
| 29537 | 884 | lemma pdivmod_rel_exists: "\<exists>q r. pdivmod_rel x y q r" | 
| 29451 | 885 | apply (cases "y = 0") | 
| 29537 | 886 | apply (fast intro!: pdivmod_rel_by_0) | 
| 29451 | 887 | apply (induct x) | 
| 29537 | 888 | apply (fast intro!: pdivmod_rel_0) | 
| 889 | apply (fast intro!: pdivmod_rel_pCons) | |
| 29451 | 890 | done | 
| 891 | ||
| 29537 | 892 | lemma pdivmod_rel_unique: | 
| 893 | assumes 1: "pdivmod_rel x y q1 r1" | |
| 894 | assumes 2: "pdivmod_rel x y q2 r2" | |
| 29451 | 895 | shows "q1 = q2 \<and> r1 = r2" | 
| 896 | proof (cases "y = 0") | |
| 897 | assume "y = 0" with assms show ?thesis | |
| 29537 | 898 | by (simp add: pdivmod_rel_def) | 
| 29451 | 899 | next | 
| 900 | assume [simp]: "y \<noteq> 0" | |
| 901 | from 1 have q1: "x = q1 * y + r1" and r1: "r1 = 0 \<or> degree r1 < degree y" | |
| 29537 | 902 | unfolding pdivmod_rel_def by simp_all | 
| 29451 | 903 | from 2 have q2: "x = q2 * y + r2" and r2: "r2 = 0 \<or> degree r2 < degree y" | 
| 29537 | 904 | unfolding pdivmod_rel_def by simp_all | 
| 29451 | 905 | from q1 q2 have q3: "(q1 - q2) * y = r2 - r1" | 
| 29667 | 906 | by (simp add: algebra_simps) | 
| 29451 | 907 | from r1 r2 have r3: "(r2 - r1) = 0 \<or> degree (r2 - r1) < degree y" | 
| 29453 | 908 | by (auto intro: degree_diff_less) | 
| 29451 | 909 | |
| 910 | show "q1 = q2 \<and> r1 = r2" | |
| 911 | proof (rule ccontr) | |
| 912 | assume "\<not> (q1 = q2 \<and> r1 = r2)" | |
| 913 | with q3 have "q1 \<noteq> q2" and "r1 \<noteq> r2" by auto | |
| 914 | with r3 have "degree (r2 - r1) < degree y" by simp | |
| 915 | also have "degree y \<le> degree (q1 - q2) + degree y" by simp | |
| 916 | also have "\<dots> = degree ((q1 - q2) * y)" | |
| 917 | using `q1 \<noteq> q2` by (simp add: degree_mult_eq) | |
| 918 | also have "\<dots> = degree (r2 - r1)" | |
| 919 | using q3 by simp | |
| 920 | finally have "degree (r2 - r1) < degree (r2 - r1)" . | |
| 921 | then show "False" by simp | |
| 922 | qed | |
| 923 | qed | |
| 924 | ||
| 29660 | 925 | lemma pdivmod_rel_0_iff: "pdivmod_rel 0 y q r \<longleftrightarrow> q = 0 \<and> r = 0" | 
| 926 | by (auto dest: pdivmod_rel_unique intro: pdivmod_rel_0) | |
| 927 | ||
| 928 | lemma pdivmod_rel_by_0_iff: "pdivmod_rel x 0 q r \<longleftrightarrow> q = 0 \<and> r = x" | |
| 929 | by (auto dest: pdivmod_rel_unique intro: pdivmod_rel_by_0) | |
| 930 | ||
| 29537 | 931 | lemmas pdivmod_rel_unique_div = | 
| 932 | pdivmod_rel_unique [THEN conjunct1, standard] | |
| 29451 | 933 | |
| 29537 | 934 | lemmas pdivmod_rel_unique_mod = | 
| 935 | pdivmod_rel_unique [THEN conjunct2, standard] | |
| 29451 | 936 | |
| 937 | instantiation poly :: (field) ring_div | |
| 938 | begin | |
| 939 | ||
| 940 | definition div_poly where | |
| 37765 | 941 | "x div y = (THE q. \<exists>r. pdivmod_rel x y q r)" | 
| 29451 | 942 | |
| 943 | definition mod_poly where | |
| 37765 | 944 | "x mod y = (THE r. \<exists>q. pdivmod_rel x y q r)" | 
| 29451 | 945 | |
| 946 | lemma div_poly_eq: | |
| 29537 | 947 | "pdivmod_rel x y q r \<Longrightarrow> x div y = q" | 
| 29451 | 948 | unfolding div_poly_def | 
| 29537 | 949 | by (fast elim: pdivmod_rel_unique_div) | 
| 29451 | 950 | |
| 951 | lemma mod_poly_eq: | |
| 29537 | 952 | "pdivmod_rel x y q r \<Longrightarrow> x mod y = r" | 
| 29451 | 953 | unfolding mod_poly_def | 
| 29537 | 954 | by (fast elim: pdivmod_rel_unique_mod) | 
| 29451 | 955 | |
| 29537 | 956 | lemma pdivmod_rel: | 
| 957 | "pdivmod_rel x y (x div y) (x mod y)" | |
| 29451 | 958 | proof - | 
| 29537 | 959 | from pdivmod_rel_exists | 
| 960 | obtain q r where "pdivmod_rel x y q r" by fast | |
| 29451 | 961 | thus ?thesis | 
| 962 | by (simp add: div_poly_eq mod_poly_eq) | |
| 963 | qed | |
| 964 | ||
| 965 | instance proof | |
| 966 | fix x y :: "'a poly" | |
| 967 | show "x div y * y + x mod y = x" | |
| 29537 | 968 | using pdivmod_rel [of x y] | 
| 969 | by (simp add: pdivmod_rel_def) | |
| 29451 | 970 | next | 
| 971 | fix x :: "'a poly" | |
| 29537 | 972 | have "pdivmod_rel x 0 0 x" | 
| 973 | by (rule pdivmod_rel_by_0) | |
| 29451 | 974 | thus "x div 0 = 0" | 
| 975 | by (rule div_poly_eq) | |
| 976 | next | |
| 977 | fix y :: "'a poly" | |
| 29537 | 978 | have "pdivmod_rel 0 y 0 0" | 
| 979 | by (rule pdivmod_rel_0) | |
| 29451 | 980 | thus "0 div y = 0" | 
| 981 | by (rule div_poly_eq) | |
| 982 | next | |
| 983 | fix x y z :: "'a poly" | |
| 984 | assume "y \<noteq> 0" | |
| 29537 | 985 | hence "pdivmod_rel (x + z * y) y (z + x div y) (x mod y)" | 
| 986 | using pdivmod_rel [of x y] | |
| 987 | by (simp add: pdivmod_rel_def left_distrib) | |
| 29451 | 988 | thus "(x + z * y) div y = z + x div y" | 
| 989 | by (rule div_poly_eq) | |
| 30930 | 990 | next | 
| 991 | fix x y z :: "'a poly" | |
| 992 | assume "x \<noteq> 0" | |
| 993 | show "(x * y) div (x * z) = y div z" | |
| 994 | proof (cases "y \<noteq> 0 \<and> z \<noteq> 0") | |
| 995 | have "\<And>x::'a poly. pdivmod_rel x 0 0 x" | |
| 996 | by (rule pdivmod_rel_by_0) | |
| 997 | then have [simp]: "\<And>x::'a poly. x div 0 = 0" | |
| 998 | by (rule div_poly_eq) | |
| 999 | have "\<And>x::'a poly. pdivmod_rel 0 x 0 0" | |
| 1000 | by (rule pdivmod_rel_0) | |
| 1001 | then have [simp]: "\<And>x::'a poly. 0 div x = 0" | |
| 1002 | by (rule div_poly_eq) | |
| 1003 | case False then show ?thesis by auto | |
| 1004 | next | |
| 1005 | case True then have "y \<noteq> 0" and "z \<noteq> 0" by auto | |
| 1006 | with `x \<noteq> 0` | |
| 1007 | have "\<And>q r. pdivmod_rel y z q r \<Longrightarrow> pdivmod_rel (x * y) (x * z) q (x * r)" | |
| 1008 | by (auto simp add: pdivmod_rel_def algebra_simps) | |
| 1009 | (rule classical, simp add: degree_mult_eq) | |
| 1010 | moreover from pdivmod_rel have "pdivmod_rel y z (y div z) (y mod z)" . | |
| 1011 | ultimately have "pdivmod_rel (x * y) (x * z) (y div z) (x * (y mod z))" . | |
| 1012 | then show ?thesis by (simp add: div_poly_eq) | |
| 1013 | qed | |
| 29451 | 1014 | qed | 
| 1015 | ||
| 1016 | end | |
| 1017 | ||
| 1018 | lemma degree_mod_less: | |
| 1019 | "y \<noteq> 0 \<Longrightarrow> x mod y = 0 \<or> degree (x mod y) < degree y" | |
| 29537 | 1020 | using pdivmod_rel [of x y] | 
| 1021 | unfolding pdivmod_rel_def by simp | |
| 29451 | 1022 | |
| 1023 | lemma div_poly_less: "degree x < degree y \<Longrightarrow> x div y = 0" | |
| 1024 | proof - | |
| 1025 | assume "degree x < degree y" | |
| 29537 | 1026 | hence "pdivmod_rel x y 0 x" | 
| 1027 | by (simp add: pdivmod_rel_def) | |
| 29451 | 1028 | thus "x div y = 0" by (rule div_poly_eq) | 
| 1029 | qed | |
| 1030 | ||
| 1031 | lemma mod_poly_less: "degree x < degree y \<Longrightarrow> x mod y = x" | |
| 1032 | proof - | |
| 1033 | assume "degree x < degree y" | |
| 29537 | 1034 | hence "pdivmod_rel x y 0 x" | 
| 1035 | by (simp add: pdivmod_rel_def) | |
| 29451 | 1036 | thus "x mod y = x" by (rule mod_poly_eq) | 
| 1037 | qed | |
| 1038 | ||
| 29659 | 1039 | lemma pdivmod_rel_smult_left: | 
| 1040 | "pdivmod_rel x y q r | |
| 1041 | \<Longrightarrow> pdivmod_rel (smult a x) y (smult a q) (smult a r)" | |
| 1042 | unfolding pdivmod_rel_def by (simp add: smult_add_right) | |
| 1043 | ||
| 1044 | lemma div_smult_left: "(smult a x) div y = smult a (x div y)" | |
| 1045 | by (rule div_poly_eq, rule pdivmod_rel_smult_left, rule pdivmod_rel) | |
| 1046 | ||
| 1047 | lemma mod_smult_left: "(smult a x) mod y = smult a (x mod y)" | |
| 1048 | by (rule mod_poly_eq, rule pdivmod_rel_smult_left, rule pdivmod_rel) | |
| 1049 | ||
| 30072 | 1050 | lemma poly_div_minus_left [simp]: | 
| 1051 | fixes x y :: "'a::field poly" | |
| 1052 | shows "(- x) div y = - (x div y)" | |
| 1053 | using div_smult_left [of "- 1::'a"] by simp | |
| 1054 | ||
| 1055 | lemma poly_mod_minus_left [simp]: | |
| 1056 | fixes x y :: "'a::field poly" | |
| 1057 | shows "(- x) mod y = - (x mod y)" | |
| 1058 | using mod_smult_left [of "- 1::'a"] by simp | |
| 1059 | ||
| 29659 | 1060 | lemma pdivmod_rel_smult_right: | 
| 1061 | "\<lbrakk>a \<noteq> 0; pdivmod_rel x y q r\<rbrakk> | |
| 1062 | \<Longrightarrow> pdivmod_rel x (smult a y) (smult (inverse a) q) r" | |
| 1063 | unfolding pdivmod_rel_def by simp | |
| 1064 | ||
| 1065 | lemma div_smult_right: | |
| 1066 | "a \<noteq> 0 \<Longrightarrow> x div (smult a y) = smult (inverse a) (x div y)" | |
| 1067 | by (rule div_poly_eq, erule pdivmod_rel_smult_right, rule pdivmod_rel) | |
| 1068 | ||
| 1069 | lemma mod_smult_right: "a \<noteq> 0 \<Longrightarrow> x mod (smult a y) = x mod y" | |
| 1070 | by (rule mod_poly_eq, erule pdivmod_rel_smult_right, rule pdivmod_rel) | |
| 1071 | ||
| 30072 | 1072 | lemma poly_div_minus_right [simp]: | 
| 1073 | fixes x y :: "'a::field poly" | |
| 1074 | shows "x div (- y) = - (x div y)" | |
| 1075 | using div_smult_right [of "- 1::'a"] | |
| 1076 | by (simp add: nonzero_inverse_minus_eq) | |
| 1077 | ||
| 1078 | lemma poly_mod_minus_right [simp]: | |
| 1079 | fixes x y :: "'a::field poly" | |
| 1080 | shows "x mod (- y) = x mod y" | |
| 1081 | using mod_smult_right [of "- 1::'a"] by simp | |
| 1082 | ||
| 29660 | 1083 | lemma pdivmod_rel_mult: | 
| 1084 | "\<lbrakk>pdivmod_rel x y q r; pdivmod_rel q z q' r'\<rbrakk> | |
| 1085 | \<Longrightarrow> pdivmod_rel x (y * z) q' (y * r' + r)" | |
| 1086 | apply (cases "z = 0", simp add: pdivmod_rel_def) | |
| 1087 | apply (cases "y = 0", simp add: pdivmod_rel_by_0_iff pdivmod_rel_0_iff) | |
| 1088 | apply (cases "r = 0") | |
| 1089 | apply (cases "r' = 0") | |
| 1090 | apply (simp add: pdivmod_rel_def) | |
| 36350 | 1091 | apply (simp add: pdivmod_rel_def field_simps degree_mult_eq) | 
| 29660 | 1092 | apply (cases "r' = 0") | 
| 1093 | apply (simp add: pdivmod_rel_def degree_mult_eq) | |
| 36350 | 1094 | apply (simp add: pdivmod_rel_def field_simps) | 
| 29660 | 1095 | apply (simp add: degree_mult_eq degree_add_less) | 
| 1096 | done | |
| 1097 | ||
| 1098 | lemma poly_div_mult_right: | |
| 1099 | fixes x y z :: "'a::field poly" | |
| 1100 | shows "x div (y * z) = (x div y) div z" | |
| 1101 | by (rule div_poly_eq, rule pdivmod_rel_mult, (rule pdivmod_rel)+) | |
| 1102 | ||
| 1103 | lemma poly_mod_mult_right: | |
| 1104 | fixes x y z :: "'a::field poly" | |
| 1105 | shows "x mod (y * z) = y * (x div y mod z) + x mod y" | |
| 1106 | by (rule mod_poly_eq, rule pdivmod_rel_mult, (rule pdivmod_rel)+) | |
| 1107 | ||
| 29451 | 1108 | lemma mod_pCons: | 
| 1109 | fixes a and x | |
| 1110 | assumes y: "y \<noteq> 0" | |
| 1111 | defines b: "b \<equiv> coeff (pCons a (x mod y)) (degree y) / coeff y (degree y)" | |
| 1112 | shows "(pCons a x) mod y = (pCons a (x mod y) - smult b y)" | |
| 1113 | unfolding b | |
| 1114 | apply (rule mod_poly_eq) | |
| 29537 | 1115 | apply (rule pdivmod_rel_pCons [OF pdivmod_rel y refl]) | 
| 29451 | 1116 | done | 
| 1117 | ||
| 1118 | ||
| 31663 | 1119 | subsection {* GCD of polynomials *}
 | 
| 1120 | ||
| 1121 | function | |
| 1122 | poly_gcd :: "'a::field poly \<Rightarrow> 'a poly \<Rightarrow> 'a poly" where | |
| 1123 | "poly_gcd x 0 = smult (inverse (coeff x (degree x))) x" | |
| 1124 | | "y \<noteq> 0 \<Longrightarrow> poly_gcd x y = poly_gcd y (x mod y)" | |
| 1125 | by auto | |
| 1126 | ||
| 1127 | termination poly_gcd | |
| 1128 | by (relation "measure (\<lambda>(x, y). if y = 0 then 0 else Suc (degree y))") | |
| 1129 | (auto dest: degree_mod_less) | |
| 1130 | ||
| 37765 | 1131 | declare poly_gcd.simps [simp del] | 
| 31663 | 1132 | |
| 1133 | lemma poly_gcd_dvd1 [iff]: "poly_gcd x y dvd x" | |
| 1134 | and poly_gcd_dvd2 [iff]: "poly_gcd x y dvd y" | |
| 1135 | apply (induct x y rule: poly_gcd.induct) | |
| 1136 | apply (simp_all add: poly_gcd.simps) | |
| 1137 | apply (fastsimp simp add: smult_dvd_iff dest: inverse_zero_imp_zero) | |
| 1138 | apply (blast dest: dvd_mod_imp_dvd) | |
| 1139 | done | |
| 1140 | ||
| 1141 | lemma poly_gcd_greatest: "k dvd x \<Longrightarrow> k dvd y \<Longrightarrow> k dvd poly_gcd x y" | |
| 1142 | by (induct x y rule: poly_gcd.induct) | |
| 1143 | (simp_all add: poly_gcd.simps dvd_mod dvd_smult) | |
| 1144 | ||
| 1145 | lemma dvd_poly_gcd_iff [iff]: | |
| 1146 | "k dvd poly_gcd x y \<longleftrightarrow> k dvd x \<and> k dvd y" | |
| 1147 | by (blast intro!: poly_gcd_greatest intro: dvd_trans) | |
| 1148 | ||
| 1149 | lemma poly_gcd_monic: | |
| 1150 | "coeff (poly_gcd x y) (degree (poly_gcd x y)) = | |
| 1151 | (if x = 0 \<and> y = 0 then 0 else 1)" | |
| 1152 | by (induct x y rule: poly_gcd.induct) | |
| 1153 | (simp_all add: poly_gcd.simps nonzero_imp_inverse_nonzero) | |
| 1154 | ||
| 1155 | lemma poly_gcd_zero_iff [simp]: | |
| 1156 | "poly_gcd x y = 0 \<longleftrightarrow> x = 0 \<and> y = 0" | |
| 1157 | by (simp only: dvd_0_left_iff [symmetric] dvd_poly_gcd_iff) | |
| 1158 | ||
| 1159 | lemma poly_gcd_0_0 [simp]: "poly_gcd 0 0 = 0" | |
| 1160 | by simp | |
| 1161 | ||
| 1162 | lemma poly_dvd_antisym: | |
| 1163 | fixes p q :: "'a::idom poly" | |
| 1164 | assumes coeff: "coeff p (degree p) = coeff q (degree q)" | |
| 1165 | assumes dvd1: "p dvd q" and dvd2: "q dvd p" shows "p = q" | |
| 1166 | proof (cases "p = 0") | |
| 1167 | case True with coeff show "p = q" by simp | |
| 1168 | next | |
| 1169 | case False with coeff have "q \<noteq> 0" by auto | |
| 1170 | have degree: "degree p = degree q" | |
| 1171 | using `p dvd q` `q dvd p` `p \<noteq> 0` `q \<noteq> 0` | |
| 1172 | by (intro order_antisym dvd_imp_degree_le) | |
| 1173 | ||
| 1174 | from `p dvd q` obtain a where a: "q = p * a" .. | |
| 1175 | with `q \<noteq> 0` have "a \<noteq> 0" by auto | |
| 1176 | with degree a `p \<noteq> 0` have "degree a = 0" | |
| 1177 | by (simp add: degree_mult_eq) | |
| 1178 | with coeff a show "p = q" | |
| 1179 | by (cases a, auto split: if_splits) | |
| 1180 | qed | |
| 1181 | ||
| 1182 | lemma poly_gcd_unique: | |
| 1183 | assumes dvd1: "d dvd x" and dvd2: "d dvd y" | |
| 1184 | and greatest: "\<And>k. k dvd x \<Longrightarrow> k dvd y \<Longrightarrow> k dvd d" | |
| 1185 | and monic: "coeff d (degree d) = (if x = 0 \<and> y = 0 then 0 else 1)" | |
| 1186 | shows "poly_gcd x y = d" | |
| 1187 | proof - | |
| 1188 | have "coeff (poly_gcd x y) (degree (poly_gcd x y)) = coeff d (degree d)" | |
| 1189 | by (simp_all add: poly_gcd_monic monic) | |
| 1190 | moreover have "poly_gcd x y dvd d" | |
| 1191 | using poly_gcd_dvd1 poly_gcd_dvd2 by (rule greatest) | |
| 1192 | moreover have "d dvd poly_gcd x y" | |
| 1193 | using dvd1 dvd2 by (rule poly_gcd_greatest) | |
| 1194 | ultimately show ?thesis | |
| 1195 | by (rule poly_dvd_antisym) | |
| 1196 | qed | |
| 1197 | ||
| 37770 
cddb3106adb8
avoid explicit mandatory prefix markers when prefixes are mandatory implicitly
 haftmann parents: 
37765diff
changeset | 1198 | interpretation poly_gcd: abel_semigroup poly_gcd | 
| 34973 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1199 | proof | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1200 | fix x y z :: "'a poly" | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1201 | show "poly_gcd (poly_gcd x y) z = poly_gcd x (poly_gcd y z)" | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1202 | by (rule poly_gcd_unique) (auto intro: dvd_trans simp add: poly_gcd_monic) | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1203 | show "poly_gcd x y = poly_gcd y x" | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1204 | by (rule poly_gcd_unique) (simp_all add: poly_gcd_monic) | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1205 | qed | 
| 31663 | 1206 | |
| 34973 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1207 | lemmas poly_gcd_assoc = poly_gcd.assoc | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1208 | lemmas poly_gcd_commute = poly_gcd.commute | 
| 
ae634fad947e
dropped mk_left_commute; use interpretation of locale abel_semigroup instead
 haftmann parents: 
34915diff
changeset | 1209 | lemmas poly_gcd_left_commute = poly_gcd.left_commute | 
| 31663 | 1210 | |
| 1211 | lemmas poly_gcd_ac = poly_gcd_assoc poly_gcd_commute poly_gcd_left_commute | |
| 1212 | ||
| 1213 | lemma poly_gcd_1_left [simp]: "poly_gcd 1 y = 1" | |
| 1214 | by (rule poly_gcd_unique) simp_all | |
| 1215 | ||
| 1216 | lemma poly_gcd_1_right [simp]: "poly_gcd x 1 = 1" | |
| 1217 | by (rule poly_gcd_unique) simp_all | |
| 1218 | ||
| 1219 | lemma poly_gcd_minus_left [simp]: "poly_gcd (- x) y = poly_gcd x y" | |
| 1220 | by (rule poly_gcd_unique) (simp_all add: poly_gcd_monic) | |
| 1221 | ||
| 1222 | lemma poly_gcd_minus_right [simp]: "poly_gcd x (- y) = poly_gcd x y" | |
| 1223 | by (rule poly_gcd_unique) (simp_all add: poly_gcd_monic) | |
| 1224 | ||
| 1225 | ||
| 29451 | 1226 | subsection {* Evaluation of polynomials *}
 | 
| 1227 | ||
| 1228 | definition | |
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1229 | poly :: "'a::comm_semiring_0 poly \<Rightarrow> 'a \<Rightarrow> 'a" where | 
| 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1230 | "poly = poly_rec (\<lambda>x. 0) (\<lambda>a p f x. a + x * f x)" | 
| 29451 | 1231 | |
| 1232 | lemma poly_0 [simp]: "poly 0 x = 0" | |
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1233 | unfolding poly_def by (simp add: poly_rec_0) | 
| 29451 | 1234 | |
| 1235 | lemma poly_pCons [simp]: "poly (pCons a p) x = a + x * poly p x" | |
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1236 | unfolding poly_def by (simp add: poly_rec_pCons) | 
| 29451 | 1237 | |
| 1238 | lemma poly_1 [simp]: "poly 1 x = 1" | |
| 1239 | unfolding one_poly_def by simp | |
| 1240 | ||
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1241 | lemma poly_monom: | 
| 31021 | 1242 |   fixes a x :: "'a::{comm_semiring_1}"
 | 
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1243 | shows "poly (monom a n) x = a * x ^ n" | 
| 29451 | 1244 | by (induct n, simp add: monom_0, simp add: monom_Suc power_Suc mult_ac) | 
| 1245 | ||
| 1246 | lemma poly_add [simp]: "poly (p + q) x = poly p x + poly q x" | |
| 1247 | apply (induct p arbitrary: q, simp) | |
| 29667 | 1248 | apply (case_tac q, simp, simp add: algebra_simps) | 
| 29451 | 1249 | done | 
| 1250 | ||
| 1251 | lemma poly_minus [simp]: | |
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1252 | fixes x :: "'a::comm_ring" | 
| 29451 | 1253 | shows "poly (- p) x = - poly p x" | 
| 1254 | by (induct p, simp_all) | |
| 1255 | ||
| 1256 | lemma poly_diff [simp]: | |
| 29454 
b0f586f38dd7
add recursion combinator poly_rec; define poly function using poly_rec
 huffman parents: 
29453diff
changeset | 1257 | fixes x :: "'a::comm_ring" | 
| 29451 | 1258 | shows "poly (p - q) x = poly p x - poly q x" | 
| 1259 | by (simp add: diff_minus) | |
| 1260 | ||
| 1261 | lemma poly_setsum: "poly (\<Sum>k\<in>A. p k) x = (\<Sum>k\<in>A. poly (p k) x)" | |
| 1262 | by (cases "finite A", induct set: finite, simp_all) | |
| 1263 | ||
| 1264 | lemma poly_smult [simp]: "poly (smult a p) x = a * poly p x" | |
| 29667 | 1265 | by (induct p, simp, simp add: algebra_simps) | 
| 29451 | 1266 | |
| 1267 | lemma poly_mult [simp]: "poly (p * q) x = poly p x * poly q x" | |
| 29667 | 1268 | by (induct p, simp_all, simp add: algebra_simps) | 
| 29451 | 1269 | |
| 29462 | 1270 | lemma poly_power [simp]: | 
| 31021 | 1271 |   fixes p :: "'a::{comm_semiring_1} poly"
 | 
| 29462 | 1272 | shows "poly (p ^ n) x = poly p x ^ n" | 
| 1273 | by (induct n, simp, simp add: power_Suc) | |
| 1274 | ||
| 29456 | 1275 | |
| 1276 | subsection {* Synthetic division *}
 | |
| 1277 | ||
| 29980 | 1278 | text {*
 | 
| 1279 | Synthetic division is simply division by the | |
| 1280 |   linear polynomial @{term "x - c"}.
 | |
| 1281 | *} | |
| 1282 | ||
| 29456 | 1283 | definition | 
| 1284 | synthetic_divmod :: "'a::comm_semiring_0 poly \<Rightarrow> 'a \<Rightarrow> 'a poly \<times> 'a" | |
| 37765 | 1285 | where | 
| 29456 | 1286 | "synthetic_divmod p c = | 
| 1287 | poly_rec (0, 0) (\<lambda>a p (q, r). (pCons r q, a + c * r)) p" | |
| 1288 | ||
| 1289 | definition | |
| 1290 | synthetic_div :: "'a::comm_semiring_0 poly \<Rightarrow> 'a \<Rightarrow> 'a poly" | |
| 1291 | where | |
| 1292 | "synthetic_div p c = fst (synthetic_divmod p c)" | |
| 1293 | ||
| 1294 | lemma synthetic_divmod_0 [simp]: | |
| 1295 | "synthetic_divmod 0 c = (0, 0)" | |
| 1296 | unfolding synthetic_divmod_def | |
| 1297 | by (simp add: poly_rec_0) | |
| 1298 | ||
| 1299 | lemma synthetic_divmod_pCons [simp]: | |
| 1300 | "synthetic_divmod (pCons a p) c = | |
| 1301 | (\<lambda>(q, r). (pCons r q, a + c * r)) (synthetic_divmod p c)" | |
| 1302 | unfolding synthetic_divmod_def | |
| 1303 | by (simp add: poly_rec_pCons) | |
| 1304 | ||
| 1305 | lemma snd_synthetic_divmod: "snd (synthetic_divmod p c) = poly p c" | |
| 1306 | by (induct p, simp, simp add: split_def) | |
| 1307 | ||
| 1308 | lemma synthetic_div_0 [simp]: "synthetic_div 0 c = 0" | |
| 1309 | unfolding synthetic_div_def by simp | |
| 1310 | ||
| 1311 | lemma synthetic_div_pCons [simp]: | |
| 1312 | "synthetic_div (pCons a p) c = pCons (poly p c) (synthetic_div p c)" | |
| 1313 | unfolding synthetic_div_def | |
| 1314 | by (simp add: split_def snd_synthetic_divmod) | |
| 1315 | ||
| 29460 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1316 | lemma synthetic_div_eq_0_iff: | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1317 | "synthetic_div p c = 0 \<longleftrightarrow> degree p = 0" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1318 | by (induct p, simp, case_tac p, simp) | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1319 | |
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1320 | lemma degree_synthetic_div: | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1321 | "degree (synthetic_div p c) = degree p - 1" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1322 | by (induct p, simp, simp add: synthetic_div_eq_0_iff) | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1323 | |
| 29457 | 1324 | lemma synthetic_div_correct: | 
| 29456 | 1325 | "p + smult c (synthetic_div p c) = pCons (poly p c) (synthetic_div p c)" | 
| 1326 | by (induct p) simp_all | |
| 1327 | ||
| 29457 | 1328 | lemma synthetic_div_unique_lemma: "smult c p = pCons a p \<Longrightarrow> p = 0" | 
| 1329 | by (induct p arbitrary: a) simp_all | |
| 1330 | ||
| 1331 | lemma synthetic_div_unique: | |
| 1332 | "p + smult c q = pCons r q \<Longrightarrow> r = poly p c \<and> q = synthetic_div p c" | |
| 1333 | apply (induct p arbitrary: q r) | |
| 1334 | apply (simp, frule synthetic_div_unique_lemma, simp) | |
| 1335 | apply (case_tac q, force) | |
| 1336 | done | |
| 1337 | ||
| 1338 | lemma synthetic_div_correct': | |
| 1339 | fixes c :: "'a::comm_ring_1" | |
| 1340 | shows "[:-c, 1:] * synthetic_div p c + [:poly p c:] = p" | |
| 1341 | using synthetic_div_correct [of p c] | |
| 29667 | 1342 | by (simp add: algebra_simps) | 
| 29457 | 1343 | |
| 29460 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1344 | lemma poly_eq_0_iff_dvd: | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1345 | fixes c :: "'a::idom" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1346 | shows "poly p c = 0 \<longleftrightarrow> [:-c, 1:] dvd p" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1347 | proof | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1348 | assume "poly p c = 0" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1349 | with synthetic_div_correct' [of c p] | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1350 | have "p = [:-c, 1:] * synthetic_div p c" by simp | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1351 | then show "[:-c, 1:] dvd p" .. | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1352 | next | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1353 | assume "[:-c, 1:] dvd p" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1354 | then obtain k where "p = [:-c, 1:] * k" by (rule dvdE) | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1355 | then show "poly p c = 0" by simp | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1356 | qed | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1357 | |
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1358 | lemma dvd_iff_poly_eq_0: | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1359 | fixes c :: "'a::idom" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1360 | shows "[:c, 1:] dvd p \<longleftrightarrow> poly p (-c) = 0" | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1361 | by (simp add: poly_eq_0_iff_dvd) | 
| 
ad87e5d1488b
new lemmas about synthetic_div; declare degree_pCons_eq_if [simp]
 huffman parents: 
29457diff
changeset | 1362 | |
| 29462 | 1363 | lemma poly_roots_finite: | 
| 1364 | fixes p :: "'a::idom poly" | |
| 1365 |   shows "p \<noteq> 0 \<Longrightarrow> finite {x. poly p x = 0}"
 | |
| 1366 | proof (induct n \<equiv> "degree p" arbitrary: p) | |
| 1367 | case (0 p) | |
| 1368 | then obtain a where "a \<noteq> 0" and "p = [:a:]" | |
| 1369 | by (cases p, simp split: if_splits) | |
| 1370 |   then show "finite {x. poly p x = 0}" by simp
 | |
| 1371 | next | |
| 1372 | case (Suc n p) | |
| 1373 |   show "finite {x. poly p x = 0}"
 | |
| 1374 | proof (cases "\<exists>x. poly p x = 0") | |
| 1375 | case False | |
| 1376 |     then show "finite {x. poly p x = 0}" by simp
 | |
| 1377 | next | |
| 1378 | case True | |
| 1379 | then obtain a where "poly p a = 0" .. | |
| 1380 | then have "[:-a, 1:] dvd p" by (simp only: poly_eq_0_iff_dvd) | |
| 1381 | then obtain k where k: "p = [:-a, 1:] * k" .. | |
| 1382 | with `p \<noteq> 0` have "k \<noteq> 0" by auto | |
| 1383 | with k have "degree p = Suc (degree k)" | |
| 1384 | by (simp add: degree_mult_eq del: mult_pCons_left) | |
| 1385 | with `Suc n = degree p` have "n = degree k" by simp | |
| 34915 | 1386 |     then have "finite {x. poly k x = 0}" using `k \<noteq> 0` by (rule Suc.hyps)
 | 
| 29462 | 1387 |     then have "finite (insert a {x. poly k x = 0})" by simp
 | 
| 1388 |     then show "finite {x. poly p x = 0}"
 | |
| 1389 | by (simp add: k uminus_add_conv_diff Collect_disj_eq | |
| 1390 | del: mult_pCons_left) | |
| 1391 | qed | |
| 1392 | qed | |
| 1393 | ||
| 29979 | 1394 | lemma poly_zero: | 
| 1395 |   fixes p :: "'a::{idom,ring_char_0} poly"
 | |
| 1396 | shows "poly p = poly 0 \<longleftrightarrow> p = 0" | |
| 1397 | apply (cases "p = 0", simp_all) | |
| 1398 | apply (drule poly_roots_finite) | |
| 1399 | apply (auto simp add: infinite_UNIV_char_0) | |
| 1400 | done | |
| 1401 | ||
| 1402 | lemma poly_eq_iff: | |
| 1403 |   fixes p q :: "'a::{idom,ring_char_0} poly"
 | |
| 1404 | shows "poly p = poly q \<longleftrightarrow> p = q" | |
| 1405 | using poly_zero [of "p - q"] | |
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 1406 | by (simp add: fun_eq_iff) | 
| 29979 | 1407 | |
| 29478 | 1408 | |
| 29980 | 1409 | subsection {* Composition of polynomials *}
 | 
| 1410 | ||
| 1411 | definition | |
| 1412 | pcompose :: "'a::comm_semiring_0 poly \<Rightarrow> 'a poly \<Rightarrow> 'a poly" | |
| 1413 | where | |
| 1414 | "pcompose p q = poly_rec 0 (\<lambda>a _ c. [:a:] + q * c) p" | |
| 1415 | ||
| 1416 | lemma pcompose_0 [simp]: "pcompose 0 q = 0" | |
| 1417 | unfolding pcompose_def by (simp add: poly_rec_0) | |
| 1418 | ||
| 1419 | lemma pcompose_pCons: | |
| 1420 | "pcompose (pCons a p) q = [:a:] + q * pcompose p q" | |
| 1421 | unfolding pcompose_def by (simp add: poly_rec_pCons) | |
| 1422 | ||
| 1423 | lemma poly_pcompose: "poly (pcompose p q) x = poly p (poly q x)" | |
| 1424 | by (induct p) (simp_all add: pcompose_pCons) | |
| 1425 | ||
| 1426 | lemma degree_pcompose_le: | |
| 1427 | "degree (pcompose p q) \<le> degree p * degree q" | |
| 1428 | apply (induct p, simp) | |
| 1429 | apply (simp add: pcompose_pCons, clarify) | |
| 1430 | apply (rule degree_add_le, simp) | |
| 1431 | apply (rule order_trans [OF degree_mult_le], simp) | |
| 1432 | done | |
| 1433 | ||
| 1434 | ||
| 29977 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1435 | subsection {* Order of polynomial roots *}
 | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1436 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1437 | definition | 
| 29979 | 1438 | order :: "'a::idom \<Rightarrow> 'a poly \<Rightarrow> nat" | 
| 29977 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1439 | where | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1440 | "order a p = (LEAST n. \<not> [:-a, 1:] ^ Suc n dvd p)" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1441 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1442 | lemma coeff_linear_power: | 
| 29979 | 1443 | fixes a :: "'a::comm_semiring_1" | 
| 29977 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1444 | shows "coeff ([:a, 1:] ^ n) n = 1" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1445 | apply (induct n, simp_all) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1446 | apply (subst coeff_eq_0) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1447 | apply (auto intro: le_less_trans degree_power_le) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1448 | done | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1449 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1450 | lemma degree_linear_power: | 
| 29979 | 1451 | fixes a :: "'a::comm_semiring_1" | 
| 29977 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1452 | shows "degree ([:a, 1:] ^ n) = n" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1453 | apply (rule order_antisym) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1454 | apply (rule ord_le_eq_trans [OF degree_power_le], simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1455 | apply (rule le_degree, simp add: coeff_linear_power) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1456 | done | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1457 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1458 | lemma order_1: "[:-a, 1:] ^ order a p dvd p" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1459 | apply (cases "p = 0", simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1460 | apply (cases "order a p", simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1461 | apply (subgoal_tac "nat < (LEAST n. \<not> [:-a, 1:] ^ Suc n dvd p)") | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1462 | apply (drule not_less_Least, simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1463 | apply (fold order_def, simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1464 | done | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1465 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1466 | lemma order_2: "p \<noteq> 0 \<Longrightarrow> \<not> [:-a, 1:] ^ Suc (order a p) dvd p" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1467 | unfolding order_def | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1468 | apply (rule LeastI_ex) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1469 | apply (rule_tac x="degree p" in exI) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1470 | apply (rule notI) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1471 | apply (drule (1) dvd_imp_degree_le) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1472 | apply (simp only: degree_linear_power) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1473 | done | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1474 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1475 | lemma order: | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1476 | "p \<noteq> 0 \<Longrightarrow> [:-a, 1:] ^ order a p dvd p \<and> \<not> [:-a, 1:] ^ Suc (order a p) dvd p" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1477 | by (rule conjI [OF order_1 order_2]) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1478 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1479 | lemma order_degree: | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1480 | assumes p: "p \<noteq> 0" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1481 | shows "order a p \<le> degree p" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1482 | proof - | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1483 | have "order a p = degree ([:-a, 1:] ^ order a p)" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1484 | by (simp only: degree_linear_power) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1485 | also have "\<dots> \<le> degree p" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1486 | using order_1 p by (rule dvd_imp_degree_le) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1487 | finally show ?thesis . | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1488 | qed | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1489 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1490 | lemma order_root: "poly p a = 0 \<longleftrightarrow> p = 0 \<or> order a p \<noteq> 0" | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1491 | apply (cases "p = 0", simp_all) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1492 | apply (rule iffI) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1493 | apply (rule ccontr, simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1494 | apply (frule order_2 [where a=a], simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1495 | apply (simp add: poly_eq_0_iff_dvd) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1496 | apply (simp add: poly_eq_0_iff_dvd) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1497 | apply (simp only: order_def) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1498 | apply (drule not_less_Least, simp) | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1499 | done | 
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1500 | |
| 
d76b830366bc
move polynomial order stuff from Fundamental_Theorem_Algebra to Polynomial
 huffman parents: 
29904diff
changeset | 1501 | |
| 29478 | 1502 | subsection {* Configuration of the code generator *}
 | 
| 1503 | ||
| 1504 | code_datatype "0::'a::zero poly" pCons | |
| 1505 | ||
| 31998 
2c7a24f74db9
code attributes use common underscore convention
 haftmann parents: 
31663diff
changeset | 1506 | declare pCons_0_0 [code_post] | 
| 29480 | 1507 | |
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1508 | instantiation poly :: ("{zero, equal}") equal
 | 
| 29478 | 1509 | begin | 
| 1510 | ||
| 37765 | 1511 | definition | 
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1512 | "HOL.equal (p::'a poly) q \<longleftrightarrow> p = q" | 
| 29478 | 1513 | |
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1514 | instance proof | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1515 | qed (rule equal_poly_def) | 
| 29478 | 1516 | |
| 29451 | 1517 | end | 
| 29478 | 1518 | |
| 1519 | lemma eq_poly_code [code]: | |
| 38857 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1520 | "HOL.equal (0::_ poly) (0::_ poly) \<longleftrightarrow> True" | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1521 | "HOL.equal (0::_ poly) (pCons b q) \<longleftrightarrow> HOL.equal 0 b \<and> HOL.equal 0 q" | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1522 | "HOL.equal (pCons a p) (0::_ poly) \<longleftrightarrow> HOL.equal a 0 \<and> HOL.equal p 0" | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1523 | "HOL.equal (pCons a p) (pCons b q) \<longleftrightarrow> HOL.equal a b \<and> HOL.equal p q" | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1524 | by (simp_all add: equal) | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1525 | |
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1526 | lemma [code nbe]: | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1527 | "HOL.equal (p :: _ poly) p \<longleftrightarrow> True" | 
| 
97775f3e8722
renamed class/constant eq to equal; tuned some instantiations
 haftmann parents: 
37770diff
changeset | 1528 | by (fact equal_refl) | 
| 29478 | 1529 | |
| 1530 | lemmas coeff_code [code] = | |
| 1531 | coeff_0 coeff_pCons_0 coeff_pCons_Suc | |
| 1532 | ||
| 1533 | lemmas degree_code [code] = | |
| 1534 | degree_0 degree_pCons_eq_if | |
| 1535 | ||
| 1536 | lemmas monom_poly_code [code] = | |
| 1537 | monom_0 monom_Suc | |
| 1538 | ||
| 1539 | lemma add_poly_code [code]: | |
| 1540 | "0 + q = (q :: _ poly)" | |
| 1541 | "p + 0 = (p :: _ poly)" | |
| 1542 | "pCons a p + pCons b q = pCons (a + b) (p + q)" | |
| 1543 | by simp_all | |
| 1544 | ||
| 1545 | lemma minus_poly_code [code]: | |
| 1546 | "- 0 = (0 :: _ poly)" | |
| 1547 | "- pCons a p = pCons (- a) (- p)" | |
| 1548 | by simp_all | |
| 1549 | ||
| 1550 | lemma diff_poly_code [code]: | |
| 1551 | "0 - q = (- q :: _ poly)" | |
| 1552 | "p - 0 = (p :: _ poly)" | |
| 1553 | "pCons a p - pCons b q = pCons (a - b) (p - q)" | |
| 1554 | by simp_all | |
| 1555 | ||
| 1556 | lemmas smult_poly_code [code] = | |
| 1557 | smult_0_right smult_pCons | |
| 1558 | ||
| 1559 | lemma mult_poly_code [code]: | |
| 1560 | "0 * q = (0 :: _ poly)" | |
| 1561 | "pCons a p * q = smult a q + pCons 0 (p * q)" | |
| 1562 | by simp_all | |
| 1563 | ||
| 1564 | lemmas poly_code [code] = | |
| 1565 | poly_0 poly_pCons | |
| 1566 | ||
| 1567 | lemmas synthetic_divmod_code [code] = | |
| 1568 | synthetic_divmod_0 synthetic_divmod_pCons | |
| 1569 | ||
| 1570 | text {* code generator setup for div and mod *}
 | |
| 1571 | ||
| 1572 | definition | |
| 29537 | 1573 | pdivmod :: "'a::field poly \<Rightarrow> 'a poly \<Rightarrow> 'a poly \<times> 'a poly" | 
| 29478 | 1574 | where | 
| 37765 | 1575 | "pdivmod x y = (x div y, x mod y)" | 
| 29478 | 1576 | |
| 29537 | 1577 | lemma div_poly_code [code]: "x div y = fst (pdivmod x y)" | 
| 1578 | unfolding pdivmod_def by simp | |
| 29478 | 1579 | |
| 29537 | 1580 | lemma mod_poly_code [code]: "x mod y = snd (pdivmod x y)" | 
| 1581 | unfolding pdivmod_def by simp | |
| 29478 | 1582 | |
| 29537 | 1583 | lemma pdivmod_0 [code]: "pdivmod 0 y = (0, 0)" | 
| 1584 | unfolding pdivmod_def by simp | |
| 29478 | 1585 | |
| 29537 | 1586 | lemma pdivmod_pCons [code]: | 
| 1587 | "pdivmod (pCons a x) y = | |
| 29478 | 1588 | (if y = 0 then (0, pCons a x) else | 
| 29537 | 1589 | (let (q, r) = pdivmod x y; | 
| 29478 | 1590 | b = coeff (pCons a r) (degree y) / coeff y (degree y) | 
| 1591 | in (pCons b q, pCons a r - smult b y)))" | |
| 29537 | 1592 | apply (simp add: pdivmod_def Let_def, safe) | 
| 29478 | 1593 | apply (rule div_poly_eq) | 
| 29537 | 1594 | apply (erule pdivmod_rel_pCons [OF pdivmod_rel _ refl]) | 
| 29478 | 1595 | apply (rule mod_poly_eq) | 
| 29537 | 1596 | apply (erule pdivmod_rel_pCons [OF pdivmod_rel _ refl]) | 
| 29478 | 1597 | done | 
| 1598 | ||
| 31663 | 1599 | lemma poly_gcd_code [code]: | 
| 1600 | "poly_gcd x y = | |
| 1601 | (if y = 0 then smult (inverse (coeff x (degree x))) x | |
| 1602 | else poly_gcd y (x mod y))" | |
| 1603 | by (simp add: poly_gcd.simps) | |
| 1604 | ||
| 29478 | 1605 | end |