author | haftmann |
Tue, 23 Jun 2009 14:24:58 +0200 | |
changeset 31776 | 151c3f5f28f9 |
parent 31706 | 1db0c8f235fb |
child 31952 | 40501bb2d57c |
permissions | -rw-r--r-- |
21256 | 1 |
(* Title: HOL/GCD.thy |
2 |
Author: Christophe Tabacznyj and Lawrence C Paulson |
|
3 |
Copyright 1996 University of Cambridge |
|
4 |
*) |
|
5 |
||
6 |
header {* The Greatest Common Divisor *} |
|
7 |
||
31706 | 8 |
theory Legacy_GCD |
30738 | 9 |
imports Main |
21256 | 10 |
begin |
11 |
||
12 |
text {* |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
13 |
See \cite{davenport92}. \bigskip |
21256 | 14 |
*} |
15 |
||
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
16 |
subsection {* Specification of GCD on nats *} |
21256 | 17 |
|
21263 | 18 |
definition |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
19 |
is_gcd :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> bool" where -- {* @{term gcd} as a relation *} |
28562 | 20 |
[code del]: "is_gcd m n p \<longleftrightarrow> p dvd m \<and> p dvd n \<and> |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
21 |
(\<forall>d. d dvd m \<longrightarrow> d dvd n \<longrightarrow> d dvd p)" |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
22 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
23 |
text {* Uniqueness *} |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
24 |
|
27556 | 25 |
lemma is_gcd_unique: "is_gcd a b m \<Longrightarrow> is_gcd a b n \<Longrightarrow> m = n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
26 |
by (simp add: is_gcd_def) (blast intro: dvd_anti_sym) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
27 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
28 |
text {* Connection to divides relation *} |
21256 | 29 |
|
27556 | 30 |
lemma is_gcd_dvd: "is_gcd a b m \<Longrightarrow> k dvd a \<Longrightarrow> k dvd b \<Longrightarrow> k dvd m" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
31 |
by (auto simp add: is_gcd_def) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
32 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
33 |
text {* Commutativity *} |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
34 |
|
27556 | 35 |
lemma is_gcd_commute: "is_gcd m n k = is_gcd n m k" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
36 |
by (auto simp add: is_gcd_def) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
37 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
38 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
39 |
subsection {* GCD on nat by Euclid's algorithm *} |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
40 |
|
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
41 |
fun |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
42 |
gcd :: "nat => nat => nat" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
43 |
where |
27556 | 44 |
"gcd m n = (if n = 0 then m else gcd n (m mod n))" |
45 |
lemma gcd_induct [case_names "0" rec]: |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
46 |
fixes m n :: nat |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
47 |
assumes "\<And>m. P m 0" |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
48 |
and "\<And>m n. 0 < n \<Longrightarrow> P n (m mod n) \<Longrightarrow> P m n" |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
49 |
shows "P m n" |
27556 | 50 |
proof (induct m n rule: gcd.induct) |
51 |
case (1 m n) with assms show ?case by (cases "n = 0") simp_all |
|
52 |
qed |
|
21256 | 53 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
54 |
lemma gcd_0 [simp, algebra]: "gcd m 0 = m" |
21263 | 55 |
by simp |
21256 | 56 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
57 |
lemma gcd_0_left [simp,algebra]: "gcd 0 m = m" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
58 |
by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
59 |
|
27556 | 60 |
lemma gcd_non_0: "n > 0 \<Longrightarrow> gcd m n = gcd n (m mod n)" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
61 |
by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
62 |
|
30082
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
63 |
lemma gcd_1 [simp, algebra]: "gcd m (Suc 0) = Suc 0" |
21263 | 64 |
by simp |
21256 | 65 |
|
30082
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
66 |
lemma nat_gcd_1_right [simp, algebra]: "gcd m 1 = 1" |
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
67 |
unfolding One_nat_def by (rule gcd_1) |
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
68 |
|
21256 | 69 |
declare gcd.simps [simp del] |
70 |
||
71 |
text {* |
|
27556 | 72 |
\medskip @{term "gcd m n"} divides @{text m} and @{text n}. The |
21256 | 73 |
conjunctions don't seem provable separately. |
74 |
*} |
|
75 |
||
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
76 |
lemma gcd_dvd1 [iff, algebra]: "gcd m n dvd m" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
77 |
and gcd_dvd2 [iff, algebra]: "gcd m n dvd n" |
21256 | 78 |
apply (induct m n rule: gcd_induct) |
21263 | 79 |
apply (simp_all add: gcd_non_0) |
21256 | 80 |
apply (blast dest: dvd_mod_imp_dvd) |
81 |
done |
|
82 |
||
83 |
text {* |
|
84 |
\medskip Maximality: for all @{term m}, @{term n}, @{term k} |
|
85 |
naturals, if @{term k} divides @{term m} and @{term k} divides |
|
27556 | 86 |
@{term n} then @{term k} divides @{term "gcd m n"}. |
21256 | 87 |
*} |
88 |
||
27556 | 89 |
lemma gcd_greatest: "k dvd m \<Longrightarrow> k dvd n \<Longrightarrow> k dvd gcd m n" |
21263 | 90 |
by (induct m n rule: gcd_induct) (simp_all add: gcd_non_0 dvd_mod) |
21256 | 91 |
|
92 |
text {* |
|
93 |
\medskip Function gcd yields the Greatest Common Divisor. |
|
94 |
*} |
|
95 |
||
27556 | 96 |
lemma is_gcd: "is_gcd m n (gcd m n) " |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
97 |
by (simp add: is_gcd_def gcd_greatest) |
21256 | 98 |
|
99 |
||
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
100 |
subsection {* Derived laws for GCD *} |
21256 | 101 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
102 |
lemma gcd_greatest_iff [iff, algebra]: "k dvd gcd m n \<longleftrightarrow> k dvd m \<and> k dvd n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
103 |
by (blast intro!: gcd_greatest intro: dvd_trans) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
104 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
105 |
lemma gcd_zero[algebra]: "gcd m n = 0 \<longleftrightarrow> m = 0 \<and> n = 0" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
106 |
by (simp only: dvd_0_left_iff [symmetric] gcd_greatest_iff) |
21256 | 107 |
|
27556 | 108 |
lemma gcd_commute: "gcd m n = gcd n m" |
21256 | 109 |
apply (rule is_gcd_unique) |
110 |
apply (rule is_gcd) |
|
111 |
apply (subst is_gcd_commute) |
|
112 |
apply (simp add: is_gcd) |
|
113 |
done |
|
114 |
||
27556 | 115 |
lemma gcd_assoc: "gcd (gcd k m) n = gcd k (gcd m n)" |
21256 | 116 |
apply (rule is_gcd_unique) |
117 |
apply (rule is_gcd) |
|
118 |
apply (simp add: is_gcd_def) |
|
119 |
apply (blast intro: dvd_trans) |
|
120 |
done |
|
121 |
||
30082
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
122 |
lemma gcd_1_left [simp, algebra]: "gcd (Suc 0) m = Suc 0" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
123 |
by (simp add: gcd_commute) |
21256 | 124 |
|
30082
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
125 |
lemma nat_gcd_1_left [simp, algebra]: "gcd 1 m = 1" |
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
126 |
unfolding One_nat_def by (rule gcd_1_left) |
43c5b7bfc791
make more proofs work whether or not One_nat_def is a simp rule
huffman
parents:
30042
diff
changeset
|
127 |
|
21256 | 128 |
text {* |
129 |
\medskip Multiplication laws |
|
130 |
*} |
|
131 |
||
27556 | 132 |
lemma gcd_mult_distrib2: "k * gcd m n = gcd (k * m) (k * n)" |
21256 | 133 |
-- {* \cite[page 27]{davenport92} *} |
134 |
apply (induct m n rule: gcd_induct) |
|
135 |
apply simp |
|
136 |
apply (case_tac "k = 0") |
|
137 |
apply (simp_all add: mod_geq gcd_non_0 mod_mult_distrib2) |
|
138 |
done |
|
139 |
||
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
140 |
lemma gcd_mult [simp, algebra]: "gcd k (k * n) = k" |
21256 | 141 |
apply (rule gcd_mult_distrib2 [of k 1 n, simplified, symmetric]) |
142 |
done |
|
143 |
||
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
144 |
lemma gcd_self [simp, algebra]: "gcd k k = k" |
21256 | 145 |
apply (rule gcd_mult [of k 1, simplified]) |
146 |
done |
|
147 |
||
27556 | 148 |
lemma relprime_dvd_mult: "gcd k n = 1 ==> k dvd m * n ==> k dvd m" |
21256 | 149 |
apply (insert gcd_mult_distrib2 [of m k n]) |
150 |
apply simp |
|
151 |
apply (erule_tac t = m in ssubst) |
|
152 |
apply simp |
|
153 |
done |
|
154 |
||
27556 | 155 |
lemma relprime_dvd_mult_iff: "gcd k n = 1 ==> (k dvd m * n) = (k dvd m)" |
27651
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
haftmann
parents:
27568
diff
changeset
|
156 |
by (auto intro: relprime_dvd_mult dvd_mult2) |
21256 | 157 |
|
27556 | 158 |
lemma gcd_mult_cancel: "gcd k n = 1 ==> gcd (k * m) n = gcd m n" |
21256 | 159 |
apply (rule dvd_anti_sym) |
160 |
apply (rule gcd_greatest) |
|
161 |
apply (rule_tac n = k in relprime_dvd_mult) |
|
162 |
apply (simp add: gcd_assoc) |
|
163 |
apply (simp add: gcd_commute) |
|
164 |
apply (simp_all add: mult_commute) |
|
165 |
done |
|
166 |
||
167 |
||
168 |
text {* \medskip Addition laws *} |
|
169 |
||
27676 | 170 |
lemma gcd_add1 [simp, algebra]: "gcd (m + n) n = gcd m n" |
171 |
by (cases "n = 0") (auto simp add: gcd_non_0) |
|
21256 | 172 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
173 |
lemma gcd_add2 [simp, algebra]: "gcd m (m + n) = gcd m n" |
21256 | 174 |
proof - |
27556 | 175 |
have "gcd m (m + n) = gcd (m + n) m" by (rule gcd_commute) |
176 |
also have "... = gcd (n + m) m" by (simp add: add_commute) |
|
177 |
also have "... = gcd n m" by simp |
|
178 |
also have "... = gcd m n" by (rule gcd_commute) |
|
21256 | 179 |
finally show ?thesis . |
180 |
qed |
|
181 |
||
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
182 |
lemma gcd_add2' [simp, algebra]: "gcd m (n + m) = gcd m n" |
21256 | 183 |
apply (subst add_commute) |
184 |
apply (rule gcd_add2) |
|
185 |
done |
|
186 |
||
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
187 |
lemma gcd_add_mult[algebra]: "gcd m (k * m + n) = gcd m n" |
21263 | 188 |
by (induct k) (simp_all add: add_assoc) |
21256 | 189 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
190 |
lemma gcd_dvd_prod: "gcd m n dvd m * n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
191 |
using mult_dvd_mono [of 1] by auto |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
192 |
|
22367 | 193 |
text {* |
194 |
\medskip Division by gcd yields rrelatively primes. |
|
195 |
*} |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
196 |
|
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
197 |
lemma div_gcd_relprime: |
22367 | 198 |
assumes nz: "a \<noteq> 0 \<or> b \<noteq> 0" |
27556 | 199 |
shows "gcd (a div gcd a b) (b div gcd a b) = 1" |
22367 | 200 |
proof - |
27556 | 201 |
let ?g = "gcd a b" |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
202 |
let ?a' = "a div ?g" |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
203 |
let ?b' = "b div ?g" |
27556 | 204 |
let ?g' = "gcd ?a' ?b'" |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
205 |
have dvdg: "?g dvd a" "?g dvd b" by simp_all |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
206 |
have dvdg': "?g' dvd ?a'" "?g' dvd ?b'" by simp_all |
22367 | 207 |
from dvdg dvdg' obtain ka kb ka' kb' where |
208 |
kab: "a = ?g * ka" "b = ?g * kb" "?a' = ?g' * ka'" "?b' = ?g' * kb'" |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
209 |
unfolding dvd_def by blast |
22367 | 210 |
then have "?g * ?a' = (?g * ?g') * ka'" "?g * ?b' = (?g * ?g') * kb'" by simp_all |
211 |
then have dvdgg':"?g * ?g' dvd a" "?g* ?g' dvd b" |
|
212 |
by (auto simp add: dvd_mult_div_cancel [OF dvdg(1)] |
|
213 |
dvd_mult_div_cancel [OF dvdg(2)] dvd_def) |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
214 |
have "?g \<noteq> 0" using nz by (simp add: gcd_zero) |
22367 | 215 |
then have gp: "?g > 0" by simp |
216 |
from gcd_greatest [OF dvdgg'] have "?g * ?g' dvd ?g" . |
|
217 |
with dvd_mult_cancel1 [OF gp] show "?g' = 1" by simp |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
218 |
qed |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
219 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
220 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
221 |
lemma gcd_unique: "d dvd a\<and>d dvd b \<and> (\<forall>e. e dvd a \<and> e dvd b \<longrightarrow> e dvd d) \<longleftrightarrow> d = gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
222 |
proof(auto) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
223 |
assume H: "d dvd a" "d dvd b" "\<forall>e. e dvd a \<and> e dvd b \<longrightarrow> e dvd d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
224 |
from H(3)[rule_format] gcd_dvd1[of a b] gcd_dvd2[of a b] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
225 |
have th: "gcd a b dvd d" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
226 |
from dvd_anti_sym[OF th gcd_greatest[OF H(1,2)]] show "d = gcd a b" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
227 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
228 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
229 |
lemma gcd_eq: assumes H: "\<forall>d. d dvd x \<and> d dvd y \<longleftrightarrow> d dvd u \<and> d dvd v" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
230 |
shows "gcd x y = gcd u v" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
231 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
232 |
from H have "\<forall>d. d dvd x \<and> d dvd y \<longleftrightarrow> d dvd gcd u v" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
233 |
with gcd_unique[of "gcd u v" x y] show ?thesis by auto |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
234 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
235 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
236 |
lemma ind_euclid: |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
237 |
assumes c: " \<forall>a b. P (a::nat) b \<longleftrightarrow> P b a" and z: "\<forall>a. P a 0" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
238 |
and add: "\<forall>a b. P a b \<longrightarrow> P a (a + b)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
239 |
shows "P a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
240 |
proof(induct n\<equiv>"a+b" arbitrary: a b rule: nat_less_induct) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
241 |
fix n a b |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
242 |
assume H: "\<forall>m < n. \<forall>a b. m = a + b \<longrightarrow> P a b" "n = a + b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
243 |
have "a = b \<or> a < b \<or> b < a" by arith |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
244 |
moreover {assume eq: "a= b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
245 |
from add[rule_format, OF z[rule_format, of a]] have "P a b" using eq by simp} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
246 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
247 |
{assume lt: "a < b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
248 |
hence "a + b - a < n \<or> a = 0" using H(2) by arith |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
249 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
250 |
{assume "a =0" with z c have "P a b" by blast } |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
251 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
252 |
{assume ab: "a + b - a < n" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
253 |
have th0: "a + b - a = a + (b - a)" using lt by arith |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
254 |
from add[rule_format, OF H(1)[rule_format, OF ab th0]] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
255 |
have "P a b" by (simp add: th0[symmetric])} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
256 |
ultimately have "P a b" by blast} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
257 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
258 |
{assume lt: "a > b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
259 |
hence "b + a - b < n \<or> b = 0" using H(2) by arith |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
260 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
261 |
{assume "b =0" with z c have "P a b" by blast } |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
262 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
263 |
{assume ab: "b + a - b < n" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
264 |
have th0: "b + a - b = b + (a - b)" using lt by arith |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
265 |
from add[rule_format, OF H(1)[rule_format, OF ab th0]] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
266 |
have "P b a" by (simp add: th0[symmetric]) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
267 |
hence "P a b" using c by blast } |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
268 |
ultimately have "P a b" by blast} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
269 |
ultimately show "P a b" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
270 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
271 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
272 |
lemma bezout_lemma: |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
273 |
assumes ex: "\<exists>(d::nat) x y. d dvd a \<and> d dvd b \<and> (a * x = b * y + d \<or> b * x = a * y + d)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
274 |
shows "\<exists>d x y. d dvd a \<and> d dvd a + b \<and> (a * x = (a + b) * y + d \<or> (a + b) * x = a * y + d)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
275 |
using ex |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
276 |
apply clarsimp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
277 |
apply (rule_tac x="d" in exI, simp add: dvd_add) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
278 |
apply (case_tac "a * x = b * y + d" , simp_all) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
279 |
apply (rule_tac x="x + y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
280 |
apply (rule_tac x="y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
281 |
apply algebra |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
282 |
apply (rule_tac x="x" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
283 |
apply (rule_tac x="x + y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
284 |
apply algebra |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
285 |
done |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
286 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
287 |
lemma bezout_add: "\<exists>(d::nat) x y. d dvd a \<and> d dvd b \<and> (a * x = b * y + d \<or> b * x = a * y + d)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
288 |
apply(induct a b rule: ind_euclid) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
289 |
apply blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
290 |
apply clarify |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
291 |
apply (rule_tac x="a" in exI, simp add: dvd_add) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
292 |
apply clarsimp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
293 |
apply (rule_tac x="d" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
294 |
apply (case_tac "a * x = b * y + d", simp_all add: dvd_add) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
295 |
apply (rule_tac x="x+y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
296 |
apply (rule_tac x="y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
297 |
apply algebra |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
298 |
apply (rule_tac x="x" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
299 |
apply (rule_tac x="x+y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
300 |
apply algebra |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
301 |
done |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
302 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
303 |
lemma bezout: "\<exists>(d::nat) x y. d dvd a \<and> d dvd b \<and> (a * x - b * y = d \<or> b * x - a * y = d)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
304 |
using bezout_add[of a b] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
305 |
apply clarsimp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
306 |
apply (rule_tac x="d" in exI, simp) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
307 |
apply (rule_tac x="x" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
308 |
apply (rule_tac x="y" in exI) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
309 |
apply auto |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
310 |
done |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
311 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
312 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
313 |
text {* We can get a stronger version with a nonzeroness assumption. *} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
314 |
lemma divides_le: "m dvd n ==> m <= n \<or> n = (0::nat)" by (auto simp add: dvd_def) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
315 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
316 |
lemma bezout_add_strong: assumes nz: "a \<noteq> (0::nat)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
317 |
shows "\<exists>d x y. d dvd a \<and> d dvd b \<and> a * x = b * y + d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
318 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
319 |
from nz have ap: "a > 0" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
320 |
from bezout_add[of a b] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
321 |
have "(\<exists>d x y. d dvd a \<and> d dvd b \<and> a * x = b * y + d) \<or> (\<exists>d x y. d dvd a \<and> d dvd b \<and> b * x = a * y + d)" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
322 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
323 |
{fix d x y assume H: "d dvd a" "d dvd b" "a * x = b * y + d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
324 |
from H have ?thesis by blast } |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
325 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
326 |
{fix d x y assume H: "d dvd a" "d dvd b" "b * x = a * y + d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
327 |
{assume b0: "b = 0" with H have ?thesis by simp} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
328 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
329 |
{assume b: "b \<noteq> 0" hence bp: "b > 0" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
330 |
from divides_le[OF H(2)] b have "d < b \<or> d = b" using le_less by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
331 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
332 |
{assume db: "d=b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
333 |
from prems have ?thesis apply simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
334 |
apply (rule exI[where x = b], simp) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
335 |
apply (rule exI[where x = b]) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
336 |
by (rule exI[where x = "a - 1"], simp add: diff_mult_distrib2)} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
337 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
338 |
{assume db: "d < b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
339 |
{assume "x=0" hence ?thesis using prems by simp } |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
340 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
341 |
{assume x0: "x \<noteq> 0" hence xp: "x > 0" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
342 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
343 |
from db have "d \<le> b - 1" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
344 |
hence "d*b \<le> b*(b - 1)" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
345 |
with xp mult_mono[of "1" "x" "d*b" "b*(b - 1)"] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
346 |
have dble: "d*b \<le> x*b*(b - 1)" using bp by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
347 |
from H (3) have "a * ((b - 1) * y) + d * (b - 1 + 1) = d + x*b*(b - 1)" by algebra |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
348 |
hence "a * ((b - 1) * y) = d + x*b*(b - 1) - d*b" using bp by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
349 |
hence "a * ((b - 1) * y) = d + (x*b*(b - 1) - d*b)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
350 |
by (simp only: diff_add_assoc[OF dble, of d, symmetric]) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
351 |
hence "a * ((b - 1) * y) = b*(x*(b - 1) - d) + d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
352 |
by (simp only: diff_mult_distrib2 add_commute mult_ac) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
353 |
hence ?thesis using H(1,2) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
354 |
apply - |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
355 |
apply (rule exI[where x=d], simp) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
356 |
apply (rule exI[where x="(b - 1) * y"]) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
357 |
by (rule exI[where x="x*(b - 1) - d"], simp)} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
358 |
ultimately have ?thesis by blast} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
359 |
ultimately have ?thesis by blast} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
360 |
ultimately have ?thesis by blast} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
361 |
ultimately show ?thesis by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
362 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
363 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
364 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
365 |
lemma bezout_gcd: "\<exists>x y. a * x - b * y = gcd a b \<or> b * x - a * y = gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
366 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
367 |
let ?g = "gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
368 |
from bezout[of a b] obtain d x y where d: "d dvd a" "d dvd b" "a * x - b * y = d \<or> b * x - a * y = d" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
369 |
from d(1,2) have "d dvd ?g" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
370 |
then obtain k where k: "?g = d*k" unfolding dvd_def by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
371 |
from d(3) have "(a * x - b * y)*k = d*k \<or> (b * x - a * y)*k = d*k" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
372 |
hence "a * x * k - b * y*k = d*k \<or> b * x * k - a * y*k = d*k" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
373 |
by (algebra add: diff_mult_distrib) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
374 |
hence "a * (x * k) - b * (y*k) = ?g \<or> b * (x * k) - a * (y*k) = ?g" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
375 |
by (simp add: k mult_assoc) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
376 |
thus ?thesis by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
377 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
378 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
379 |
lemma bezout_gcd_strong: assumes a: "a \<noteq> 0" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
380 |
shows "\<exists>x y. a * x = b * y + gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
381 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
382 |
let ?g = "gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
383 |
from bezout_add_strong[OF a, of b] |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
384 |
obtain d x y where d: "d dvd a" "d dvd b" "a * x = b * y + d" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
385 |
from d(1,2) have "d dvd ?g" by simp |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
386 |
then obtain k where k: "?g = d*k" unfolding dvd_def by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
387 |
from d(3) have "a * x * k = (b * y + d) *k " by algebra |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
388 |
hence "a * (x * k) = b * (y*k) + ?g" by (algebra add: k) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
389 |
thus ?thesis by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
390 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
391 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
392 |
lemma gcd_mult_distrib: "gcd(a * c) (b * c) = c * gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
393 |
by(simp add: gcd_mult_distrib2 mult_commute) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
394 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
395 |
lemma gcd_bezout: "(\<exists>x y. a * x - b * y = d \<or> b * x - a * y = d) \<longleftrightarrow> gcd a b dvd d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
396 |
(is "?lhs \<longleftrightarrow> ?rhs") |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
397 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
398 |
let ?g = "gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
399 |
{assume H: ?rhs then obtain k where k: "d = ?g*k" unfolding dvd_def by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
400 |
from bezout_gcd[of a b] obtain x y where xy: "a * x - b * y = ?g \<or> b * x - a * y = ?g" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
401 |
by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
402 |
hence "(a * x - b * y)*k = ?g*k \<or> (b * x - a * y)*k = ?g*k" by auto |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
403 |
hence "a * x*k - b * y*k = ?g*k \<or> b * x * k - a * y*k = ?g*k" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
404 |
by (simp only: diff_mult_distrib) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
405 |
hence "a * (x*k) - b * (y*k) = d \<or> b * (x * k) - a * (y*k) = d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
406 |
by (simp add: k[symmetric] mult_assoc) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
407 |
hence ?lhs by blast} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
408 |
moreover |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
409 |
{fix x y assume H: "a * x - b * y = d \<or> b * x - a * y = d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
410 |
have dv: "?g dvd a*x" "?g dvd b * y" "?g dvd b*x" "?g dvd a * y" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
411 |
using dvd_mult2[OF gcd_dvd1[of a b]] dvd_mult2[OF gcd_dvd2[of a b]] by simp_all |
30042 | 412 |
from nat_dvd_diff[OF dv(1,2)] nat_dvd_diff[OF dv(3,4)] H |
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
413 |
have ?rhs by auto} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
414 |
ultimately show ?thesis by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
415 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
416 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
417 |
lemma gcd_bezout_sum: assumes H:"a * x + b * y = d" shows "gcd a b dvd d" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
418 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
419 |
let ?g = "gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
420 |
have dv: "?g dvd a*x" "?g dvd b * y" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
421 |
using dvd_mult2[OF gcd_dvd1[of a b]] dvd_mult2[OF gcd_dvd2[of a b]] by simp_all |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
422 |
from dvd_add[OF dv] H |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
423 |
show ?thesis by auto |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
424 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
425 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
426 |
lemma gcd_mult': "gcd b (a * b) = b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
427 |
by (simp add: gcd_mult mult_commute[of a b]) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
428 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
429 |
lemma gcd_add: "gcd(a + b) b = gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
430 |
"gcd(b + a) b = gcd a b" "gcd a (a + b) = gcd a b" "gcd a (b + a) = gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
431 |
apply (simp_all add: gcd_add1) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
432 |
by (simp add: gcd_commute gcd_add1) |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
433 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
434 |
lemma gcd_sub: "b <= a ==> gcd(a - b) b = gcd a b" "a <= b ==> gcd a (b - a) = gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
435 |
proof- |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
436 |
{fix a b assume H: "b \<le> (a::nat)" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
437 |
hence th: "a - b + b = a" by arith |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
438 |
from gcd_add(1)[of "a - b" b] th have "gcd(a - b) b = gcd a b" by simp} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
439 |
note th = this |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
440 |
{ |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
441 |
assume ab: "b \<le> a" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
442 |
from th[OF ab] show "gcd (a - b) b = gcd a b" by blast |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
443 |
next |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
444 |
assume ab: "a \<le> b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
445 |
from th[OF ab] show "gcd a (b - a) = gcd a b" |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
446 |
by (simp add: gcd_commute)} |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
447 |
qed |
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
448 |
|
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
449 |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
450 |
subsection {* LCM defined by GCD *} |
22367 | 451 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
452 |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
453 |
definition |
27556 | 454 |
lcm :: "nat \<Rightarrow> nat \<Rightarrow> nat" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
455 |
where |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
456 |
lcm_def: "lcm m n = m * n div gcd m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
457 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
458 |
lemma prod_gcd_lcm: |
27556 | 459 |
"m * n = gcd m n * lcm m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
460 |
unfolding lcm_def by (simp add: dvd_mult_div_cancel [OF gcd_dvd_prod]) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
461 |
|
27556 | 462 |
lemma lcm_0 [simp]: "lcm m 0 = 0" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
463 |
unfolding lcm_def by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
464 |
|
27556 | 465 |
lemma lcm_1 [simp]: "lcm m 1 = m" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
466 |
unfolding lcm_def by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
467 |
|
27556 | 468 |
lemma lcm_0_left [simp]: "lcm 0 n = 0" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
469 |
unfolding lcm_def by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
470 |
|
27556 | 471 |
lemma lcm_1_left [simp]: "lcm 1 m = m" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
472 |
unfolding lcm_def by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
473 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
474 |
lemma dvd_pos: |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
475 |
fixes n m :: nat |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
476 |
assumes "n > 0" and "m dvd n" |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
477 |
shows "m > 0" |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
478 |
using assms by (cases m) auto |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
479 |
|
23951 | 480 |
lemma lcm_least: |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
481 |
assumes "m dvd k" and "n dvd k" |
27556 | 482 |
shows "lcm m n dvd k" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
483 |
proof (cases k) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
484 |
case 0 then show ?thesis by auto |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
485 |
next |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
486 |
case (Suc _) then have pos_k: "k > 0" by auto |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
487 |
from assms dvd_pos [OF this] have pos_mn: "m > 0" "n > 0" by auto |
27556 | 488 |
with gcd_zero [of m n] have pos_gcd: "gcd m n > 0" by simp |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
489 |
from assms obtain p where k_m: "k = m * p" using dvd_def by blast |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
490 |
from assms obtain q where k_n: "k = n * q" using dvd_def by blast |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
491 |
from pos_k k_m have pos_p: "p > 0" by auto |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
492 |
from pos_k k_n have pos_q: "q > 0" by auto |
27556 | 493 |
have "k * k * gcd q p = k * gcd (k * q) (k * p)" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
494 |
by (simp add: mult_ac gcd_mult_distrib2) |
27556 | 495 |
also have "\<dots> = k * gcd (m * p * q) (n * q * p)" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
496 |
by (simp add: k_m [symmetric] k_n [symmetric]) |
27556 | 497 |
also have "\<dots> = k * p * q * gcd m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
498 |
by (simp add: mult_ac gcd_mult_distrib2) |
27556 | 499 |
finally have "(m * p) * (n * q) * gcd q p = k * p * q * gcd m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
500 |
by (simp only: k_m [symmetric] k_n [symmetric]) |
27556 | 501 |
then have "p * q * m * n * gcd q p = p * q * k * gcd m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
502 |
by (simp add: mult_ac) |
27556 | 503 |
with pos_p pos_q have "m * n * gcd q p = k * gcd m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
504 |
by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
505 |
with prod_gcd_lcm [of m n] |
27556 | 506 |
have "lcm m n * gcd q p * gcd m n = k * gcd m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
507 |
by (simp add: mult_ac) |
27556 | 508 |
with pos_gcd have "lcm m n * gcd q p = k" by simp |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
509 |
then show ?thesis using dvd_def by auto |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
510 |
qed |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
511 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
512 |
lemma lcm_dvd1 [iff]: |
27556 | 513 |
"m dvd lcm m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
514 |
proof (cases m) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
515 |
case 0 then show ?thesis by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
516 |
next |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
517 |
case (Suc _) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
518 |
then have mpos: "m > 0" by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
519 |
show ?thesis |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
520 |
proof (cases n) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
521 |
case 0 then show ?thesis by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
522 |
next |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
523 |
case (Suc _) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
524 |
then have npos: "n > 0" by simp |
27556 | 525 |
have "gcd m n dvd n" by simp |
526 |
then obtain k where "n = gcd m n * k" using dvd_def by auto |
|
527 |
then have "m * n div gcd m n = m * (gcd m n * k) div gcd m n" by (simp add: mult_ac) |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
528 |
also have "\<dots> = m * k" using mpos npos gcd_zero by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
529 |
finally show ?thesis by (simp add: lcm_def) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
530 |
qed |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
531 |
qed |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
532 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
533 |
lemma lcm_dvd2 [iff]: |
27556 | 534 |
"n dvd lcm m n" |
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
535 |
proof (cases n) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
536 |
case 0 then show ?thesis by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
537 |
next |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
538 |
case (Suc _) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
539 |
then have npos: "n > 0" by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
540 |
show ?thesis |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
541 |
proof (cases m) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
542 |
case 0 then show ?thesis by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
543 |
next |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
544 |
case (Suc _) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
545 |
then have mpos: "m > 0" by simp |
27556 | 546 |
have "gcd m n dvd m" by simp |
547 |
then obtain k where "m = gcd m n * k" using dvd_def by auto |
|
548 |
then have "m * n div gcd m n = (gcd m n * k) * n div gcd m n" by (simp add: mult_ac) |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
549 |
also have "\<dots> = n * k" using mpos npos gcd_zero by simp |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
550 |
finally show ?thesis by (simp add: lcm_def) |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
551 |
qed |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
552 |
qed |
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
553 |
|
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
554 |
lemma gcd_add1_eq: "gcd (m + k) k = gcd (m + k) m" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
555 |
by (simp add: gcd_commute) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
556 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
557 |
lemma gcd_diff2: "m \<le> n ==> gcd n (n - m) = gcd n m" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
558 |
apply (subgoal_tac "n = m + (n - m)") |
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
559 |
apply (erule ssubst, rule gcd_add1_eq, simp) |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
560 |
done |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
561 |
|
23687
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
562 |
|
06884f7ffb18
extended - convers now basic lcm properties also
haftmann
parents:
23431
diff
changeset
|
563 |
subsection {* GCD and LCM on integers *} |
22367 | 564 |
|
565 |
definition |
|
27556 | 566 |
zgcd :: "int \<Rightarrow> int \<Rightarrow> int" where |
567 |
"zgcd i j = int (gcd (nat (abs i)) (nat (abs j)))" |
|
22367 | 568 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
569 |
lemma zgcd_zdvd1 [iff,simp, algebra]: "zgcd i j dvd i" |
29700 | 570 |
by (simp add: zgcd_def int_dvd_iff) |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
571 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
572 |
lemma zgcd_zdvd2 [iff,simp, algebra]: "zgcd i j dvd j" |
29700 | 573 |
by (simp add: zgcd_def int_dvd_iff) |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
574 |
|
27556 | 575 |
lemma zgcd_pos: "zgcd i j \<ge> 0" |
29700 | 576 |
by (simp add: zgcd_def) |
22367 | 577 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
578 |
lemma zgcd0 [simp,algebra]: "(zgcd i j = 0) = (i = 0 \<and> j = 0)" |
29700 | 579 |
by (simp add: zgcd_def gcd_zero) |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
580 |
|
27556 | 581 |
lemma zgcd_commute: "zgcd i j = zgcd j i" |
29700 | 582 |
unfolding zgcd_def by (simp add: gcd_commute) |
22367 | 583 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
584 |
lemma zgcd_zminus [simp, algebra]: "zgcd (- i) j = zgcd i j" |
29700 | 585 |
unfolding zgcd_def by simp |
22367 | 586 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
587 |
lemma zgcd_zminus2 [simp, algebra]: "zgcd i (- j) = zgcd i j" |
29700 | 588 |
unfolding zgcd_def by simp |
22367 | 589 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
590 |
(* should be solved by algebra*) |
27556 | 591 |
lemma zrelprime_dvd_mult: "zgcd i j = 1 \<Longrightarrow> i dvd k * j \<Longrightarrow> i dvd k" |
592 |
unfolding zgcd_def |
|
22367 | 593 |
proof - |
27556 | 594 |
assume "int (gcd (nat \<bar>i\<bar>) (nat \<bar>j\<bar>)) = 1" "i dvd k * j" |
595 |
then have g: "gcd (nat \<bar>i\<bar>) (nat \<bar>j\<bar>) = 1" by simp |
|
22367 | 596 |
from `i dvd k * j` obtain h where h: "k*j = i*h" unfolding dvd_def by blast |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
597 |
have th: "nat \<bar>i\<bar> dvd nat \<bar>k\<bar> * nat \<bar>j\<bar>" |
22367 | 598 |
unfolding dvd_def |
599 |
by (rule_tac x= "nat \<bar>h\<bar>" in exI, simp add: h nat_abs_mult_distrib [symmetric]) |
|
600 |
from relprime_dvd_mult [OF g th] obtain h' where h': "nat \<bar>k\<bar> = nat \<bar>i\<bar> * h'" |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
601 |
unfolding dvd_def by blast |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
602 |
from h' have "int (nat \<bar>k\<bar>) = int (nat \<bar>i\<bar> * h')" by simp |
23431
25ca91279a9b
change simp rules for of_nat to work like int did previously (reorient of_nat_Suc, remove of_nat_mult [simp]); preserve original variable names in legacy int theorems
huffman
parents:
23365
diff
changeset
|
603 |
then have "\<bar>k\<bar> = \<bar>i\<bar> * int h'" by (simp add: int_mult) |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
604 |
then show ?thesis |
30042 | 605 |
apply (subst abs_dvd_iff [symmetric]) |
606 |
apply (subst dvd_abs_iff [symmetric]) |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
607 |
apply (unfold dvd_def) |
22367 | 608 |
apply (rule_tac x = "int h'" in exI, simp) |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
609 |
done |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
610 |
qed |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
611 |
|
27556 | 612 |
lemma int_nat_abs: "int (nat (abs x)) = abs x" by arith |
22367 | 613 |
|
27556 | 614 |
lemma zgcd_greatest: |
22367 | 615 |
assumes "k dvd m" and "k dvd n" |
27556 | 616 |
shows "k dvd zgcd m n" |
22367 | 617 |
proof - |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
618 |
let ?k' = "nat \<bar>k\<bar>" |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
619 |
let ?m' = "nat \<bar>m\<bar>" |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
620 |
let ?n' = "nat \<bar>n\<bar>" |
22367 | 621 |
from `k dvd m` and `k dvd n` have dvd': "?k' dvd ?m'" "?k' dvd ?n'" |
30042 | 622 |
unfolding zdvd_int by (simp_all only: int_nat_abs abs_dvd_iff dvd_abs_iff) |
27556 | 623 |
from gcd_greatest [OF dvd'] have "int (nat \<bar>k\<bar>) dvd zgcd m n" |
624 |
unfolding zgcd_def by (simp only: zdvd_int) |
|
625 |
then have "\<bar>k\<bar> dvd zgcd m n" by (simp only: int_nat_abs) |
|
30042 | 626 |
then show "k dvd zgcd m n" by simp |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
627 |
qed |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
628 |
|
27556 | 629 |
lemma div_zgcd_relprime: |
22367 | 630 |
assumes nz: "a \<noteq> 0 \<or> b \<noteq> 0" |
27556 | 631 |
shows "zgcd (a div (zgcd a b)) (b div (zgcd a b)) = 1" |
22367 | 632 |
proof - |
25112 | 633 |
from nz have nz': "nat \<bar>a\<bar> \<noteq> 0 \<or> nat \<bar>b\<bar> \<noteq> 0" by arith |
27556 | 634 |
let ?g = "zgcd a b" |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
635 |
let ?a' = "a div ?g" |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
636 |
let ?b' = "b div ?g" |
27556 | 637 |
let ?g' = "zgcd ?a' ?b'" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
638 |
have dvdg: "?g dvd a" "?g dvd b" by (simp_all add: zgcd_zdvd1 zgcd_zdvd2) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
639 |
have dvdg': "?g' dvd ?a'" "?g' dvd ?b'" by (simp_all add: zgcd_zdvd1 zgcd_zdvd2) |
22367 | 640 |
from dvdg dvdg' obtain ka kb ka' kb' where |
641 |
kab: "a = ?g*ka" "b = ?g*kb" "?a' = ?g'*ka'" "?b' = ?g' * kb'" |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
642 |
unfolding dvd_def by blast |
22367 | 643 |
then have "?g* ?a' = (?g * ?g') * ka'" "?g* ?b' = (?g * ?g') * kb'" by simp_all |
644 |
then have dvdgg':"?g * ?g' dvd a" "?g* ?g' dvd b" |
|
645 |
by (auto simp add: zdvd_mult_div_cancel [OF dvdg(1)] |
|
646 |
zdvd_mult_div_cancel [OF dvdg(2)] dvd_def) |
|
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
647 |
have "?g \<noteq> 0" using nz by simp |
27556 | 648 |
then have gp: "?g \<noteq> 0" using zgcd_pos[where i="a" and j="b"] by arith |
649 |
from zgcd_greatest [OF dvdgg'] have "?g * ?g' dvd ?g" . |
|
22367 | 650 |
with zdvd_mult_cancel1 [OF gp] have "\<bar>?g'\<bar> = 1" by simp |
27556 | 651 |
with zgcd_pos show "?g' = 1" by simp |
22027
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
652 |
qed |
e4a08629c4bd
A few lemmas about relative primes when dividing trough gcd
chaieb
parents:
21404
diff
changeset
|
653 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
654 |
lemma zgcd_0 [simp, algebra]: "zgcd m 0 = abs m" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
655 |
by (simp add: zgcd_def abs_if) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
656 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
657 |
lemma zgcd_0_left [simp, algebra]: "zgcd 0 m = abs m" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
658 |
by (simp add: zgcd_def abs_if) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
659 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
660 |
lemma zgcd_non_0: "0 < n ==> zgcd m n = zgcd n (m mod n)" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
661 |
apply (frule_tac b = n and a = m in pos_mod_sign) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
662 |
apply (simp del: pos_mod_sign add: zgcd_def abs_if nat_mod_distrib) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
663 |
apply (auto simp add: gcd_non_0 nat_mod_distrib [symmetric] zmod_zminus1_eq_if) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
664 |
apply (frule_tac a = m in pos_mod_bound) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
665 |
apply (simp del: pos_mod_bound add: nat_diff_distrib gcd_diff2 nat_le_eq_zle) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
666 |
done |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
667 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
668 |
lemma zgcd_eq: "zgcd m n = zgcd n (m mod n)" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
669 |
apply (case_tac "n = 0", simp add: DIVISION_BY_ZERO) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
670 |
apply (auto simp add: linorder_neq_iff zgcd_non_0) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
671 |
apply (cut_tac m = "-m" and n = "-n" in zgcd_non_0, auto) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
672 |
done |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
673 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
674 |
lemma zgcd_1 [simp, algebra]: "zgcd m 1 = 1" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
675 |
by (simp add: zgcd_def abs_if) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
676 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
677 |
lemma zgcd_0_1_iff [simp, algebra]: "zgcd 0 m = 1 \<longleftrightarrow> \<bar>m\<bar> = 1" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
678 |
by (simp add: zgcd_def abs_if) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
679 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
680 |
lemma zgcd_greatest_iff[algebra]: "k dvd zgcd m n = (k dvd m \<and> k dvd n)" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
681 |
by (simp add: zgcd_def abs_if int_dvd_iff dvd_int_iff nat_dvd_iff) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
682 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
683 |
lemma zgcd_1_left [simp, algebra]: "zgcd 1 m = 1" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
684 |
by (simp add: zgcd_def gcd_1_left) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
685 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
686 |
lemma zgcd_assoc: "zgcd (zgcd k m) n = zgcd k (zgcd m n)" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
687 |
by (simp add: zgcd_def gcd_assoc) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
688 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
689 |
lemma zgcd_left_commute: "zgcd k (zgcd m n) = zgcd m (zgcd k n)" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
690 |
apply (rule zgcd_commute [THEN trans]) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
691 |
apply (rule zgcd_assoc [THEN trans]) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
692 |
apply (rule zgcd_commute [THEN arg_cong]) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
693 |
done |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
694 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
695 |
lemmas zgcd_ac = zgcd_assoc zgcd_commute zgcd_left_commute |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
696 |
-- {* addition is an AC-operator *} |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
697 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
698 |
lemma zgcd_zmult_distrib2: "0 \<le> k ==> k * zgcd m n = zgcd (k * m) (k * n)" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
699 |
by (simp del: minus_mult_right [symmetric] |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
700 |
add: minus_mult_right nat_mult_distrib zgcd_def abs_if |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
701 |
mult_less_0_iff gcd_mult_distrib2 [symmetric] zmult_int [symmetric]) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
702 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
703 |
lemma zgcd_zmult_distrib2_abs: "zgcd (k * m) (k * n) = abs k * zgcd m n" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
704 |
by (simp add: abs_if zgcd_zmult_distrib2) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
705 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
706 |
lemma zgcd_self [simp]: "0 \<le> m ==> zgcd m m = m" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
707 |
by (cut_tac k = m and m = 1 and n = 1 in zgcd_zmult_distrib2, simp_all) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
708 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
709 |
lemma zgcd_zmult_eq_self [simp]: "0 \<le> k ==> zgcd k (k * n) = k" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
710 |
by (cut_tac k = k and m = 1 and n = n in zgcd_zmult_distrib2, simp_all) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
711 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
712 |
lemma zgcd_zmult_eq_self2 [simp]: "0 \<le> k ==> zgcd (k * n) k = k" |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
713 |
by (cut_tac k = k and m = n and n = 1 in zgcd_zmult_distrib2, simp_all) |
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
714 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
715 |
|
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
716 |
definition "zlcm i j = int (lcm(nat(abs i)) (nat(abs j)))" |
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
717 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
718 |
lemma dvd_zlcm_self1[simp, algebra]: "i dvd zlcm i j" |
27556 | 719 |
by(simp add:zlcm_def dvd_int_iff) |
23983 | 720 |
|
27669
4b1642284dd7
Tuned and simplified proofs; Rules added to presburger's and algebra's context; moved Bezout theorems from Primes.thy
chaieb
parents:
27651
diff
changeset
|
721 |
lemma dvd_zlcm_self2[simp, algebra]: "j dvd zlcm i j" |
27556 | 722 |
by(simp add:zlcm_def dvd_int_iff) |
23983 | 723 |
|
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
724 |
|
27556 | 725 |
lemma dvd_imp_dvd_zlcm1: |
726 |
assumes "k dvd i" shows "k dvd (zlcm i j)" |
|
23983 | 727 |
proof - |
728 |
have "nat(abs k) dvd nat(abs i)" using `k dvd i` |
|
30042 | 729 |
by(simp add:int_dvd_iff[symmetric] dvd_int_iff[symmetric]) |
27556 | 730 |
thus ?thesis by(simp add:zlcm_def dvd_int_iff)(blast intro: dvd_trans) |
23983 | 731 |
qed |
732 |
||
27556 | 733 |
lemma dvd_imp_dvd_zlcm2: |
734 |
assumes "k dvd j" shows "k dvd (zlcm i j)" |
|
23983 | 735 |
proof - |
736 |
have "nat(abs k) dvd nat(abs j)" using `k dvd j` |
|
30042 | 737 |
by(simp add:int_dvd_iff[symmetric] dvd_int_iff[symmetric]) |
27556 | 738 |
thus ?thesis by(simp add:zlcm_def dvd_int_iff)(blast intro: dvd_trans) |
23983 | 739 |
qed |
740 |
||
23994 | 741 |
|
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
742 |
lemma zdvd_self_abs1: "(d::int) dvd (abs d)" |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
743 |
by (case_tac "d <0", simp_all) |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
744 |
|
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
745 |
lemma zdvd_self_abs2: "(abs (d::int)) dvd d" |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
746 |
by (case_tac "d<0", simp_all) |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
747 |
|
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
748 |
(* lcm a b is positive for positive a and b *) |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
749 |
|
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
750 |
lemma lcm_pos: |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
751 |
assumes mpos: "m > 0" |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
752 |
and npos: "n>0" |
27556 | 753 |
shows "lcm m n > 0" |
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
754 |
proof(rule ccontr, simp add: lcm_def gcd_zero) |
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
755 |
assume h:"m*n div gcd m n = 0" |
27556 | 756 |
from mpos npos have "gcd m n \<noteq> 0" using gcd_zero by simp |
757 |
hence gcdp: "gcd m n > 0" by simp |
|
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
758 |
with h |
27556 | 759 |
have "m*n < gcd m n" |
760 |
by (cases "m * n < gcd m n") (auto simp add: div_if[OF gcdp, where m="m*n"]) |
|
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
761 |
moreover |
27556 | 762 |
have "gcd m n dvd m" by simp |
763 |
with mpos dvd_imp_le have t1:"gcd m n \<le> m" by simp |
|
27568
9949dc7a24de
Theorem names as in IntPrimes.thy, also several theorems moved from there
chaieb
parents:
27556
diff
changeset
|
764 |
with npos have t1:"gcd m n *n \<le> m*n" by simp |
27556 | 765 |
have "gcd m n \<le> gcd m n*n" using npos by simp |
766 |
with t1 have "gcd m n \<le> m*n" by arith |
|
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
767 |
ultimately show "False" by simp |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
768 |
qed |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
769 |
|
27556 | 770 |
lemma zlcm_pos: |
23983 | 771 |
assumes anz: "a \<noteq> 0" |
772 |
and bnz: "b \<noteq> 0" |
|
27556 | 773 |
shows "0 < zlcm a b" |
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
774 |
proof- |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
775 |
let ?na = "nat (abs a)" |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
776 |
let ?nb = "nat (abs b)" |
23983 | 777 |
have nap: "?na >0" using anz by simp |
778 |
have nbp: "?nb >0" using bnz by simp |
|
27556 | 779 |
have "0 < lcm ?na ?nb" by (rule lcm_pos[OF nap nbp]) |
780 |
thus ?thesis by (simp add: zlcm_def) |
|
23244
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
781 |
qed |
1630951f0512
added lcm, ilcm (lcm for integers) and some lemmas about them;
chaieb
parents:
22367
diff
changeset
|
782 |
|
28562 | 783 |
lemma zgcd_code [code]: |
27651
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
haftmann
parents:
27568
diff
changeset
|
784 |
"zgcd k l = \<bar>if l = 0 then k else zgcd l (\<bar>k\<bar> mod \<bar>l\<bar>)\<bar>" |
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
haftmann
parents:
27568
diff
changeset
|
785 |
by (simp add: zgcd_def gcd.simps [of "nat \<bar>k\<bar>"] nat_mod_distrib) |
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
haftmann
parents:
27568
diff
changeset
|
786 |
|
21256 | 787 |
end |