| author | smolkas | 
| Thu, 14 Feb 2013 22:49:22 +0100 | |
| changeset 51129 | 1edc2cc25f19 | 
| parent 50422 | ee729dbd1b7f | 
| child 51173 | 3cbb4e95a565 | 
| permissions | -rw-r--r-- | 
| 3366 | 1 | (* Title: HOL/Divides.thy | 
| 2 | Author: Lawrence C Paulson, Cambridge University Computer Laboratory | |
| 6865 
5577ffe4c2f1
now div and mod are overloaded; dvd is polymorphic
 paulson parents: 
3366diff
changeset | 3 | Copyright 1999 University of Cambridge | 
| 18154 | 4 | *) | 
| 3366 | 5 | |
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 6 | header {* The division operators div and mod *}
 | 
| 3366 | 7 | |
| 15131 | 8 | theory Divides | 
| 47255 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 huffman parents: 
47217diff
changeset | 9 | imports Nat_Transfer | 
| 15131 | 10 | begin | 
| 3366 | 11 | |
| 25942 | 12 | subsection {* Syntactic division operations *}
 | 
| 13 | ||
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 14 | class div = dvd + | 
| 27540 | 15 | fixes div :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixl "div" 70) | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 16 | and mod :: "'a \<Rightarrow> 'a \<Rightarrow> 'a" (infixl "mod" 70) | 
| 27540 | 17 | |
| 18 | ||
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 19 | subsection {* Abstract division in commutative semirings. *}
 | 
| 25942 | 20 | |
| 30930 | 21 | class semiring_div = comm_semiring_1_cancel + no_zero_divisors + div + | 
| 25942 | 22 | assumes mod_div_equality: "a div b * b + a mod b = a" | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 23 | and div_by_0 [simp]: "a div 0 = 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 24 | and div_0 [simp]: "0 div a = 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 25 | and div_mult_self1 [simp]: "b \<noteq> 0 \<Longrightarrow> (a + c * b) div b = c + a div b" | 
| 30930 | 26 | and div_mult_mult1 [simp]: "c \<noteq> 0 \<Longrightarrow> (c * a) div (c * b) = a div b" | 
| 25942 | 27 | begin | 
| 28 | ||
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 29 | text {* @{const div} and @{const mod} *}
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 30 | |
| 26062 | 31 | lemma mod_div_equality2: "b * (a div b) + a mod b = a" | 
| 32 | unfolding mult_commute [of b] | |
| 33 | by (rule mod_div_equality) | |
| 34 | ||
| 29403 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 35 | lemma mod_div_equality': "a mod b + a div b * b = a" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 36 | using mod_div_equality [of a b] | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 37 | by (simp only: add_ac) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 38 | |
| 26062 | 39 | lemma div_mod_equality: "((a div b) * b + a mod b) + c = a + c" | 
| 30934 | 40 | by (simp add: mod_div_equality) | 
| 26062 | 41 | |
| 42 | lemma div_mod_equality2: "(b * (a div b) + a mod b) + c = a + c" | |
| 30934 | 43 | by (simp add: mod_div_equality2) | 
| 26062 | 44 | |
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 45 | lemma mod_by_0 [simp]: "a mod 0 = a" | 
| 30934 | 46 | using mod_div_equality [of a zero] by simp | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 47 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 48 | lemma mod_0 [simp]: "0 mod a = 0" | 
| 30934 | 49 | using mod_div_equality [of zero a] div_0 by simp | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 50 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 51 | lemma div_mult_self2 [simp]: | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 52 | assumes "b \<noteq> 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 53 | shows "(a + b * c) div b = c + a div b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 54 | using assms div_mult_self1 [of b a c] by (simp add: mult_commute) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 55 | |
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 56 | lemma mod_mult_self1 [simp]: "(a + c * b) mod b = a mod b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 57 | proof (cases "b = 0") | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 58 | case True then show ?thesis by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 59 | next | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 60 | case False | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 61 | have "a + c * b = (a + c * b) div b * b + (a + c * b) mod b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 62 | by (simp add: mod_div_equality) | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 63 | also from False div_mult_self1 [of b a c] have | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 64 | "\<dots> = (c + a div b) * b + (a + c * b) mod b" | 
| 29667 | 65 | by (simp add: algebra_simps) | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 66 | finally have "a = a div b * b + (a + c * b) mod b" | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 67 | by (simp add: add_commute [of a] add_assoc distrib_right) | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 68 | then have "a div b * b + (a + c * b) mod b = a div b * b + a mod b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 69 | by (simp add: mod_div_equality) | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 70 | then show ?thesis by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 71 | qed | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 72 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 73 | lemma mod_mult_self2 [simp]: "(a + b * c) mod b = a mod b" | 
| 30934 | 74 | by (simp add: mult_commute [of b]) | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 75 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 76 | lemma div_mult_self1_is_id [simp]: "b \<noteq> 0 \<Longrightarrow> b * a div b = a" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 77 | using div_mult_self2 [of b 0 a] by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 78 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 79 | lemma div_mult_self2_is_id [simp]: "b \<noteq> 0 \<Longrightarrow> a * b div b = a" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 80 | using div_mult_self1 [of b 0 a] by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 81 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 82 | lemma mod_mult_self1_is_0 [simp]: "b * a mod b = 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 83 | using mod_mult_self2 [of 0 b a] by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 84 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 85 | lemma mod_mult_self2_is_0 [simp]: "a * b mod b = 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 86 | using mod_mult_self1 [of 0 a b] by simp | 
| 26062 | 87 | |
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 88 | lemma div_by_1 [simp]: "a div 1 = a" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 89 | using div_mult_self2_is_id [of 1 a] zero_neq_one by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 90 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 91 | lemma mod_by_1 [simp]: "a mod 1 = 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 92 | proof - | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 93 | from mod_div_equality [of a one] div_by_1 have "a + a mod 1 = a" by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 94 | then have "a + a mod 1 = a + 0" by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 95 | then show ?thesis by (rule add_left_imp_eq) | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 96 | qed | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 97 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 98 | lemma mod_self [simp]: "a mod a = 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 99 | using mod_mult_self2_is_0 [of 1] by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 100 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 101 | lemma div_self [simp]: "a \<noteq> 0 \<Longrightarrow> a div a = 1" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 102 | using div_mult_self2_is_id [of _ 1] by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 103 | |
| 27676 | 104 | lemma div_add_self1 [simp]: | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 105 | assumes "b \<noteq> 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 106 | shows "(b + a) div b = a div b + 1" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 107 | using assms div_mult_self1 [of b a 1] by (simp add: add_commute) | 
| 26062 | 108 | |
| 27676 | 109 | lemma div_add_self2 [simp]: | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 110 | assumes "b \<noteq> 0" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 111 | shows "(a + b) div b = a div b + 1" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 112 | using assms div_add_self1 [of b a] by (simp add: add_commute) | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 113 | |
| 27676 | 114 | lemma mod_add_self1 [simp]: | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 115 | "(b + a) mod b = a mod b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 116 | using mod_mult_self1 [of a 1 b] by (simp add: add_commute) | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 117 | |
| 27676 | 118 | lemma mod_add_self2 [simp]: | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 119 | "(a + b) mod b = a mod b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 120 | using mod_mult_self1 [of a 1 b] by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 121 | |
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 122 | lemma mod_div_decomp: | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 123 | fixes a b | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 124 | obtains q r where "q = a div b" and "r = a mod b" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 125 | and "a = q * b + r" | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 126 | proof - | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 127 | from mod_div_equality have "a = a div b * b + a mod b" by simp | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 128 | moreover have "a div b = a div b" .. | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 129 | moreover have "a mod b = a mod b" .. | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 130 | note that ultimately show thesis by blast | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 131 | qed | 
| 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 132 | |
| 45231 
d85a2fdc586c
replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed
 bulwahn parents: 
44890diff
changeset | 133 | lemma dvd_eq_mod_eq_0 [code]: "a dvd b \<longleftrightarrow> b mod a = 0" | 
| 25942 | 134 | proof | 
| 135 | assume "b mod a = 0" | |
| 136 | with mod_div_equality [of b a] have "b div a * a = b" by simp | |
| 137 | then have "b = a * (b div a)" unfolding mult_commute .. | |
| 138 | then have "\<exists>c. b = a * c" .. | |
| 139 | then show "a dvd b" unfolding dvd_def . | |
| 140 | next | |
| 141 | assume "a dvd b" | |
| 142 | then have "\<exists>c. b = a * c" unfolding dvd_def . | |
| 143 | then obtain c where "b = a * c" .. | |
| 144 | then have "b mod a = a * c mod a" by simp | |
| 145 | then have "b mod a = c * a mod a" by (simp add: mult_commute) | |
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 146 | then show "b mod a = 0" by simp | 
| 25942 | 147 | qed | 
| 148 | ||
| 29403 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 149 | lemma mod_div_trivial [simp]: "a mod b div b = 0" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 150 | proof (cases "b = 0") | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 151 | assume "b = 0" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 152 | thus ?thesis by simp | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 153 | next | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 154 | assume "b \<noteq> 0" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 155 | hence "a div b + a mod b div b = (a mod b + a div b * b) div b" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 156 | by (rule div_mult_self1 [symmetric]) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 157 | also have "\<dots> = a div b" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 158 | by (simp only: mod_div_equality') | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 159 | also have "\<dots> = a div b + 0" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 160 | by simp | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 161 | finally show ?thesis | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 162 | by (rule add_left_imp_eq) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 163 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 164 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 165 | lemma mod_mod_trivial [simp]: "a mod b mod b = a mod b" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 166 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 167 | have "a mod b mod b = (a mod b + a div b * b) mod b" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 168 | by (simp only: mod_mult_self1) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 169 | also have "\<dots> = a mod b" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 170 | by (simp only: mod_div_equality') | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 171 | finally show ?thesis . | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 172 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 173 | |
| 29925 | 174 | lemma dvd_imp_mod_0: "a dvd b \<Longrightarrow> b mod a = 0" | 
| 29948 | 175 | by (rule dvd_eq_mod_eq_0[THEN iffD1]) | 
| 29925 | 176 | |
| 177 | lemma dvd_div_mult_self: "a dvd b \<Longrightarrow> (b div a) * a = b" | |
| 178 | by (subst (2) mod_div_equality [of b a, symmetric]) (simp add:dvd_imp_mod_0) | |
| 179 | ||
| 33274 
b6ff7db522b5
moved lemmas for dvd on nat to theories Nat and Power
 haftmann parents: 
32010diff
changeset | 180 | lemma dvd_mult_div_cancel: "a dvd b \<Longrightarrow> a * (b div a) = b" | 
| 
b6ff7db522b5
moved lemmas for dvd on nat to theories Nat and Power
 haftmann parents: 
32010diff
changeset | 181 | by (drule dvd_div_mult_self) (simp add: mult_commute) | 
| 
b6ff7db522b5
moved lemmas for dvd on nat to theories Nat and Power
 haftmann parents: 
32010diff
changeset | 182 | |
| 30052 | 183 | lemma dvd_div_mult: "a dvd b \<Longrightarrow> (b div a) * c = b * c div a" | 
| 184 | apply (cases "a = 0") | |
| 185 | apply simp | |
| 186 | apply (auto simp: dvd_def mult_assoc) | |
| 187 | done | |
| 188 | ||
| 29925 | 189 | lemma div_dvd_div[simp]: | 
| 190 | "a dvd b \<Longrightarrow> a dvd c \<Longrightarrow> (b div a dvd c div a) = (b dvd c)" | |
| 191 | apply (cases "a = 0") | |
| 192 | apply simp | |
| 193 | apply (unfold dvd_def) | |
| 194 | apply auto | |
| 195 | apply(blast intro:mult_assoc[symmetric]) | |
| 44890 
22f665a2e91c
new fastforce replacing fastsimp - less confusing name
 nipkow parents: 
44766diff
changeset | 196 | apply(fastforce simp add: mult_assoc) | 
| 29925 | 197 | done | 
| 198 | ||
| 30078 
beee83623cc9
move lemma dvd_mod_imp_dvd into class semiring_div
 huffman parents: 
30052diff
changeset | 199 | lemma dvd_mod_imp_dvd: "[| k dvd m mod n; k dvd n |] ==> k dvd m" | 
| 
beee83623cc9
move lemma dvd_mod_imp_dvd into class semiring_div
 huffman parents: 
30052diff
changeset | 200 | apply (subgoal_tac "k dvd (m div n) *n + m mod n") | 
| 
beee83623cc9
move lemma dvd_mod_imp_dvd into class semiring_div
 huffman parents: 
30052diff
changeset | 201 | apply (simp add: mod_div_equality) | 
| 
beee83623cc9
move lemma dvd_mod_imp_dvd into class semiring_div
 huffman parents: 
30052diff
changeset | 202 | apply (simp only: dvd_add dvd_mult) | 
| 
beee83623cc9
move lemma dvd_mod_imp_dvd into class semiring_div
 huffman parents: 
30052diff
changeset | 203 | done | 
| 
beee83623cc9
move lemma dvd_mod_imp_dvd into class semiring_div
 huffman parents: 
30052diff
changeset | 204 | |
| 29403 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 205 | text {* Addition respects modular equivalence. *}
 | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 206 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 207 | lemma mod_add_left_eq: "(a + b) mod c = (a mod c + b) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 208 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 209 | have "(a + b) mod c = (a div c * c + a mod c + b) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 210 | by (simp only: mod_div_equality) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 211 | also have "\<dots> = (a mod c + b + a div c * c) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 212 | by (simp only: add_ac) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 213 | also have "\<dots> = (a mod c + b) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 214 | by (rule mod_mult_self1) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 215 | finally show ?thesis . | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 216 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 217 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 218 | lemma mod_add_right_eq: "(a + b) mod c = (a + b mod c) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 219 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 220 | have "(a + b) mod c = (a + (b div c * c + b mod c)) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 221 | by (simp only: mod_div_equality) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 222 | also have "\<dots> = (a + b mod c + b div c * c) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 223 | by (simp only: add_ac) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 224 | also have "\<dots> = (a + b mod c) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 225 | by (rule mod_mult_self1) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 226 | finally show ?thesis . | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 227 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 228 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 229 | lemma mod_add_eq: "(a + b) mod c = (a mod c + b mod c) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 230 | by (rule trans [OF mod_add_left_eq mod_add_right_eq]) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 231 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 232 | lemma mod_add_cong: | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 233 | assumes "a mod c = a' mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 234 | assumes "b mod c = b' mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 235 | shows "(a + b) mod c = (a' + b') mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 236 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 237 | have "(a mod c + b mod c) mod c = (a' mod c + b' mod c) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 238 | unfolding assms .. | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 239 | thus ?thesis | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 240 | by (simp only: mod_add_eq [symmetric]) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 241 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 242 | |
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 243 | lemma div_add [simp]: "z dvd x \<Longrightarrow> z dvd y | 
| 30837 
3d4832d9f7e4
added strong_setprod_cong[cong] (in analogy with setsum)
 nipkow parents: 
30729diff
changeset | 244 | \<Longrightarrow> (x + y) div z = x div z + y div z" | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 245 | by (cases "z = 0", simp, unfold dvd_def, auto simp add: algebra_simps) | 
| 30837 
3d4832d9f7e4
added strong_setprod_cong[cong] (in analogy with setsum)
 nipkow parents: 
30729diff
changeset | 246 | |
| 29403 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 247 | text {* Multiplication respects modular equivalence. *}
 | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 248 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 249 | lemma mod_mult_left_eq: "(a * b) mod c = ((a mod c) * b) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 250 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 251 | have "(a * b) mod c = ((a div c * c + a mod c) * b) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 252 | by (simp only: mod_div_equality) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 253 | also have "\<dots> = (a mod c * b + a div c * b * c) mod c" | 
| 29667 | 254 | by (simp only: algebra_simps) | 
| 29403 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 255 | also have "\<dots> = (a mod c * b) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 256 | by (rule mod_mult_self1) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 257 | finally show ?thesis . | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 258 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 259 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 260 | lemma mod_mult_right_eq: "(a * b) mod c = (a * (b mod c)) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 261 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 262 | have "(a * b) mod c = (a * (b div c * c + b mod c)) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 263 | by (simp only: mod_div_equality) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 264 | also have "\<dots> = (a * (b mod c) + a * (b div c) * c) mod c" | 
| 29667 | 265 | by (simp only: algebra_simps) | 
| 29403 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 266 | also have "\<dots> = (a * (b mod c)) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 267 | by (rule mod_mult_self1) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 268 | finally show ?thesis . | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 269 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 270 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 271 | lemma mod_mult_eq: "(a * b) mod c = ((a mod c) * (b mod c)) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 272 | by (rule trans [OF mod_mult_left_eq mod_mult_right_eq]) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 273 | |
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 274 | lemma mod_mult_cong: | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 275 | assumes "a mod c = a' mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 276 | assumes "b mod c = b' mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 277 | shows "(a * b) mod c = (a' * b') mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 278 | proof - | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 279 | have "(a mod c * (b mod c)) mod c = (a' mod c * (b' mod c)) mod c" | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 280 | unfolding assms .. | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 281 | thus ?thesis | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 282 | by (simp only: mod_mult_eq [symmetric]) | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 283 | qed | 
| 
fe17df4e4ab3
generalize some div/mod lemmas; remove type-specific proofs
 huffman parents: 
29252diff
changeset | 284 | |
| 47164 | 285 | text {* Exponentiation respects modular equivalence. *}
 | 
| 286 | ||
| 287 | lemma power_mod: "(a mod b)^n mod b = a^n mod b" | |
| 288 | apply (induct n, simp_all) | |
| 289 | apply (rule mod_mult_right_eq [THEN trans]) | |
| 290 | apply (simp (no_asm_simp)) | |
| 291 | apply (rule mod_mult_eq [symmetric]) | |
| 292 | done | |
| 293 | ||
| 29404 | 294 | lemma mod_mod_cancel: | 
| 295 | assumes "c dvd b" | |
| 296 | shows "a mod b mod c = a mod c" | |
| 297 | proof - | |
| 298 | from `c dvd b` obtain k where "b = c * k" | |
| 299 | by (rule dvdE) | |
| 300 | have "a mod b mod c = a mod (c * k) mod c" | |
| 301 | by (simp only: `b = c * k`) | |
| 302 | also have "\<dots> = (a mod (c * k) + a div (c * k) * k * c) mod c" | |
| 303 | by (simp only: mod_mult_self1) | |
| 304 | also have "\<dots> = (a div (c * k) * (c * k) + a mod (c * k)) mod c" | |
| 305 | by (simp only: add_ac mult_ac) | |
| 306 | also have "\<dots> = a mod c" | |
| 307 | by (simp only: mod_div_equality) | |
| 308 | finally show ?thesis . | |
| 309 | qed | |
| 310 | ||
| 30930 | 311 | lemma div_mult_div_if_dvd: | 
| 312 | "y dvd x \<Longrightarrow> z dvd w \<Longrightarrow> (x div y) * (w div z) = (x * w) div (y * z)" | |
| 313 | apply (cases "y = 0", simp) | |
| 314 | apply (cases "z = 0", simp) | |
| 315 | apply (auto elim!: dvdE simp add: algebra_simps) | |
| 30476 | 316 | apply (subst mult_assoc [symmetric]) | 
| 317 | apply (simp add: no_zero_divisors) | |
| 30930 | 318 | done | 
| 319 | ||
| 35367 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 320 | lemma div_mult_swap: | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 321 | assumes "c dvd b" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 322 | shows "a * (b div c) = (a * b) div c" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 323 | proof - | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 324 | from assms have "b div c * (a div 1) = b * a div (c * 1)" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 325 | by (simp only: div_mult_div_if_dvd one_dvd) | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 326 | then show ?thesis by (simp add: mult_commute) | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 327 | qed | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 328 | |
| 30930 | 329 | lemma div_mult_mult2 [simp]: | 
| 330 | "c \<noteq> 0 \<Longrightarrow> (a * c) div (b * c) = a div b" | |
| 331 | by (drule div_mult_mult1) (simp add: mult_commute) | |
| 332 | ||
| 333 | lemma div_mult_mult1_if [simp]: | |
| 334 | "(c * a) div (c * b) = (if c = 0 then 0 else a div b)" | |
| 335 | by simp_all | |
| 30476 | 336 | |
| 30930 | 337 | lemma mod_mult_mult1: | 
| 338 | "(c * a) mod (c * b) = c * (a mod b)" | |
| 339 | proof (cases "c = 0") | |
| 340 | case True then show ?thesis by simp | |
| 341 | next | |
| 342 | case False | |
| 343 | from mod_div_equality | |
| 344 | have "((c * a) div (c * b)) * (c * b) + (c * a) mod (c * b) = c * a" . | |
| 345 | with False have "c * ((a div b) * b + a mod b) + (c * a) mod (c * b) | |
| 346 | = c * a + c * (a mod b)" by (simp add: algebra_simps) | |
| 347 | with mod_div_equality show ?thesis by simp | |
| 348 | qed | |
| 349 | ||
| 350 | lemma mod_mult_mult2: | |
| 351 | "(a * c) mod (b * c) = (a mod b) * c" | |
| 352 | using mod_mult_mult1 [of c a b] by (simp add: mult_commute) | |
| 353 | ||
| 47159 | 354 | lemma mult_mod_left: "(a mod b) * c = (a * c) mod (b * c)" | 
| 355 | by (fact mod_mult_mult2 [symmetric]) | |
| 356 | ||
| 357 | lemma mult_mod_right: "c * (a mod b) = (c * a) mod (c * b)" | |
| 358 | by (fact mod_mult_mult1 [symmetric]) | |
| 359 | ||
| 31662 
57f7ef0dba8e
generalize lemmas dvd_mod and dvd_mod_iff to class semiring_div
 huffman parents: 
31661diff
changeset | 360 | lemma dvd_mod: "k dvd m \<Longrightarrow> k dvd n \<Longrightarrow> k dvd (m mod n)" | 
| 
57f7ef0dba8e
generalize lemmas dvd_mod and dvd_mod_iff to class semiring_div
 huffman parents: 
31661diff
changeset | 361 | unfolding dvd_def by (auto simp add: mod_mult_mult1) | 
| 
57f7ef0dba8e
generalize lemmas dvd_mod and dvd_mod_iff to class semiring_div
 huffman parents: 
31661diff
changeset | 362 | |
| 
57f7ef0dba8e
generalize lemmas dvd_mod and dvd_mod_iff to class semiring_div
 huffman parents: 
31661diff
changeset | 363 | lemma dvd_mod_iff: "k dvd n \<Longrightarrow> k dvd (m mod n) \<longleftrightarrow> k dvd m" | 
| 
57f7ef0dba8e
generalize lemmas dvd_mod and dvd_mod_iff to class semiring_div
 huffman parents: 
31661diff
changeset | 364 | by (blast intro: dvd_mod_imp_dvd dvd_mod) | 
| 
57f7ef0dba8e
generalize lemmas dvd_mod and dvd_mod_iff to class semiring_div
 huffman parents: 
31661diff
changeset | 365 | |
| 31009 
41fd307cab30
dropped reference to class recpower and lemma duplicate
 haftmann parents: 
30934diff
changeset | 366 | lemma div_power: | 
| 31661 
1e252b8b2334
move lemma div_power into semiring_div context; class ring_div inherits from idom
 huffman parents: 
31009diff
changeset | 367 | "y dvd x \<Longrightarrow> (x div y) ^ n = x ^ n div y ^ n" | 
| 30476 | 368 | apply (induct n) | 
| 369 | apply simp | |
| 370 | apply(simp add: div_mult_div_if_dvd dvd_power_same) | |
| 371 | done | |
| 372 | ||
| 35367 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 373 | lemma dvd_div_eq_mult: | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 374 | assumes "a \<noteq> 0" and "a dvd b" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 375 | shows "b div a = c \<longleftrightarrow> b = c * a" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 376 | proof | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 377 | assume "b = c * a" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 378 | then show "b div a = c" by (simp add: assms) | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 379 | next | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 380 | assume "b div a = c" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 381 | then have "b div a * a = c * a" by simp | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 382 | moreover from `a dvd b` have "b div a * a = b" by (simp add: dvd_div_mult_self) | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 383 | ultimately show "b = c * a" by simp | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 384 | qed | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 385 | |
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 386 | lemma dvd_div_div_eq_mult: | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 387 | assumes "a \<noteq> 0" "c \<noteq> 0" and "a dvd b" "c dvd d" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 388 | shows "b div a = d div c \<longleftrightarrow> b * c = a * d" | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 389 | using assms by (auto simp add: mult_commute [of _ a] dvd_div_mult_self dvd_div_eq_mult div_mult_swap intro: sym) | 
| 
45a193f0ed0c
lemma div_mult_swap, dvd_div_eq_mult, dvd_div_div_eq_mult
 haftmann parents: 
35216diff
changeset | 390 | |
| 31661 
1e252b8b2334
move lemma div_power into semiring_div context; class ring_div inherits from idom
 huffman parents: 
31009diff
changeset | 391 | end | 
| 
1e252b8b2334
move lemma div_power into semiring_div context; class ring_div inherits from idom
 huffman parents: 
31009diff
changeset | 392 | |
| 35673 | 393 | class ring_div = semiring_div + comm_ring_1 | 
| 29405 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 394 | begin | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 395 | |
| 36634 | 396 | subclass ring_1_no_zero_divisors .. | 
| 397 | ||
| 29405 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 398 | text {* Negation respects modular equivalence. *}
 | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 399 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 400 | lemma mod_minus_eq: "(- a) mod b = (- (a mod b)) mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 401 | proof - | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 402 | have "(- a) mod b = (- (a div b * b + a mod b)) mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 403 | by (simp only: mod_div_equality) | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 404 | also have "\<dots> = (- (a mod b) + - (a div b) * b) mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 405 | by (simp only: minus_add_distrib minus_mult_left add_ac) | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 406 | also have "\<dots> = (- (a mod b)) mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 407 | by (rule mod_mult_self1) | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 408 | finally show ?thesis . | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 409 | qed | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 410 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 411 | lemma mod_minus_cong: | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 412 | assumes "a mod b = a' mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 413 | shows "(- a) mod b = (- a') mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 414 | proof - | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 415 | have "(- (a mod b)) mod b = (- (a' mod b)) mod b" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 416 | unfolding assms .. | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 417 | thus ?thesis | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 418 | by (simp only: mod_minus_eq [symmetric]) | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 419 | qed | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 420 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 421 | text {* Subtraction respects modular equivalence. *}
 | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 422 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 423 | lemma mod_diff_left_eq: "(a - b) mod c = (a mod c - b) mod c" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 424 | unfolding diff_minus | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 425 | by (intro mod_add_cong mod_minus_cong) simp_all | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 426 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 427 | lemma mod_diff_right_eq: "(a - b) mod c = (a - b mod c) mod c" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 428 | unfolding diff_minus | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 429 | by (intro mod_add_cong mod_minus_cong) simp_all | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 430 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 431 | lemma mod_diff_eq: "(a - b) mod c = (a mod c - b mod c) mod c" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 432 | unfolding diff_minus | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 433 | by (intro mod_add_cong mod_minus_cong) simp_all | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 434 | |
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 435 | lemma mod_diff_cong: | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 436 | assumes "a mod c = a' mod c" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 437 | assumes "b mod c = b' mod c" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 438 | shows "(a - b) mod c = (a' - b') mod c" | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 439 | unfolding diff_minus using assms | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 440 | by (intro mod_add_cong mod_minus_cong) | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 441 | |
| 30180 | 442 | lemma dvd_neg_div: "y dvd x \<Longrightarrow> -x div y = - (x div y)" | 
| 443 | apply (case_tac "y = 0") apply simp | |
| 444 | apply (auto simp add: dvd_def) | |
| 445 | apply (subgoal_tac "-(y * k) = y * - k") | |
| 446 | apply (erule ssubst) | |
| 447 | apply (erule div_mult_self1_is_id) | |
| 448 | apply simp | |
| 449 | done | |
| 450 | ||
| 451 | lemma dvd_div_neg: "y dvd x \<Longrightarrow> x div -y = - (x div y)" | |
| 452 | apply (case_tac "y = 0") apply simp | |
| 453 | apply (auto simp add: dvd_def) | |
| 454 | apply (subgoal_tac "y * k = -y * -k") | |
| 455 | apply (erule ssubst) | |
| 456 | apply (rule div_mult_self1_is_id) | |
| 457 | apply simp | |
| 458 | apply simp | |
| 459 | done | |
| 460 | ||
| 47159 | 461 | lemma div_minus_minus [simp]: "(-a) div (-b) = a div b" | 
| 462 | using div_mult_mult1 [of "- 1" a b] | |
| 463 | unfolding neg_equal_0_iff_equal by simp | |
| 464 | ||
| 465 | lemma mod_minus_minus [simp]: "(-a) mod (-b) = - (a mod b)" | |
| 466 | using mod_mult_mult1 [of "- 1" a b] by simp | |
| 467 | ||
| 468 | lemma div_minus_right: "a div (-b) = (-a) div b" | |
| 469 | using div_minus_minus [of "-a" b] by simp | |
| 470 | ||
| 471 | lemma mod_minus_right: "a mod (-b) = - ((-a) mod b)" | |
| 472 | using mod_minus_minus [of "-a" b] by simp | |
| 473 | ||
| 47160 | 474 | lemma div_minus1_right [simp]: "a div (-1) = -a" | 
| 475 | using div_minus_right [of a 1] by simp | |
| 476 | ||
| 477 | lemma mod_minus1_right [simp]: "a mod (-1) = 0" | |
| 478 | using mod_minus_right [of a 1] by simp | |
| 479 | ||
| 29405 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 480 | end | 
| 
98ab21b14f09
add class ring_div; generalize mod/diff/minus proofs for class ring_div
 huffman parents: 
29404diff
changeset | 481 | |
| 25942 | 482 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 483 | subsection {* Division on @{typ nat} *}
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 484 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 485 | text {*
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 486 |   We define @{const div} and @{const mod} on @{typ nat} by means
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 487 | of a characteristic relation with two input arguments | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 488 |   @{term "m\<Colon>nat"}, @{term "n\<Colon>nat"} and two output arguments
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 489 |   @{term "q\<Colon>nat"}(uotient) and @{term "r\<Colon>nat"}(emainder).
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 490 | *} | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 491 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 492 | definition divmod_nat_rel :: "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat \<Rightarrow> bool" where | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 493 | "divmod_nat_rel m n qr \<longleftrightarrow> | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 494 | m = fst qr * n + snd qr \<and> | 
| 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 495 | (if n = 0 then fst qr = 0 else if n > 0 then 0 \<le> snd qr \<and> snd qr < n else n < snd qr \<and> snd qr \<le> 0)" | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 496 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 497 | text {* @{const divmod_nat_rel} is total: *}
 | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 498 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 499 | lemma divmod_nat_rel_ex: | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 500 | obtains q r where "divmod_nat_rel m n (q, r)" | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 501 | proof (cases "n = 0") | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 502 | case True with that show thesis | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 503 | by (auto simp add: divmod_nat_rel_def) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 504 | next | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 505 | case False | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 506 | have "\<exists>q r. m = q * n + r \<and> r < n" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 507 | proof (induct m) | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 508 | case 0 with `n \<noteq> 0` | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 509 | have "(0\<Colon>nat) = 0 * n + 0 \<and> 0 < n" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 510 | then show ?case by blast | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 511 | next | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 512 | case (Suc m) then obtain q' r' | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 513 | where m: "m = q' * n + r'" and n: "r' < n" by auto | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 514 | then show ?case proof (cases "Suc r' < n") | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 515 | case True | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 516 | from m n have "Suc m = q' * n + Suc r'" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 517 | with True show ?thesis by blast | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 518 | next | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 519 | case False then have "n \<le> Suc r'" by auto | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 520 | moreover from n have "Suc r' \<le> n" by auto | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 521 | ultimately have "n = Suc r'" by auto | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 522 | with m have "Suc m = Suc q' * n + 0" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 523 | with `n \<noteq> 0` show ?thesis by blast | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 524 | qed | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 525 | qed | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 526 | with that show thesis | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 527 | using `n \<noteq> 0` by (auto simp add: divmod_nat_rel_def) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 528 | qed | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 529 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 530 | text {* @{const divmod_nat_rel} is injective: *}
 | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 531 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 532 | lemma divmod_nat_rel_unique: | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 533 | assumes "divmod_nat_rel m n qr" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 534 | and "divmod_nat_rel m n qr'" | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 535 | shows "qr = qr'" | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 536 | proof (cases "n = 0") | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 537 | case True with assms show ?thesis | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 538 | by (cases qr, cases qr') | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 539 | (simp add: divmod_nat_rel_def) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 540 | next | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 541 | case False | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 542 | have aux: "\<And>q r q' r'. q' * n + r' = q * n + r \<Longrightarrow> r < n \<Longrightarrow> q' \<le> (q\<Colon>nat)" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 543 | apply (rule leI) | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 544 | apply (subst less_iff_Suc_add) | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 545 | apply (auto simp add: add_mult_distrib) | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 546 | done | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 547 | from `n \<noteq> 0` assms have "fst qr = fst qr'" | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 548 | by (auto simp add: divmod_nat_rel_def intro: order_antisym dest: aux sym) | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 549 | moreover from this assms have "snd qr = snd qr'" | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 550 | by (simp add: divmod_nat_rel_def) | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 551 | ultimately show ?thesis by (cases qr, cases qr') simp | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 552 | qed | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 553 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 554 | text {*
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 555 | We instantiate divisibility on the natural numbers by | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 556 |   means of @{const divmod_nat_rel}:
 | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 557 | *} | 
| 25942 | 558 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 559 | definition divmod_nat :: "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat" where | 
| 37767 | 560 | "divmod_nat m n = (THE qr. divmod_nat_rel m n qr)" | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 561 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 562 | lemma divmod_nat_rel_divmod_nat: | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 563 | "divmod_nat_rel m n (divmod_nat m n)" | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 564 | proof - | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 565 | from divmod_nat_rel_ex | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 566 | obtain qr where rel: "divmod_nat_rel m n qr" . | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 567 | then show ?thesis | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 568 | by (auto simp add: divmod_nat_def intro: theI elim: divmod_nat_rel_unique) | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 569 | qed | 
| 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 570 | |
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 571 | lemma divmod_nat_unique: | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 572 | assumes "divmod_nat_rel m n qr" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 573 | shows "divmod_nat m n = qr" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 574 | using assms by (auto intro: divmod_nat_rel_unique divmod_nat_rel_divmod_nat) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 575 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 576 | instantiation nat :: semiring_div | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 577 | begin | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 578 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 579 | definition div_nat where | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 580 | "m div n = fst (divmod_nat m n)" | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 581 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 582 | lemma fst_divmod_nat [simp]: | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 583 | "fst (divmod_nat m n) = m div n" | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 584 | by (simp add: div_nat_def) | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 585 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 586 | definition mod_nat where | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 587 | "m mod n = snd (divmod_nat m n)" | 
| 25571 
c9e39eafc7a0
instantiation target rather than legacy instance
 haftmann parents: 
25162diff
changeset | 588 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 589 | lemma snd_divmod_nat [simp]: | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 590 | "snd (divmod_nat m n) = m mod n" | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 591 | by (simp add: mod_nat_def) | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 592 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 593 | lemma divmod_nat_div_mod: | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 594 | "divmod_nat m n = (m div n, m mod n)" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 595 | by (simp add: prod_eq_iff) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 596 | |
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 597 | lemma div_nat_unique: | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 598 | assumes "divmod_nat_rel m n (q, r)" | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 599 | shows "m div n = q" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 600 | using assms by (auto dest!: divmod_nat_unique simp add: prod_eq_iff) | 
| 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 601 | |
| 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 602 | lemma mod_nat_unique: | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 603 | assumes "divmod_nat_rel m n (q, r)" | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 604 | shows "m mod n = r" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 605 | using assms by (auto dest!: divmod_nat_unique simp add: prod_eq_iff) | 
| 25571 
c9e39eafc7a0
instantiation target rather than legacy instance
 haftmann parents: 
25162diff
changeset | 606 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 607 | lemma divmod_nat_rel: "divmod_nat_rel m n (m div n, m mod n)" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 608 | using divmod_nat_rel_divmod_nat by (simp add: divmod_nat_div_mod) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 609 | |
| 47136 | 610 | lemma divmod_nat_zero: "divmod_nat m 0 = (0, m)" | 
| 611 | by (simp add: divmod_nat_unique divmod_nat_rel_def) | |
| 612 | ||
| 613 | lemma divmod_nat_zero_left: "divmod_nat 0 n = (0, 0)" | |
| 614 | by (simp add: divmod_nat_unique divmod_nat_rel_def) | |
| 25942 | 615 | |
| 47137 | 616 | lemma divmod_nat_base: "m < n \<Longrightarrow> divmod_nat m n = (0, m)" | 
| 617 | by (simp add: divmod_nat_unique divmod_nat_rel_def) | |
| 25942 | 618 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 619 | lemma divmod_nat_step: | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 620 | assumes "0 < n" and "n \<le> m" | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 621 | shows "divmod_nat m n = (Suc ((m - n) div n), (m - n) mod n)" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 622 | proof (rule divmod_nat_unique) | 
| 47134 | 623 | have "divmod_nat_rel (m - n) n ((m - n) div n, (m - n) mod n)" | 
| 624 | by (rule divmod_nat_rel) | |
| 625 | thus "divmod_nat_rel m n (Suc ((m - n) div n), (m - n) mod n)" | |
| 626 | unfolding divmod_nat_rel_def using assms by auto | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 627 | qed | 
| 25942 | 628 | |
| 26300 | 629 | text {* The ''recursion'' equations for @{const div} and @{const mod} *}
 | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 630 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 631 | lemma div_less [simp]: | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 632 | fixes m n :: nat | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 633 | assumes "m < n" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 634 | shows "m div n = 0" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 635 | using assms divmod_nat_base by (simp add: prod_eq_iff) | 
| 25942 | 636 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 637 | lemma le_div_geq: | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 638 | fixes m n :: nat | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 639 | assumes "0 < n" and "n \<le> m" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 640 | shows "m div n = Suc ((m - n) div n)" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 641 | using assms divmod_nat_step by (simp add: prod_eq_iff) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 642 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 643 | lemma mod_less [simp]: | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 644 | fixes m n :: nat | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 645 | assumes "m < n" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 646 | shows "m mod n = m" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 647 | using assms divmod_nat_base by (simp add: prod_eq_iff) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 648 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 649 | lemma le_mod_geq: | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 650 | fixes m n :: nat | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 651 | assumes "n \<le> m" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 652 | shows "m mod n = (m - n) mod n" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 653 | using assms divmod_nat_step by (cases "n = 0") (simp_all add: prod_eq_iff) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 654 | |
| 47136 | 655 | instance proof | 
| 656 | fix m n :: nat | |
| 657 | show "m div n * n + m mod n = m" | |
| 658 | using divmod_nat_rel [of m n] by (simp add: divmod_nat_rel_def) | |
| 659 | next | |
| 660 | fix m n q :: nat | |
| 661 | assume "n \<noteq> 0" | |
| 662 | then show "(q + m * n) div n = m + q div n" | |
| 663 | by (induct m) (simp_all add: le_div_geq) | |
| 664 | next | |
| 665 | fix m n q :: nat | |
| 666 | assume "m \<noteq> 0" | |
| 667 | hence "\<And>a b. divmod_nat_rel n q (a, b) \<Longrightarrow> divmod_nat_rel (m * n) (m * q) (a, m * b)" | |
| 668 | unfolding divmod_nat_rel_def | |
| 669 | by (auto split: split_if_asm, simp_all add: algebra_simps) | |
| 670 | moreover from divmod_nat_rel have "divmod_nat_rel n q (n div q, n mod q)" . | |
| 671 | ultimately have "divmod_nat_rel (m * n) (m * q) (n div q, m * (n mod q))" . | |
| 672 | thus "(m * n) div (m * q) = n div q" by (rule div_nat_unique) | |
| 673 | next | |
| 674 | fix n :: nat show "n div 0 = 0" | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 675 | by (simp add: div_nat_def divmod_nat_zero) | 
| 47136 | 676 | next | 
| 677 | fix n :: nat show "0 div n = 0" | |
| 678 | by (simp add: div_nat_def divmod_nat_zero_left) | |
| 25942 | 679 | qed | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 680 | |
| 25942 | 681 | end | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 682 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 683 | lemma divmod_nat_if [code]: "divmod_nat m n = (if n = 0 \<or> m < n then (0, m) else | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 684 | let (q, r) = divmod_nat (m - n) n in (Suc q, r))" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 685 | by (simp add: prod_eq_iff prod_case_beta not_less le_div_geq le_mod_geq) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 686 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 687 | text {* Simproc for cancelling @{const div} and @{const mod} *}
 | 
| 25942 | 688 | |
| 30934 | 689 | ML {*
 | 
| 43594 | 690 | structure Cancel_Div_Mod_Nat = Cancel_Div_Mod | 
| 41550 | 691 | ( | 
| 30934 | 692 |   val div_name = @{const_name div};
 | 
| 693 |   val mod_name = @{const_name mod};
 | |
| 694 | val mk_binop = HOLogic.mk_binop; | |
| 48561 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 695 |   val mk_plus = HOLogic.mk_binop @{const_name Groups.plus};
 | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 696 |   val dest_plus = HOLogic.dest_bin @{const_name Groups.plus} HOLogic.natT;
 | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 697 | fun mk_sum [] = HOLogic.zero | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 698 | | mk_sum [t] = t | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 699 | | mk_sum (t :: ts) = mk_plus (t, mk_sum ts); | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 700 | fun dest_sum tm = | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 701 | if HOLogic.is_zero tm then [] | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 702 | else | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 703 | (case try HOLogic.dest_Suc tm of | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 704 | SOME t => HOLogic.Suc_zero :: dest_sum t | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 705 | | NONE => | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 706 | (case try dest_plus tm of | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 707 | SOME (t, u) => dest_sum t @ dest_sum u | 
| 
12aa0cb2b447
move ML functions from nat_arith.ML to Divides.thy, which is the only place they are used
 huffman parents: 
47268diff
changeset | 708 | | NONE => [tm])); | 
| 25942 | 709 | |
| 30934 | 710 |   val div_mod_eqs = map mk_meta_eq [@{thm div_mod_equality}, @{thm div_mod_equality2}];
 | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 711 | |
| 30934 | 712 | val prove_eq_sums = Arith_Data.prove_conv2 all_tac (Arith_Data.simp_all_tac | 
| 35050 
9f841f20dca6
renamed OrderedGroup to Groups; split theory Ring_and_Field into Rings Fields
 haftmann parents: 
34982diff
changeset | 713 |     (@{thm add_0_left} :: @{thm add_0_right} :: @{thms add_ac}))
 | 
| 41550 | 714 | ) | 
| 25942 | 715 | *} | 
| 716 | ||
| 43594 | 717 | simproc_setup cancel_div_mod_nat ("(m::nat) + n") = {* K Cancel_Div_Mod_Nat.proc *}
 | 
| 718 | ||
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 719 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 720 | subsubsection {* Quotient *}
 | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 721 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 722 | lemma div_geq: "0 < n \<Longrightarrow> \<not> m < n \<Longrightarrow> m div n = Suc ((m - n) div n)" | 
| 29667 | 723 | by (simp add: le_div_geq linorder_not_less) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 724 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 725 | lemma div_if: "0 < n \<Longrightarrow> m div n = (if m < n then 0 else Suc ((m - n) div n))" | 
| 29667 | 726 | by (simp add: div_geq) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 727 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 728 | lemma div_mult_self_is_m [simp]: "0<n ==> (m*n) div n = (m::nat)" | 
| 29667 | 729 | by simp | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 730 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 731 | lemma div_mult_self1_is_m [simp]: "0<n ==> (n*m) div n = (m::nat)" | 
| 29667 | 732 | by simp | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 733 | |
| 25942 | 734 | |
| 735 | subsubsection {* Remainder *}
 | |
| 736 | ||
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 737 | lemma mod_less_divisor [simp]: | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 738 | fixes m n :: nat | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 739 | assumes "n > 0" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 740 | shows "m mod n < (n::nat)" | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 741 | using assms divmod_nat_rel [of m n] unfolding divmod_nat_rel_def by auto | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 742 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 743 | lemma mod_less_eq_dividend [simp]: | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 744 | fixes m n :: nat | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 745 | shows "m mod n \<le> m" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 746 | proof (rule add_leD2) | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 747 | from mod_div_equality have "m div n * n + m mod n = m" . | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 748 | then show "m div n * n + m mod n \<le> m" by auto | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 749 | qed | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 750 | |
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 751 | lemma mod_geq: "\<not> m < (n\<Colon>nat) \<Longrightarrow> m mod n = (m - n) mod n" | 
| 29667 | 752 | by (simp add: le_mod_geq linorder_not_less) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 753 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 754 | lemma mod_if: "m mod (n\<Colon>nat) = (if m < n then m else (m - n) mod n)" | 
| 29667 | 755 | by (simp add: le_mod_geq) | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 756 | |
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 757 | lemma mod_1 [simp]: "m mod Suc 0 = 0" | 
| 29667 | 758 | by (induct m) (simp_all add: mod_geq) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 759 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 760 | (* a simple rearrangement of mod_div_equality: *) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 761 | lemma mult_div_cancel: "(n::nat) * (m div n) = m - (m mod n)" | 
| 47138 | 762 | using mod_div_equality2 [of n m] by arith | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 763 | |
| 15439 | 764 | lemma mod_le_divisor[simp]: "0 < n \<Longrightarrow> m mod n \<le> (n::nat)" | 
| 22718 | 765 | apply (drule mod_less_divisor [where m = m]) | 
| 766 | apply simp | |
| 767 | done | |
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 768 | |
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 769 | subsubsection {* Quotient and Remainder *}
 | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 770 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 771 | lemma divmod_nat_rel_mult1_eq: | 
| 46552 | 772 | "divmod_nat_rel b c (q, r) | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 773 | \<Longrightarrow> divmod_nat_rel (a * b) c (a * q + a * r div c, a * r mod c)" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 774 | by (auto simp add: split_ifs divmod_nat_rel_def algebra_simps) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 775 | |
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 776 | lemma div_mult1_eq: | 
| 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 777 | "(a * b) div c = a * (b div c) + a * (b mod c) div (c::nat)" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 778 | by (blast intro: divmod_nat_rel_mult1_eq [THEN div_nat_unique] divmod_nat_rel) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 779 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 780 | lemma divmod_nat_rel_add1_eq: | 
| 46552 | 781 | "divmod_nat_rel a c (aq, ar) \<Longrightarrow> divmod_nat_rel b c (bq, br) | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 782 | \<Longrightarrow> divmod_nat_rel (a + b) c (aq + bq + (ar + br) div c, (ar + br) mod c)" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 783 | by (auto simp add: split_ifs divmod_nat_rel_def algebra_simps) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 784 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 785 | (*NOT suitable for rewriting: the RHS has an instance of the LHS*) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 786 | lemma div_add1_eq: | 
| 25134 
3d4953e88449
Eliminated most of the neq0_conv occurrences. As a result, many
 nipkow parents: 
25112diff
changeset | 787 | "(a+b) div (c::nat) = a div c + b div c + ((a mod c + b mod c) div c)" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 788 | by (blast intro: divmod_nat_rel_add1_eq [THEN div_nat_unique] divmod_nat_rel) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 789 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 790 | lemma mod_lemma: "[| (0::nat) < c; r < b |] ==> b * (q mod c) + r < b * c" | 
| 22718 | 791 | apply (cut_tac m = q and n = c in mod_less_divisor) | 
| 792 | apply (drule_tac [2] m = "q mod c" in less_imp_Suc_add, auto) | |
| 793 | apply (erule_tac P = "%x. ?lhs < ?rhs x" in ssubst) | |
| 794 | apply (simp add: add_mult_distrib2) | |
| 795 | done | |
| 10559 
d3fd54fc659b
many new div and mod properties (borrowed from Integ/IntDiv)
 paulson parents: 
10214diff
changeset | 796 | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 797 | lemma divmod_nat_rel_mult2_eq: | 
| 46552 | 798 | "divmod_nat_rel a b (q, r) | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 799 | \<Longrightarrow> divmod_nat_rel a (b * c) (q div c, b *(q mod c) + r)" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 800 | by (auto simp add: mult_ac divmod_nat_rel_def add_mult_distrib2 [symmetric] mod_lemma) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 801 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 802 | lemma div_mult2_eq: "a div (b*c) = (a div b) div (c::nat)" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 803 | by (force simp add: divmod_nat_rel [THEN divmod_nat_rel_mult2_eq, THEN div_nat_unique]) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 804 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 805 | lemma mod_mult2_eq: "a mod (b*c) = b*(a div b mod c) + a mod (b::nat)" | 
| 47135 
fb67b596067f
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
 huffman parents: 
47134diff
changeset | 806 | by (auto simp add: mult_commute divmod_nat_rel [THEN divmod_nat_rel_mult2_eq, THEN mod_nat_unique]) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 807 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 808 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 809 | subsubsection {* Further Facts about Quotient and Remainder *}
 | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 810 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 811 | lemma div_1 [simp]: "m div Suc 0 = m" | 
| 29667 | 812 | by (induct m) (simp_all add: div_geq) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 813 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 814 | (* Monotonicity of div in first argument *) | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 815 | lemma div_le_mono [rule_format (no_asm)]: | 
| 22718 | 816 | "\<forall>m::nat. m \<le> n --> (m div k) \<le> (n div k)" | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 817 | apply (case_tac "k=0", simp) | 
| 15251 | 818 | apply (induct "n" rule: nat_less_induct, clarify) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 819 | apply (case_tac "n<k") | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 820 | (* 1 case n<k *) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 821 | apply simp | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 822 | (* 2 case n >= k *) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 823 | apply (case_tac "m<k") | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 824 | (* 2.1 case m<k *) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 825 | apply simp | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 826 | (* 2.2 case m>=k *) | 
| 15439 | 827 | apply (simp add: div_geq diff_le_mono) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 828 | done | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 829 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 830 | (* Antimonotonicity of div in second argument *) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 831 | lemma div_le_mono2: "!!m::nat. [| 0<m; m\<le>n |] ==> (k div n) \<le> (k div m)" | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 832 | apply (subgoal_tac "0<n") | 
| 22718 | 833 | prefer 2 apply simp | 
| 15251 | 834 | apply (induct_tac k rule: nat_less_induct) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 835 | apply (rename_tac "k") | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 836 | apply (case_tac "k<n", simp) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 837 | apply (subgoal_tac "~ (k<m) ") | 
| 22718 | 838 | prefer 2 apply simp | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 839 | apply (simp add: div_geq) | 
| 15251 | 840 | apply (subgoal_tac "(k-n) div n \<le> (k-m) div n") | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 841 | prefer 2 | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 842 | apply (blast intro: div_le_mono diff_le_mono2) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 843 | apply (rule le_trans, simp) | 
| 15439 | 844 | apply (simp) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 845 | done | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 846 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 847 | lemma div_le_dividend [simp]: "m div n \<le> (m::nat)" | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 848 | apply (case_tac "n=0", simp) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 849 | apply (subgoal_tac "m div n \<le> m div 1", simp) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 850 | apply (rule div_le_mono2) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 851 | apply (simp_all (no_asm_simp)) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 852 | done | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 853 | |
| 22718 | 854 | (* Similar for "less than" *) | 
| 47138 | 855 | lemma div_less_dividend [simp]: | 
| 856 | "\<lbrakk>(1::nat) < n; 0 < m\<rbrakk> \<Longrightarrow> m div n < m" | |
| 857 | apply (induct m rule: nat_less_induct) | |
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 858 | apply (rename_tac "m") | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 859 | apply (case_tac "m<n", simp) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 860 | apply (subgoal_tac "0<n") | 
| 22718 | 861 | prefer 2 apply simp | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 862 | apply (simp add: div_geq) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 863 | apply (case_tac "n<m") | 
| 15251 | 864 | apply (subgoal_tac "(m-n) div n < (m-n) ") | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 865 | apply (rule impI less_trans_Suc)+ | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 866 | apply assumption | 
| 15439 | 867 | apply (simp_all) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 868 | done | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 869 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 870 | text{*A fact for the mutilated chess board*}
 | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 871 | lemma mod_Suc: "Suc(m) mod n = (if Suc(m mod n) = n then 0 else Suc(m mod n))" | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 872 | apply (case_tac "n=0", simp) | 
| 15251 | 873 | apply (induct "m" rule: nat_less_induct) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 874 | apply (case_tac "Suc (na) <n") | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 875 | (* case Suc(na) < n *) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 876 | apply (frule lessI [THEN less_trans], simp add: less_not_refl3) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 877 | (* case n \<le> Suc(na) *) | 
| 16796 | 878 | apply (simp add: linorder_not_less le_Suc_eq mod_geq) | 
| 15439 | 879 | apply (auto simp add: Suc_diff_le le_mod_geq) | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 880 | done | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 881 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 882 | lemma mod_eq_0_iff: "(m mod d = 0) = (\<exists>q::nat. m = d*q)" | 
| 29667 | 883 | by (auto simp add: dvd_eq_mod_eq_0 [symmetric] dvd_def) | 
| 17084 
fb0a80aef0be
classical rules must have names for ATP integration
 paulson parents: 
16796diff
changeset | 884 | |
| 22718 | 885 | lemmas mod_eq_0D [dest!] = mod_eq_0_iff [THEN iffD1] | 
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 886 | |
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 887 | (*Loses information, namely we also have r<d provided d is nonzero*) | 
| 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 888 | lemma mod_eqD: "(m mod d = r) ==> \<exists>q::nat. m = r + q*d" | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 889 | apply (cut_tac a = m in mod_div_equality) | 
| 22718 | 890 | apply (simp only: add_ac) | 
| 891 | apply (blast intro: sym) | |
| 892 | done | |
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 893 | |
| 13152 | 894 | lemma split_div: | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 895 | "P(n div k :: nat) = | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 896 | ((k = 0 \<longrightarrow> P 0) \<and> (k \<noteq> 0 \<longrightarrow> (!i. !j<k. n = k*i + j \<longrightarrow> P i)))" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 897 | (is "?P = ?Q" is "_ = (_ \<and> (_ \<longrightarrow> ?R))") | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 898 | proof | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 899 | assume P: ?P | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 900 | show ?Q | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 901 | proof (cases) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 902 | assume "k = 0" | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 903 | with P show ?Q by simp | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 904 | next | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 905 | assume not0: "k \<noteq> 0" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 906 | thus ?Q | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 907 | proof (simp, intro allI impI) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 908 | fix i j | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 909 | assume n: "n = k*i + j" and j: "j < k" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 910 | show "P i" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 911 | proof (cases) | 
| 22718 | 912 | assume "i = 0" | 
| 913 | with n j P show "P i" by simp | |
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 914 | next | 
| 22718 | 915 | assume "i \<noteq> 0" | 
| 916 | with not0 n j P show "P i" by(simp add:add_ac) | |
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 917 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 918 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 919 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 920 | next | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 921 | assume Q: ?Q | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 922 | show ?P | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 923 | proof (cases) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 924 | assume "k = 0" | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 925 | with Q show ?P by simp | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 926 | next | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 927 | assume not0: "k \<noteq> 0" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 928 | with Q have R: ?R by simp | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 929 | from not0 R[THEN spec,of "n div k",THEN spec, of "n mod k"] | 
| 13517 | 930 | show ?P by simp | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 931 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 932 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 933 | |
| 13882 | 934 | lemma split_div_lemma: | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 935 | assumes "0 < n" | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 936 | shows "n * q \<le> m \<and> m < n * Suc q \<longleftrightarrow> q = ((m\<Colon>nat) div n)" (is "?lhs \<longleftrightarrow> ?rhs") | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 937 | proof | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 938 | assume ?rhs | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 939 | with mult_div_cancel have nq: "n * q = m - (m mod n)" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 940 | then have A: "n * q \<le> m" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 941 | have "n - (m mod n) > 0" using mod_less_divisor assms by auto | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 942 | then have "m < m + (n - (m mod n))" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 943 | then have "m < n + (m - (m mod n))" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 944 | with nq have "m < n + n * q" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 945 | then have B: "m < n * Suc q" by simp | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 946 | from A B show ?lhs .. | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 947 | next | 
| 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 948 | assume P: ?lhs | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 949 | then have "divmod_nat_rel m n (q, m - n * q)" | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 950 | unfolding divmod_nat_rel_def by (auto simp add: mult_ac) | 
| 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 951 | with divmod_nat_rel_unique divmod_nat_rel [of m n] | 
| 30923 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 952 | have "(q, m - n * q) = (m div n, m mod n)" by auto | 
| 
2697a1d1d34a
more coherent developement in Divides.thy and IntDiv.thy
 haftmann parents: 
30840diff
changeset | 953 | then show ?rhs by simp | 
| 26100 
fbc60cd02ae2
using only an relation predicate to construct div and mod
 haftmann parents: 
26072diff
changeset | 954 | qed | 
| 13882 | 955 | |
| 956 | theorem split_div': | |
| 957 | "P ((m::nat) div n) = ((n = 0 \<and> P 0) \<or> | |
| 14267 
b963e9cee2a0
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
 paulson parents: 
14208diff
changeset | 958 | (\<exists>q. (n * q \<le> m \<and> m < n * (Suc q)) \<and> P q))" | 
| 13882 | 959 | apply (case_tac "0 < n") | 
| 960 | apply (simp only: add: split_div_lemma) | |
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 961 | apply simp_all | 
| 13882 | 962 | done | 
| 963 | ||
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 964 | lemma split_mod: | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 965 | "P(n mod k :: nat) = | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 966 | ((k = 0 \<longrightarrow> P n) \<and> (k \<noteq> 0 \<longrightarrow> (!i. !j<k. n = k*i + j \<longrightarrow> P j)))" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 967 | (is "?P = ?Q" is "_ = (_ \<and> (_ \<longrightarrow> ?R))") | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 968 | proof | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 969 | assume P: ?P | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 970 | show ?Q | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 971 | proof (cases) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 972 | assume "k = 0" | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 973 | with P show ?Q by simp | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 974 | next | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 975 | assume not0: "k \<noteq> 0" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 976 | thus ?Q | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 977 | proof (simp, intro allI impI) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 978 | fix i j | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 979 | assume "n = k*i + j" "j < k" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 980 | thus "P j" using not0 P by(simp add:add_ac mult_ac) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 981 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 982 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 983 | next | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 984 | assume Q: ?Q | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 985 | show ?P | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 986 | proof (cases) | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 987 | assume "k = 0" | 
| 27651 
16a26996c30e
moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
 haftmann parents: 
27540diff
changeset | 988 | with Q show ?P by simp | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 989 | next | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 990 | assume not0: "k \<noteq> 0" | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 991 | with Q have R: ?R by simp | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 992 | from not0 R[THEN spec,of "n div k",THEN spec, of "n mod k"] | 
| 13517 | 993 | show ?P by simp | 
| 13189 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 994 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 995 | qed | 
| 
81ed5c6de890
Now arith can deal with div/mod arbitrary nat numerals.
 nipkow parents: 
13152diff
changeset | 996 | |
| 13882 | 997 | theorem mod_div_equality': "(m::nat) mod n = m - (m div n) * n" | 
| 47138 | 998 | using mod_div_equality [of m n] by arith | 
| 999 | ||
| 1000 | lemma div_mod_equality': "(m::nat) div n * n = m - m mod n" | |
| 1001 | using mod_div_equality [of m n] by arith | |
| 1002 | (* FIXME: very similar to mult_div_cancel *) | |
| 22800 | 1003 | |
| 1004 | ||
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1005 | subsubsection {* An ``induction'' law for modulus arithmetic. *}
 | 
| 14640 | 1006 | |
| 1007 | lemma mod_induct_0: | |
| 1008 | assumes step: "\<forall>i<p. P i \<longrightarrow> P ((Suc i) mod p)" | |
| 1009 | and base: "P i" and i: "i<p" | |
| 1010 | shows "P 0" | |
| 1011 | proof (rule ccontr) | |
| 1012 | assume contra: "\<not>(P 0)" | |
| 1013 | from i have p: "0<p" by simp | |
| 1014 | have "\<forall>k. 0<k \<longrightarrow> \<not> P (p-k)" (is "\<forall>k. ?A k") | |
| 1015 | proof | |
| 1016 | fix k | |
| 1017 | show "?A k" | |
| 1018 | proof (induct k) | |
| 1019 | show "?A 0" by simp -- "by contradiction" | |
| 1020 | next | |
| 1021 | fix n | |
| 1022 | assume ih: "?A n" | |
| 1023 | show "?A (Suc n)" | |
| 1024 | proof (clarsimp) | |
| 22718 | 1025 | assume y: "P (p - Suc n)" | 
| 1026 | have n: "Suc n < p" | |
| 1027 | proof (rule ccontr) | |
| 1028 | assume "\<not>(Suc n < p)" | |
| 1029 | hence "p - Suc n = 0" | |
| 1030 | by simp | |
| 1031 | with y contra show "False" | |
| 1032 | by simp | |
| 1033 | qed | |
| 1034 | hence n2: "Suc (p - Suc n) = p-n" by arith | |
| 1035 | from p have "p - Suc n < p" by arith | |
| 1036 | with y step have z: "P ((Suc (p - Suc n)) mod p)" | |
| 1037 | by blast | |
| 1038 | show "False" | |
| 1039 | proof (cases "n=0") | |
| 1040 | case True | |
| 1041 | with z n2 contra show ?thesis by simp | |
| 1042 | next | |
| 1043 | case False | |
| 1044 | with p have "p-n < p" by arith | |
| 1045 | with z n2 False ih show ?thesis by simp | |
| 1046 | qed | |
| 14640 | 1047 | qed | 
| 1048 | qed | |
| 1049 | qed | |
| 1050 | moreover | |
| 1051 | from i obtain k where "0<k \<and> i+k=p" | |
| 1052 | by (blast dest: less_imp_add_positive) | |
| 1053 | hence "0<k \<and> i=p-k" by auto | |
| 1054 | moreover | |
| 1055 | note base | |
| 1056 | ultimately | |
| 1057 | show "False" by blast | |
| 1058 | qed | |
| 1059 | ||
| 1060 | lemma mod_induct: | |
| 1061 | assumes step: "\<forall>i<p. P i \<longrightarrow> P ((Suc i) mod p)" | |
| 1062 | and base: "P i" and i: "i<p" and j: "j<p" | |
| 1063 | shows "P j" | |
| 1064 | proof - | |
| 1065 | have "\<forall>j<p. P j" | |
| 1066 | proof | |
| 1067 | fix j | |
| 1068 | show "j<p \<longrightarrow> P j" (is "?A j") | |
| 1069 | proof (induct j) | |
| 1070 | from step base i show "?A 0" | |
| 22718 | 1071 | by (auto elim: mod_induct_0) | 
| 14640 | 1072 | next | 
| 1073 | fix k | |
| 1074 | assume ih: "?A k" | |
| 1075 | show "?A (Suc k)" | |
| 1076 | proof | |
| 22718 | 1077 | assume suc: "Suc k < p" | 
| 1078 | hence k: "k<p" by simp | |
| 1079 | with ih have "P k" .. | |
| 1080 | with step k have "P (Suc k mod p)" | |
| 1081 | by blast | |
| 1082 | moreover | |
| 1083 | from suc have "Suc k mod p = Suc k" | |
| 1084 | by simp | |
| 1085 | ultimately | |
| 1086 | show "P (Suc k)" by simp | |
| 14640 | 1087 | qed | 
| 1088 | qed | |
| 1089 | qed | |
| 1090 | with j show ?thesis by blast | |
| 1091 | qed | |
| 1092 | ||
| 33296 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1093 | lemma div2_Suc_Suc [simp]: "Suc (Suc m) div 2 = Suc (m div 2)" | 
| 47138 | 1094 | by (simp add: numeral_2_eq_2 le_div_geq) | 
| 1095 | ||
| 1096 | lemma mod2_Suc_Suc [simp]: "Suc (Suc m) mod 2 = m mod 2" | |
| 1097 | by (simp add: numeral_2_eq_2 le_mod_geq) | |
| 33296 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1098 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1099 | lemma add_self_div_2 [simp]: "(m + m) div 2 = (m::nat)" | 
| 47217 
501b9bbd0d6e
removed redundant nat-specific copies of theorems
 huffman parents: 
47167diff
changeset | 1100 | by (simp add: mult_2 [symmetric]) | 
| 33296 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1101 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1102 | lemma mod2_gr_0 [simp]: "0 < (m\<Colon>nat) mod 2 \<longleftrightarrow> m mod 2 = 1" | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1103 | proof - | 
| 35815 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 1104 |   { fix n :: nat have  "(n::nat) < 2 \<Longrightarrow> n = 0 \<or> n = 1" by (cases n) simp_all }
 | 
| 33296 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1105 | moreover have "m mod 2 < 2" by simp | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1106 | ultimately have "m mod 2 = 0 \<or> m mod 2 = 1" . | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1107 | then show ?thesis by auto | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1108 | qed | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1109 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1110 | text{*These lemmas collapse some needless occurrences of Suc:
 | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1111 | at least three Sucs, since two and fewer are rewritten back to Suc again! | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1112 | We already have some rules to simplify operands smaller than 3.*} | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1113 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1114 | lemma div_Suc_eq_div_add3 [simp]: "m div (Suc (Suc (Suc n))) = m div (3+n)" | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1115 | by (simp add: Suc3_eq_add_3) | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1116 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1117 | lemma mod_Suc_eq_mod_add3 [simp]: "m mod (Suc (Suc (Suc n))) = m mod (3+n)" | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1118 | by (simp add: Suc3_eq_add_3) | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1119 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1120 | lemma Suc_div_eq_add3_div: "(Suc (Suc (Suc m))) div n = (3+m) div n" | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1121 | by (simp add: Suc3_eq_add_3) | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1122 | |
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1123 | lemma Suc_mod_eq_add3_mod: "(Suc (Suc (Suc m))) mod n = (3+m) mod n" | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1124 | by (simp add: Suc3_eq_add_3) | 
| 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1125 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1126 | lemmas Suc_div_eq_add3_div_numeral [simp] = Suc_div_eq_add3_div [of _ "numeral v"] for v | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1127 | lemmas Suc_mod_eq_add3_mod_numeral [simp] = Suc_mod_eq_add3_mod [of _ "numeral v"] for v | 
| 33296 
a3924d1069e5
moved theory Divides after theory Nat_Numeral; tuned some proof texts
 haftmann parents: 
33274diff
changeset | 1128 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1129 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1130 | lemma Suc_times_mod_eq: "1<k ==> Suc (k * m) mod k = 1" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1131 | apply (induct "m") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1132 | apply (simp_all add: mod_Suc) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1133 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1134 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1135 | declare Suc_times_mod_eq [of "numeral w", simp] for w | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1136 | |
| 47138 | 1137 | lemma Suc_div_le_mono [simp]: "n div k \<le> (Suc n) div k" | 
| 1138 | by (simp add: div_le_mono) | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1139 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1140 | lemma Suc_n_div_2_gt_zero [simp]: "(0::nat) < n ==> 0 < (n + 1) div 2" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1141 | by (cases n) simp_all | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1142 | |
| 35815 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 1143 | lemma div_2_gt_zero [simp]: assumes A: "(1::nat) < n" shows "0 < n div 2" | 
| 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 1144 | proof - | 
| 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 1145 | from A have B: "0 < n - 1" and C: "n - 1 + 1 = n" by simp_all | 
| 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 1146 | from Suc_n_div_2_gt_zero [OF B] C show ?thesis by simp | 
| 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 1147 | qed | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1148 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1149 | (* Potential use of algebra : Equality modulo n*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1150 | lemma mod_mult_self3 [simp]: "(k*n + m) mod n = m mod (n::nat)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1151 | by (simp add: mult_ac add_ac) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1152 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1153 | lemma mod_mult_self4 [simp]: "Suc (k*n + m) mod n = Suc m mod n" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1154 | proof - | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1155 | have "Suc (k * n + m) mod n = (k * n + Suc m) mod n" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1156 | also have "... = Suc m mod n" by (rule mod_mult_self3) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1157 | finally show ?thesis . | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1158 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1159 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1160 | lemma mod_Suc_eq_Suc_mod: "Suc m mod n = Suc (m mod n) mod n" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1161 | apply (subst mod_Suc [of m]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1162 | apply (subst mod_Suc [of "m mod n"], simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1163 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1164 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1165 | lemma mod_2_not_eq_zero_eq_one_nat: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1166 | fixes n :: nat | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1167 | shows "n mod 2 \<noteq> 0 \<longleftrightarrow> n mod 2 = 1" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1168 | by simp | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1169 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1170 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1171 | subsection {* Division on @{typ int} *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1172 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1173 | definition divmod_int_rel :: "int \<Rightarrow> int \<Rightarrow> int \<times> int \<Rightarrow> bool" where | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1174 |     --{*definition of quotient and remainder*}
 | 
| 47139 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1175 | "divmod_int_rel a b = (\<lambda>(q, r). a = b * q + r \<and> | 
| 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1176 | (if 0 < b then 0 \<le> r \<and> r < b else if b < 0 then b < r \<and> r \<le> 0 else q = 0))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1177 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1178 | definition adjust :: "int \<Rightarrow> int \<times> int \<Rightarrow> int \<times> int" where | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1179 |     --{*for the division algorithm*}
 | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1180 | "adjust b = (\<lambda>(q, r). if 0 \<le> r - b then (2 * q + 1, r - b) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1181 | else (2 * q, r))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1182 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1183 | text{*algorithm for the case @{text "a\<ge>0, b>0"}*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1184 | function posDivAlg :: "int \<Rightarrow> int \<Rightarrow> int \<times> int" where | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1185 | "posDivAlg a b = (if a < b \<or> b \<le> 0 then (0, a) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1186 | else adjust b (posDivAlg a (2 * b)))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1187 | by auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1188 | termination by (relation "measure (\<lambda>(a, b). nat (a - b + 1))") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1189 | (auto simp add: mult_2) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1190 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1191 | text{*algorithm for the case @{text "a<0, b>0"}*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1192 | function negDivAlg :: "int \<Rightarrow> int \<Rightarrow> int \<times> int" where | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1193 | "negDivAlg a b = (if 0 \<le>a + b \<or> b \<le> 0 then (-1, a + b) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1194 | else adjust b (negDivAlg a (2 * b)))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1195 | by auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1196 | termination by (relation "measure (\<lambda>(a, b). nat (- a - b))") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1197 | (auto simp add: mult_2) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1198 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1199 | text{*algorithm for the general case @{term "b\<noteq>0"}*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1200 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1201 | definition divmod_int :: "int \<Rightarrow> int \<Rightarrow> int \<times> int" where | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1202 |     --{*The full division algorithm considers all possible signs for a, b
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1203 |        including the special case @{text "a=0, b<0"} because 
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1204 |        @{term negDivAlg} requires @{term "a<0"}.*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1205 | "divmod_int a b = (if 0 \<le> a then if 0 \<le> b then posDivAlg a b | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1206 | else if a = 0 then (0, 0) | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1207 | else apsnd uminus (negDivAlg (-a) (-b)) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1208 | else | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1209 | if 0 < b then negDivAlg a b | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1210 | else apsnd uminus (posDivAlg (-a) (-b)))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1211 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1212 | instantiation int :: Divides.div | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1213 | begin | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1214 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1215 | definition div_int where | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1216 | "a div b = fst (divmod_int a b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1217 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1218 | lemma fst_divmod_int [simp]: | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1219 | "fst (divmod_int a b) = a div b" | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1220 | by (simp add: div_int_def) | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1221 | |
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1222 | definition mod_int where | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1223 | "a mod b = snd (divmod_int a b)" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1224 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1225 | lemma snd_divmod_int [simp]: | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1226 | "snd (divmod_int a b) = a mod b" | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1227 | by (simp add: mod_int_def) | 
| 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1228 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1229 | instance .. | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1230 | |
| 3366 | 1231 | end | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1232 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1233 | lemma divmod_int_mod_div: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1234 | "divmod_int p q = (p div q, p mod q)" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1235 | by (simp add: prod_eq_iff) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1236 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1237 | text{*
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1238 | Here is the division algorithm in ML: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1239 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1240 | \begin{verbatim}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1241 | fun posDivAlg (a,b) = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1242 | if a<b then (0,a) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1243 | else let val (q,r) = posDivAlg(a, 2*b) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1244 | in if 0\<le>r-b then (2*q+1, r-b) else (2*q, r) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1245 | end | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1246 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1247 | fun negDivAlg (a,b) = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1248 | if 0\<le>a+b then (~1,a+b) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1249 | else let val (q,r) = negDivAlg(a, 2*b) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1250 | in if 0\<le>r-b then (2*q+1, r-b) else (2*q, r) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1251 | end; | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1252 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1253 | fun negateSnd (q,r:int) = (q,~r); | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1254 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1255 | fun divmod (a,b) = if 0\<le>a then | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1256 | if b>0 then posDivAlg (a,b) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1257 | else if a=0 then (0,0) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1258 | else negateSnd (negDivAlg (~a,~b)) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1259 | else | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1260 | if 0<b then negDivAlg (a,b) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1261 | else negateSnd (posDivAlg (~a,~b)); | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1262 | \end{verbatim}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1263 | *} | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1264 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1265 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1266 | subsubsection {* Uniqueness and Monotonicity of Quotients and Remainders *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1267 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1268 | lemma unique_quotient_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1269 | "[| b*q' + r' \<le> b*q + r; 0 \<le> r'; r' < b; r < b |] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1270 | ==> q' \<le> (q::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1271 | apply (subgoal_tac "r' + b * (q'-q) \<le> r") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1272 | prefer 2 apply (simp add: right_diff_distrib) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1273 | apply (subgoal_tac "0 < b * (1 + q - q') ") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1274 | apply (erule_tac [2] order_le_less_trans) | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1275 | prefer 2 apply (simp add: right_diff_distrib distrib_left) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1276 | apply (subgoal_tac "b * q' < b * (1 + q) ") | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1277 | prefer 2 apply (simp add: right_diff_distrib distrib_left) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1278 | apply (simp add: mult_less_cancel_left) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1279 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1280 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1281 | lemma unique_quotient_lemma_neg: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1282 | "[| b*q' + r' \<le> b*q + r; r \<le> 0; b < r; b < r' |] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1283 | ==> q \<le> (q'::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1284 | by (rule_tac b = "-b" and r = "-r'" and r' = "-r" in unique_quotient_lemma, | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1285 | auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1286 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1287 | lemma unique_quotient: | 
| 46552 | 1288 | "[| divmod_int_rel a b (q, r); divmod_int_rel a b (q', r') |] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1289 | ==> q = q'" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1290 | apply (simp add: divmod_int_rel_def linorder_neq_iff split: split_if_asm) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1291 | apply (blast intro: order_antisym | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1292 | dest: order_eq_refl [THEN unique_quotient_lemma] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1293 | order_eq_refl [THEN unique_quotient_lemma_neg] sym)+ | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1294 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1295 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1296 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1297 | lemma unique_remainder: | 
| 46552 | 1298 | "[| divmod_int_rel a b (q, r); divmod_int_rel a b (q', r') |] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1299 | ==> r = r'" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1300 | apply (subgoal_tac "q = q'") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1301 | apply (simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1302 | apply (blast intro: unique_quotient) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1303 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1304 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1305 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1306 | subsubsection {* Correctness of @{term posDivAlg}, the Algorithm for Non-Negative Dividends *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1307 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1308 | text{*And positive divisors*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1309 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1310 | lemma adjust_eq [simp]: | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1311 | "adjust b (q, r) = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1312 | (let diff = r - b in | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1313 | if 0 \<le> diff then (2 * q + 1, diff) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1314 | else (2*q, r))" | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1315 | by (simp add: Let_def adjust_def) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1316 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1317 | declare posDivAlg.simps [simp del] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1318 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1319 | text{*use with a simproc to avoid repeatedly proving the premise*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1320 | lemma posDivAlg_eqn: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1321 | "0 < b ==> | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1322 | posDivAlg a b = (if a<b then (0,a) else adjust b (posDivAlg a (2*b)))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1323 | by (rule posDivAlg.simps [THEN trans], simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1324 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1325 | text{*Correctness of @{term posDivAlg}: it computes quotients correctly*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1326 | theorem posDivAlg_correct: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1327 | assumes "0 \<le> a" and "0 < b" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1328 | shows "divmod_int_rel a b (posDivAlg a b)" | 
| 41550 | 1329 | using assms | 
| 1330 | apply (induct a b rule: posDivAlg.induct) | |
| 1331 | apply auto | |
| 1332 | apply (simp add: divmod_int_rel_def) | |
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1333 | apply (subst posDivAlg_eqn, simp add: distrib_left) | 
| 41550 | 1334 | apply (case_tac "a < b") | 
| 1335 | apply simp_all | |
| 1336 | apply (erule splitE) | |
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1337 | apply (auto simp add: distrib_left Let_def mult_ac mult_2_right) | 
| 41550 | 1338 | done | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1339 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1340 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1341 | subsubsection {* Correctness of @{term negDivAlg}, the Algorithm for Negative Dividends *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1342 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1343 | text{*And positive divisors*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1344 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1345 | declare negDivAlg.simps [simp del] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1346 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1347 | text{*use with a simproc to avoid repeatedly proving the premise*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1348 | lemma negDivAlg_eqn: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1349 | "0 < b ==> | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1350 | negDivAlg a b = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1351 | (if 0\<le>a+b then (-1,a+b) else adjust b (negDivAlg a (2*b)))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1352 | by (rule negDivAlg.simps [THEN trans], simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1353 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1354 | (*Correctness of negDivAlg: it computes quotients correctly | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1355 | It doesn't work if a=0 because the 0/b equals 0, not -1*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1356 | lemma negDivAlg_correct: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1357 | assumes "a < 0" and "b > 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1358 | shows "divmod_int_rel a b (negDivAlg a b)" | 
| 41550 | 1359 | using assms | 
| 1360 | apply (induct a b rule: negDivAlg.induct) | |
| 1361 | apply (auto simp add: linorder_not_le) | |
| 1362 | apply (simp add: divmod_int_rel_def) | |
| 1363 | apply (subst negDivAlg_eqn, assumption) | |
| 1364 | apply (case_tac "a + b < (0\<Colon>int)") | |
| 1365 | apply simp_all | |
| 1366 | apply (erule splitE) | |
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1367 | apply (auto simp add: distrib_left Let_def mult_ac mult_2_right) | 
| 41550 | 1368 | done | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1369 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1370 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1371 | subsubsection {* Existence Shown by Proving the Division Algorithm to be Correct *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1372 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1373 | (*the case a=0*) | 
| 47139 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1374 | lemma divmod_int_rel_0: "divmod_int_rel 0 b (0, 0)" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1375 | by (auto simp add: divmod_int_rel_def linorder_neq_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1376 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1377 | lemma posDivAlg_0 [simp]: "posDivAlg 0 b = (0, 0)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1378 | by (subst posDivAlg.simps, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1379 | |
| 47139 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1380 | lemma posDivAlg_0_right [simp]: "posDivAlg a 0 = (0, a)" | 
| 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1381 | by (subst posDivAlg.simps, auto) | 
| 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1382 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1383 | lemma negDivAlg_minus1 [simp]: "negDivAlg -1 b = (-1, b - 1)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1384 | by (subst negDivAlg.simps, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1385 | |
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1386 | lemma divmod_int_rel_neg: "divmod_int_rel (-a) (-b) qr ==> divmod_int_rel a b (apsnd uminus qr)" | 
| 47139 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1387 | by (auto simp add: divmod_int_rel_def) | 
| 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1388 | |
| 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1389 | lemma divmod_int_correct: "divmod_int_rel a b (divmod_int a b)" | 
| 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1390 | apply (cases "b = 0", simp add: divmod_int_def divmod_int_rel_def) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1391 | by (force simp add: linorder_neq_iff divmod_int_rel_0 divmod_int_def divmod_int_rel_neg | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1392 | posDivAlg_correct negDivAlg_correct) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1393 | |
| 47141 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1394 | lemma divmod_int_unique: | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1395 | assumes "divmod_int_rel a b qr" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1396 | shows "divmod_int a b = qr" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1397 | using assms divmod_int_correct [of a b] | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1398 | using unique_quotient [of a b] unique_remainder [of a b] | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1399 | by (metis pair_collapse) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1400 | |
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1401 | lemma divmod_int_rel_div_mod: "divmod_int_rel a b (a div b, a mod b)" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1402 | using divmod_int_correct by (simp add: divmod_int_mod_div) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1403 | |
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1404 | lemma div_int_unique: "divmod_int_rel a b (q, r) \<Longrightarrow> a div b = q" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1405 | by (simp add: divmod_int_rel_div_mod [THEN unique_quotient]) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1406 | |
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1407 | lemma mod_int_unique: "divmod_int_rel a b (q, r) \<Longrightarrow> a mod b = r" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1408 | by (simp add: divmod_int_rel_div_mod [THEN unique_remainder]) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1409 | |
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1410 | instance int :: ring_div | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1411 | proof | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1412 | fix a b :: int | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1413 | show "a div b * b + a mod b = a" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1414 | using divmod_int_rel_div_mod [of a b] | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1415 | unfolding divmod_int_rel_def by (simp add: mult_commute) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1416 | next | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1417 | fix a b c :: int | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1418 | assume "b \<noteq> 0" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1419 | hence "divmod_int_rel (a + c * b) b (c + a div b, a mod b)" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1420 | using divmod_int_rel_div_mod [of a b] | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1421 | unfolding divmod_int_rel_def by (auto simp: algebra_simps) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1422 | thus "(a + c * b) div b = c + a div b" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1423 | by (rule div_int_unique) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1424 | next | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1425 | fix a b c :: int | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1426 | assume "c \<noteq> 0" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1427 | hence "\<And>q r. divmod_int_rel a b (q, r) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1428 | \<Longrightarrow> divmod_int_rel (c * a) (c * b) (q, c * r)" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1429 | unfolding divmod_int_rel_def | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1430 | by - (rule linorder_cases [of 0 b], auto simp: algebra_simps | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1431 | mult_less_0_iff zero_less_mult_iff mult_strict_right_mono | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1432 | mult_strict_right_mono_neg zero_le_mult_iff mult_le_0_iff) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1433 | hence "divmod_int_rel (c * a) (c * b) (a div b, c * (a mod b))" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1434 | using divmod_int_rel_div_mod [of a b] . | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1435 | thus "(c * a) div (c * b) = a div b" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1436 | by (rule div_int_unique) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1437 | next | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1438 | fix a :: int show "a div 0 = 0" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1439 | by (rule div_int_unique, simp add: divmod_int_rel_def) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1440 | next | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1441 | fix a :: int show "0 div a = 0" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1442 | by (rule div_int_unique, auto simp add: divmod_int_rel_def) | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1443 | qed | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1444 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1445 | text{*Basic laws about division and remainder*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1446 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1447 | lemma zmod_zdiv_equality: "(a::int) = b * (a div b) + (a mod b)" | 
| 47141 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1448 | by (fact mod_div_equality2 [symmetric]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1449 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1450 | text {* Tool setup *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1451 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1452 | (* FIXME: Theorem list add_0s doesn't exist, because Numeral0 has gone. *) | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1453 | lemmas add_0s = add_0_left add_0_right | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1454 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1455 | ML {*
 | 
| 43594 | 1456 | structure Cancel_Div_Mod_Int = Cancel_Div_Mod | 
| 41550 | 1457 | ( | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1458 |   val div_name = @{const_name div};
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1459 |   val mod_name = @{const_name mod};
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1460 | val mk_binop = HOLogic.mk_binop; | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1461 | val mk_sum = Arith_Data.mk_sum HOLogic.intT; | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1462 | val dest_sum = Arith_Data.dest_sum; | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1463 | |
| 47165 | 1464 |   val div_mod_eqs = map mk_meta_eq [@{thm div_mod_equality}, @{thm div_mod_equality2}];
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1465 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1466 | val prove_eq_sums = Arith_Data.prove_conv2 all_tac (Arith_Data.simp_all_tac | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1467 |     (@{thm diff_minus} :: @{thms add_0s} @ @{thms add_ac}))
 | 
| 41550 | 1468 | ) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1469 | *} | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1470 | |
| 43594 | 1471 | simproc_setup cancel_div_mod_int ("(k::int) + l") = {* K Cancel_Div_Mod_Int.proc *}
 | 
| 1472 | ||
| 47141 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1473 | lemma pos_mod_conj: "(0::int) < b \<Longrightarrow> 0 \<le> a mod b \<and> a mod b < b" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1474 | using divmod_int_correct [of a b] | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1475 | by (auto simp add: divmod_int_rel_def prod_eq_iff) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1476 | |
| 45607 | 1477 | lemmas pos_mod_sign [simp] = pos_mod_conj [THEN conjunct1] | 
| 1478 | and pos_mod_bound [simp] = pos_mod_conj [THEN conjunct2] | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1479 | |
| 47141 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1480 | lemma neg_mod_conj: "b < (0::int) \<Longrightarrow> a mod b \<le> 0 \<and> b < a mod b" | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1481 | using divmod_int_correct [of a b] | 
| 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1482 | by (auto simp add: divmod_int_rel_def prod_eq_iff) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1483 | |
| 45607 | 1484 | lemmas neg_mod_sign [simp] = neg_mod_conj [THEN conjunct1] | 
| 1485 | and neg_mod_bound [simp] = neg_mod_conj [THEN conjunct2] | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1486 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1487 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1488 | subsubsection {* General Properties of div and mod *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1489 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1490 | lemma div_pos_pos_trivial: "[| (0::int) \<le> a; a < b |] ==> a div b = 0" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1491 | apply (rule div_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1492 | apply (auto simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1493 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1494 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1495 | lemma div_neg_neg_trivial: "[| a \<le> (0::int); b < a |] ==> a div b = 0" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1496 | apply (rule div_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1497 | apply (auto simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1498 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1499 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1500 | lemma div_pos_neg_trivial: "[| (0::int) < a; a+b \<le> 0 |] ==> a div b = -1" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1501 | apply (rule div_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1502 | apply (auto simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1503 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1504 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1505 | (*There is no div_neg_pos_trivial because 0 div b = 0 would supersede it*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1506 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1507 | lemma mod_pos_pos_trivial: "[| (0::int) \<le> a; a < b |] ==> a mod b = a" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1508 | apply (rule_tac q = 0 in mod_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1509 | apply (auto simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1510 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1511 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1512 | lemma mod_neg_neg_trivial: "[| a \<le> (0::int); b < a |] ==> a mod b = a" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1513 | apply (rule_tac q = 0 in mod_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1514 | apply (auto simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1515 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1516 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1517 | lemma mod_pos_neg_trivial: "[| (0::int) < a; a+b \<le> 0 |] ==> a mod b = a+b" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1518 | apply (rule_tac q = "-1" in mod_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1519 | apply (auto simp add: divmod_int_rel_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1520 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1521 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1522 | text{*There is no @{text mod_neg_pos_trivial}.*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1523 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1524 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1525 | subsubsection {* Laws for div and mod with Unary Minus *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1526 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1527 | lemma zminus1_lemma: | 
| 47139 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1528 | "divmod_int_rel a b (q, r) ==> b \<noteq> 0 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1529 | ==> divmod_int_rel (-a) b (if r=0 then -q else -q - 1, | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1530 | if r=0 then 0 else b-r)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1531 | by (force simp add: split_ifs divmod_int_rel_def linorder_neq_iff right_diff_distrib) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1532 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1533 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1534 | lemma zdiv_zminus1_eq_if: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1535 | "b \<noteq> (0::int) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1536 | ==> (-a) div b = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1537 | (if a mod b = 0 then - (a div b) else - (a div b) - 1)" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1538 | by (blast intro: divmod_int_rel_div_mod [THEN zminus1_lemma, THEN div_int_unique]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1539 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1540 | lemma zmod_zminus1_eq_if: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1541 | "(-a::int) mod b = (if a mod b = 0 then 0 else b - (a mod b))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1542 | apply (case_tac "b = 0", simp) | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1543 | apply (blast intro: divmod_int_rel_div_mod [THEN zminus1_lemma, THEN mod_int_unique]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1544 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1545 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1546 | lemma zmod_zminus1_not_zero: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1547 | fixes k l :: int | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1548 | shows "- k mod l \<noteq> 0 \<Longrightarrow> k mod l \<noteq> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1549 | unfolding zmod_zminus1_eq_if by auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1550 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1551 | lemma zdiv_zminus2_eq_if: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1552 | "b \<noteq> (0::int) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1553 | ==> a div (-b) = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1554 | (if a mod b = 0 then - (a div b) else - (a div b) - 1)" | 
| 47159 | 1555 | by (simp add: zdiv_zminus1_eq_if div_minus_right) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1556 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1557 | lemma zmod_zminus2_eq_if: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1558 | "a mod (-b::int) = (if a mod b = 0 then 0 else (a mod b) - b)" | 
| 47159 | 1559 | by (simp add: zmod_zminus1_eq_if mod_minus_right) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1560 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1561 | lemma zmod_zminus2_not_zero: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1562 | fixes k l :: int | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1563 | shows "k mod - l \<noteq> 0 \<Longrightarrow> k mod l \<noteq> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1564 | unfolding zmod_zminus2_eq_if by auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1565 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1566 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1567 | subsubsection {* Computation of Division and Remainder *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1568 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1569 | lemma div_eq_minus1: "(0::int) < b ==> -1 div b = -1" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1570 | by (simp add: div_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1571 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1572 | lemma zmod_minus1: "(0::int) < b ==> -1 mod b = b - 1" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1573 | by (simp add: mod_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1574 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1575 | text{*a positive, b positive *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1576 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1577 | lemma div_pos_pos: "[| 0 < a; 0 \<le> b |] ==> a div b = fst (posDivAlg a b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1578 | by (simp add: div_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1579 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1580 | lemma mod_pos_pos: "[| 0 < a; 0 \<le> b |] ==> a mod b = snd (posDivAlg a b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1581 | by (simp add: mod_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1582 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1583 | text{*a negative, b positive *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1584 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1585 | lemma div_neg_pos: "[| a < 0; 0 < b |] ==> a div b = fst (negDivAlg a b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1586 | by (simp add: div_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1587 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1588 | lemma mod_neg_pos: "[| a < 0; 0 < b |] ==> a mod b = snd (negDivAlg a b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1589 | by (simp add: mod_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1590 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1591 | text{*a positive, b negative *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1592 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1593 | lemma div_pos_neg: | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1594 | "[| 0 < a; b < 0 |] ==> a div b = fst (apsnd uminus (negDivAlg (-a) (-b)))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1595 | by (simp add: div_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1596 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1597 | lemma mod_pos_neg: | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1598 | "[| 0 < a; b < 0 |] ==> a mod b = snd (apsnd uminus (negDivAlg (-a) (-b)))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1599 | by (simp add: mod_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1600 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1601 | text{*a negative, b negative *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1602 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1603 | lemma div_neg_neg: | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1604 | "[| a < 0; b \<le> 0 |] ==> a div b = fst (apsnd uminus (posDivAlg (-a) (-b)))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1605 | by (simp add: div_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1606 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1607 | lemma mod_neg_neg: | 
| 46560 
8e252a608765
remove constant negateSnd in favor of 'apsnd uminus' (from Florian Haftmann)
 huffman parents: 
46552diff
changeset | 1608 | "[| a < 0; b \<le> 0 |] ==> a mod b = snd (apsnd uminus (posDivAlg (-a) (-b)))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1609 | by (simp add: mod_int_def divmod_int_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1610 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1611 | text {*Simplify expresions in which div and mod combine numerical constants*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1612 | |
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1613 | lemma int_div_pos_eq: "\<lbrakk>(a::int) = b * q + r; 0 \<le> r; r < b\<rbrakk> \<Longrightarrow> a div b = q" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1614 | by (rule div_int_unique [of a b q r]) (simp add: divmod_int_rel_def) | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1615 | |
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1616 | lemma int_div_neg_eq: "\<lbrakk>(a::int) = b * q + r; r \<le> 0; b < r\<rbrakk> \<Longrightarrow> a div b = q" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1617 | by (rule div_int_unique [of a b q r], | 
| 46552 | 1618 | simp add: divmod_int_rel_def) | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1619 | |
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1620 | lemma int_mod_pos_eq: "\<lbrakk>(a::int) = b * q + r; 0 \<le> r; r < b\<rbrakk> \<Longrightarrow> a mod b = r" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1621 | by (rule mod_int_unique [of a b q r], | 
| 46552 | 1622 | simp add: divmod_int_rel_def) | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1623 | |
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1624 | lemma int_mod_neg_eq: "\<lbrakk>(a::int) = b * q + r; r \<le> 0; b < r\<rbrakk> \<Longrightarrow> a mod b = r" | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1625 | by (rule mod_int_unique [of a b q r], | 
| 46552 | 1626 | simp add: divmod_int_rel_def) | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1627 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1628 | (* simprocs adapted from HOL/ex/Binary.thy *) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1629 | ML {*
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1630 | local | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1631 | val mk_number = HOLogic.mk_number HOLogic.intT | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1632 |   val plus = @{term "plus :: int \<Rightarrow> int \<Rightarrow> int"}
 | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1633 |   val times = @{term "times :: int \<Rightarrow> int \<Rightarrow> int"}
 | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1634 |   val zero = @{term "0 :: int"}
 | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1635 |   val less = @{term "op < :: int \<Rightarrow> int \<Rightarrow> bool"}
 | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1636 |   val le = @{term "op \<le> :: int \<Rightarrow> int \<Rightarrow> bool"}
 | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1637 |   val simps = @{thms arith_simps} @ @{thms rel_simps} @
 | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1638 |     map (fn th => th RS sym) [@{thm numeral_1_eq_1}]
 | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1639 | fun prove ctxt goal = Goal.prove ctxt [] [] (HOLogic.mk_Trueprop goal) | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1640 | (K (ALLGOALS (full_simp_tac (HOL_basic_ss addsimps simps)))); | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1641 | fun binary_proc proc ss ct = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1642 | (case Thm.term_of ct of | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1643 | _ $ t $ u => | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1644 | (case try (pairself (`(snd o HOLogic.dest_number))) (t, u) of | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1645 | SOME args => proc (Simplifier.the_context ss) args | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1646 | | NONE => NONE) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1647 | | _ => NONE); | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1648 | in | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1649 | fun divmod_proc posrule negrule = | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1650 | binary_proc (fn ctxt => fn ((a, t), (b, u)) => | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1651 | if b = 0 then NONE else let | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1652 | val (q, r) = pairself mk_number (Integer.div_mod a b) | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1653 | val goal1 = HOLogic.mk_eq (t, plus $ (times $ u $ q) $ r) | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1654 | val (goal2, goal3, rule) = if b > 0 | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1655 | then (le $ zero $ r, less $ r $ u, posrule RS eq_reflection) | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1656 | else (le $ r $ zero, less $ u $ r, negrule RS eq_reflection) | 
| 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1657 | in SOME (rule OF map (prove ctxt) [goal1, goal2, goal3]) end) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1658 | end | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1659 | *} | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1660 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1661 | simproc_setup binary_int_div | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1662 |   ("numeral m div numeral n :: int" |
 | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1663 | "numeral m div neg_numeral n :: int" | | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1664 | "neg_numeral m div numeral n :: int" | | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1665 | "neg_numeral m div neg_numeral n :: int") = | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1666 |   {* K (divmod_proc @{thm int_div_pos_eq} @{thm int_div_neg_eq}) *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1667 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1668 | simproc_setup binary_int_mod | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1669 |   ("numeral m mod numeral n :: int" |
 | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1670 | "numeral m mod neg_numeral n :: int" | | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1671 | "neg_numeral m mod numeral n :: int" | | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1672 | "neg_numeral m mod neg_numeral n :: int") = | 
| 45530 
0c4853bb77bf
rewrite integer numeral div/mod simprocs to not return conditional rewrites; add regression tests
 huffman parents: 
45231diff
changeset | 1673 |   {* K (divmod_proc @{thm int_mod_pos_eq} @{thm int_mod_neg_eq}) *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1674 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1675 | lemmas posDivAlg_eqn_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1676 | posDivAlg_eqn [of "numeral v" "numeral w", OF zero_less_numeral] for v w | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1677 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1678 | lemmas negDivAlg_eqn_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1679 | negDivAlg_eqn [of "numeral v" "neg_numeral w", OF zero_less_numeral] for v w | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1680 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1681 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1682 | text{*Special-case simplification *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1683 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1684 | (** The last remaining special cases for constant arithmetic: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1685 | 1 div z and 1 mod z **) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1686 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1687 | lemmas div_pos_pos_1_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1688 | div_pos_pos [OF zero_less_one, of "numeral w", OF zero_le_numeral] for w | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1689 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1690 | lemmas div_pos_neg_1_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1691 | div_pos_neg [OF zero_less_one, of "neg_numeral w", | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1692 | OF neg_numeral_less_zero] for w | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1693 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1694 | lemmas mod_pos_pos_1_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1695 | mod_pos_pos [OF zero_less_one, of "numeral w", OF zero_le_numeral] for w | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1696 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1697 | lemmas mod_pos_neg_1_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1698 | mod_pos_neg [OF zero_less_one, of "neg_numeral w", | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1699 | OF neg_numeral_less_zero] for w | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1700 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1701 | lemmas posDivAlg_eqn_1_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1702 | posDivAlg_eqn [of concl: 1 "numeral w", OF zero_less_numeral] for w | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1703 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1704 | lemmas negDivAlg_eqn_1_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1705 | negDivAlg_eqn [of concl: 1 "numeral w", OF zero_less_numeral] for w | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1706 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1707 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1708 | subsubsection {* Monotonicity in the First Argument (Dividend) *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1709 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1710 | lemma zdiv_mono1: "[| a \<le> a'; 0 < (b::int) |] ==> a div b \<le> a' div b" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1711 | apply (cut_tac a = a and b = b in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1712 | apply (cut_tac a = a' and b = b in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1713 | apply (rule unique_quotient_lemma) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1714 | apply (erule subst) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1715 | apply (erule subst, simp_all) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1716 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1717 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1718 | lemma zdiv_mono1_neg: "[| a \<le> a'; (b::int) < 0 |] ==> a' div b \<le> a div b" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1719 | apply (cut_tac a = a and b = b in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1720 | apply (cut_tac a = a' and b = b in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1721 | apply (rule unique_quotient_lemma_neg) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1722 | apply (erule subst) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1723 | apply (erule subst, simp_all) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1724 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1725 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1726 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1727 | subsubsection {* Monotonicity in the Second Argument (Divisor) *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1728 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1729 | lemma q_pos_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1730 | "[| 0 \<le> b'*q' + r'; r' < b'; 0 < b' |] ==> 0 \<le> (q'::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1731 | apply (subgoal_tac "0 < b'* (q' + 1) ") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1732 | apply (simp add: zero_less_mult_iff) | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1733 | apply (simp add: distrib_left) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1734 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1735 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1736 | lemma zdiv_mono2_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1737 | "[| b*q + r = b'*q' + r'; 0 \<le> b'*q' + r'; | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1738 | r' < b'; 0 \<le> r; 0 < b'; b' \<le> b |] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1739 | ==> q \<le> (q'::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1740 | apply (frule q_pos_lemma, assumption+) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1741 | apply (subgoal_tac "b*q < b* (q' + 1) ") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1742 | apply (simp add: mult_less_cancel_left) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1743 | apply (subgoal_tac "b*q = r' - r + b'*q'") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1744 | prefer 2 apply simp | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1745 | apply (simp (no_asm_simp) add: distrib_left) | 
| 44766 | 1746 | apply (subst add_commute, rule add_less_le_mono, arith) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1747 | apply (rule mult_right_mono, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1748 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1749 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1750 | lemma zdiv_mono2: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1751 | "[| (0::int) \<le> a; 0 < b'; b' \<le> b |] ==> a div b \<le> a div b'" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1752 | apply (subgoal_tac "b \<noteq> 0") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1753 | prefer 2 apply arith | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1754 | apply (cut_tac a = a and b = b in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1755 | apply (cut_tac a = a and b = b' in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1756 | apply (rule zdiv_mono2_lemma) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1757 | apply (erule subst) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1758 | apply (erule subst, simp_all) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1759 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1760 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1761 | lemma q_neg_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1762 | "[| b'*q' + r' < 0; 0 \<le> r'; 0 < b' |] ==> q' \<le> (0::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1763 | apply (subgoal_tac "b'*q' < 0") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1764 | apply (simp add: mult_less_0_iff, arith) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1765 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1766 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1767 | lemma zdiv_mono2_neg_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1768 | "[| b*q + r = b'*q' + r'; b'*q' + r' < 0; | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1769 | r < b; 0 \<le> r'; 0 < b'; b' \<le> b |] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1770 | ==> q' \<le> (q::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1771 | apply (frule q_neg_lemma, assumption+) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1772 | apply (subgoal_tac "b*q' < b* (q + 1) ") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1773 | apply (simp add: mult_less_cancel_left) | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1774 | apply (simp add: distrib_left) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1775 | apply (subgoal_tac "b*q' \<le> b'*q'") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1776 | prefer 2 apply (simp add: mult_right_mono_neg, arith) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1777 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1778 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1779 | lemma zdiv_mono2_neg: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1780 | "[| a < (0::int); 0 < b'; b' \<le> b |] ==> a div b' \<le> a div b" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1781 | apply (cut_tac a = a and b = b in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1782 | apply (cut_tac a = a and b = b' in zmod_zdiv_equality) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1783 | apply (rule zdiv_mono2_neg_lemma) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1784 | apply (erule subst) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1785 | apply (erule subst, simp_all) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1786 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1787 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1788 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1789 | subsubsection {* More Algebraic Laws for div and mod *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1790 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1791 | text{*proving (a*b) div c = a * (b div c) + a * (b mod c) *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1792 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1793 | lemma zmult1_lemma: | 
| 46552 | 1794 | "[| divmod_int_rel b c (q, r) |] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1795 | ==> divmod_int_rel (a * b) c (a*q + a*r div c, a*r mod c)" | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1796 | by (auto simp add: split_ifs divmod_int_rel_def linorder_neq_iff distrib_left mult_ac) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1797 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1798 | lemma zdiv_zmult1_eq: "(a*b) div c = a*(b div c) + a*(b mod c) div (c::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1799 | apply (case_tac "c = 0", simp) | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1800 | apply (blast intro: divmod_int_rel_div_mod [THEN zmult1_lemma, THEN div_int_unique]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1801 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1802 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1803 | text{*proving (a+b) div c = a div c + b div c + ((a mod c + b mod c) div c) *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1804 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1805 | lemma zadd1_lemma: | 
| 46552 | 1806 | "[| divmod_int_rel a c (aq, ar); divmod_int_rel b c (bq, br) |] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1807 | ==> divmod_int_rel (a+b) c (aq + bq + (ar+br) div c, (ar+br) mod c)" | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1808 | by (force simp add: split_ifs divmod_int_rel_def linorder_neq_iff distrib_left) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1809 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1810 | (*NOT suitable for rewriting: the RHS has an instance of the LHS*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1811 | lemma zdiv_zadd1_eq: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1812 | "(a+b) div (c::int) = a div c + b div c + ((a mod c + b mod c) div c)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1813 | apply (case_tac "c = 0", simp) | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1814 | apply (blast intro: zadd1_lemma [OF divmod_int_rel_div_mod divmod_int_rel_div_mod] div_int_unique) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1815 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1816 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1817 | lemma posDivAlg_div_mod: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1818 | assumes "k \<ge> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1819 | and "l \<ge> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1820 | shows "posDivAlg k l = (k div l, k mod l)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1821 | proof (cases "l = 0") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1822 | case True then show ?thesis by (simp add: posDivAlg.simps) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1823 | next | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1824 | case False with assms posDivAlg_correct | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1825 | have "divmod_int_rel k l (fst (posDivAlg k l), snd (posDivAlg k l))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1826 | by simp | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1827 | from div_int_unique [OF this] mod_int_unique [OF this] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1828 | show ?thesis by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1829 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1830 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1831 | lemma negDivAlg_div_mod: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1832 | assumes "k < 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1833 | and "l > 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1834 | shows "negDivAlg k l = (k div l, k mod l)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1835 | proof - | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1836 | from assms have "l \<noteq> 0" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1837 | from assms negDivAlg_correct | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1838 | have "divmod_int_rel k l (fst (negDivAlg k l), snd (negDivAlg k l))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1839 | by simp | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1840 | from div_int_unique [OF this] mod_int_unique [OF this] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1841 | show ?thesis by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1842 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1843 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1844 | lemma zmod_eq_0_iff: "(m mod d = 0) = (EX q::int. m = d*q)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1845 | by (simp add: dvd_eq_mod_eq_0 [symmetric] dvd_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1846 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1847 | (* REVISIT: should this be generalized to all semiring_div types? *) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1848 | lemmas zmod_eq_0D [dest!] = zmod_eq_0_iff [THEN iffD1] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1849 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1850 | lemma zmod_zdiv_equality': | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1851 | "(m\<Colon>int) mod n = m - (m div n) * n" | 
| 47141 
02d6b816e4b3
move int::ring_div instance upward, simplify several proofs
 huffman parents: 
47140diff
changeset | 1852 | using mod_div_equality [of m n] by arith | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1853 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1854 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1855 | subsubsection {* Proving  @{term "a div (b*c) = (a div b) div c"} *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1856 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1857 | (*The condition c>0 seems necessary. Consider that 7 div ~6 = ~2 but | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1858 | 7 div 2 div ~3 = 3 div ~3 = ~1. The subcase (a div b) mod c = 0 seems | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1859 | to cause particular problems.*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1860 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1861 | text{*first, four lemmas to bound the remainder for the cases b<0 and b>0 *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1862 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1863 | lemma zmult2_lemma_aux1: "[| (0::int) < c; b < r; r \<le> 0 |] ==> b*c < b*(q mod c) + r" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1864 | apply (subgoal_tac "b * (c - q mod c) < r * 1") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1865 | apply (simp add: algebra_simps) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1866 | apply (rule order_le_less_trans) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1867 | apply (erule_tac [2] mult_strict_right_mono) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1868 | apply (rule mult_left_mono_neg) | 
| 35216 | 1869 | using add1_zle_eq[of "q mod c"]apply(simp add: algebra_simps) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1870 | apply (simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1871 | apply (simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1872 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1873 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1874 | lemma zmult2_lemma_aux2: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1875 | "[| (0::int) < c; b < r; r \<le> 0 |] ==> b * (q mod c) + r \<le> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1876 | apply (subgoal_tac "b * (q mod c) \<le> 0") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1877 | apply arith | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1878 | apply (simp add: mult_le_0_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1879 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1880 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1881 | lemma zmult2_lemma_aux3: "[| (0::int) < c; 0 \<le> r; r < b |] ==> 0 \<le> b * (q mod c) + r" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1882 | apply (subgoal_tac "0 \<le> b * (q mod c) ") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1883 | apply arith | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1884 | apply (simp add: zero_le_mult_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1885 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1886 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1887 | lemma zmult2_lemma_aux4: "[| (0::int) < c; 0 \<le> r; r < b |] ==> b * (q mod c) + r < b * c" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1888 | apply (subgoal_tac "r * 1 < b * (c - q mod c) ") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1889 | apply (simp add: right_diff_distrib) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1890 | apply (rule order_less_le_trans) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1891 | apply (erule mult_strict_right_mono) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1892 | apply (rule_tac [2] mult_left_mono) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1893 | apply simp | 
| 35216 | 1894 | using add1_zle_eq[of "q mod c"] apply (simp add: algebra_simps) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1895 | apply simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1896 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1897 | |
| 46552 | 1898 | lemma zmult2_lemma: "[| divmod_int_rel a b (q, r); 0 < c |] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1899 | ==> divmod_int_rel a (b * c) (q div c, b*(q mod c) + r)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1900 | by (auto simp add: mult_ac divmod_int_rel_def linorder_neq_iff | 
| 49962 
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
 webertj parents: 
48891diff
changeset | 1901 | zero_less_mult_iff distrib_left [symmetric] | 
| 47139 
98bddfa0f717
extend definition of divmod_int_rel to handle denominator=0 case
 huffman parents: 
47138diff
changeset | 1902 | zmult2_lemma_aux1 zmult2_lemma_aux2 zmult2_lemma_aux3 zmult2_lemma_aux4 mult_less_0_iff split: split_if_asm) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1903 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1904 | lemma zdiv_zmult2_eq: "(0::int) < c ==> a div (b*c) = (a div b) div c" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1905 | apply (case_tac "b = 0", simp) | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1906 | apply (force simp add: divmod_int_rel_div_mod [THEN zmult2_lemma, THEN div_int_unique]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1907 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1908 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1909 | lemma zmod_zmult2_eq: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1910 | "(0::int) < c ==> a mod (b*c) = b*(a div b mod c) + a mod b" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1911 | apply (case_tac "b = 0", simp) | 
| 47140 
97c3676c5c94
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
 huffman parents: 
47139diff
changeset | 1912 | apply (force simp add: divmod_int_rel_div_mod [THEN zmult2_lemma, THEN mod_int_unique]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1913 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1914 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1915 | lemma div_pos_geq: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1916 | fixes k l :: int | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1917 | assumes "0 < l" and "l \<le> k" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1918 | shows "k div l = (k - l) div l + 1" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1919 | proof - | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1920 | have "k = (k - l) + l" by simp | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1921 | then obtain j where k: "k = j + l" .. | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1922 | with assms show ?thesis by simp | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1923 | qed | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1924 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1925 | lemma mod_pos_geq: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1926 | fixes k l :: int | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1927 | assumes "0 < l" and "l \<le> k" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1928 | shows "k mod l = (k - l) mod l" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1929 | proof - | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1930 | have "k = (k - l) + l" by simp | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1931 | then obtain j where k: "k = j + l" .. | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1932 | with assms show ?thesis by simp | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1933 | qed | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1934 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1935 | |
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 1936 | subsubsection {* Splitting Rules for div and mod *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1937 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1938 | text{*The proofs of the two lemmas below are essentially identical*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1939 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1940 | lemma split_pos_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1941 | "0<k ==> | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1942 | P(n div k :: int)(n mod k) = (\<forall>i j. 0\<le>j & j<k & n = k*i + j --> P i j)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1943 | apply (rule iffI, clarify) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1944 | apply (erule_tac P="P ?x ?y" in rev_mp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1945 | apply (subst mod_add_eq) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1946 | apply (subst zdiv_zadd1_eq) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1947 | apply (simp add: div_pos_pos_trivial mod_pos_pos_trivial) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1948 | txt{*converse direction*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1949 | apply (drule_tac x = "n div k" in spec) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1950 | apply (drule_tac x = "n mod k" in spec, simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1951 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1952 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1953 | lemma split_neg_lemma: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1954 | "k<0 ==> | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1955 | P(n div k :: int)(n mod k) = (\<forall>i j. k<j & j\<le>0 & n = k*i + j --> P i j)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1956 | apply (rule iffI, clarify) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1957 | apply (erule_tac P="P ?x ?y" in rev_mp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1958 | apply (subst mod_add_eq) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1959 | apply (subst zdiv_zadd1_eq) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1960 | apply (simp add: div_neg_neg_trivial mod_neg_neg_trivial) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1961 | txt{*converse direction*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1962 | apply (drule_tac x = "n div k" in spec) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1963 | apply (drule_tac x = "n mod k" in spec, simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1964 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1965 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1966 | lemma split_zdiv: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1967 | "P(n div k :: int) = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1968 | ((k = 0 --> P 0) & | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1969 | (0<k --> (\<forall>i j. 0\<le>j & j<k & n = k*i + j --> P i)) & | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1970 | (k<0 --> (\<forall>i j. k<j & j\<le>0 & n = k*i + j --> P i)))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1971 | apply (case_tac "k=0", simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1972 | apply (simp only: linorder_neq_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1973 | apply (erule disjE) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1974 | apply (simp_all add: split_pos_lemma [of concl: "%x y. P x"] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1975 | split_neg_lemma [of concl: "%x y. P x"]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1976 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1977 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1978 | lemma split_zmod: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1979 | "P(n mod k :: int) = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1980 | ((k = 0 --> P n) & | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1981 | (0<k --> (\<forall>i j. 0\<le>j & j<k & n = k*i + j --> P j)) & | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1982 | (k<0 --> (\<forall>i j. k<j & j\<le>0 & n = k*i + j --> P j)))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1983 | apply (case_tac "k=0", simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1984 | apply (simp only: linorder_neq_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1985 | apply (erule disjE) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1986 | apply (simp_all add: split_pos_lemma [of concl: "%x y. P y"] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1987 | split_neg_lemma [of concl: "%x y. P y"]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1988 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1989 | |
| 33730 
1755ca4ec022
Fixed splitting of div and mod on integers (split theorem differed from implementation).
 webertj parents: 
33728diff
changeset | 1990 | text {* Enable (lin)arith to deal with @{const div} and @{const mod}
 | 
| 
1755ca4ec022
Fixed splitting of div and mod on integers (split theorem differed from implementation).
 webertj parents: 
33728diff
changeset | 1991 | when these are applied to some constant that is of the form | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1992 |   @{term "numeral k"}: *}
 | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1993 | declare split_zdiv [of _ _ "numeral k", arith_split] for k | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 1994 | declare split_zmod [of _ _ "numeral k", arith_split] for k | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1995 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 1996 | |
| 47166 | 1997 | subsubsection {* Computing @{text "div"} and @{text "mod"} with shifting *}
 | 
| 1998 | ||
| 1999 | lemma pos_divmod_int_rel_mult_2: | |
| 2000 | assumes "0 \<le> b" | |
| 2001 | assumes "divmod_int_rel a b (q, r)" | |
| 2002 | shows "divmod_int_rel (1 + 2*a) (2*b) (q, 1 + 2*r)" | |
| 2003 | using assms unfolding divmod_int_rel_def by auto | |
| 2004 | ||
| 2005 | lemma neg_divmod_int_rel_mult_2: | |
| 2006 | assumes "b \<le> 0" | |
| 2007 | assumes "divmod_int_rel (a + 1) b (q, r)" | |
| 2008 | shows "divmod_int_rel (1 + 2*a) (2*b) (q, 2*r - 1)" | |
| 2009 | using assms unfolding divmod_int_rel_def by auto | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2010 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2011 | text{*computing div by shifting *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2012 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2013 | lemma pos_zdiv_mult_2: "(0::int) \<le> a ==> (1 + 2*b) div (2*a) = b div a" | 
| 47166 | 2014 | using pos_divmod_int_rel_mult_2 [OF _ divmod_int_rel_div_mod] | 
| 2015 | by (rule div_int_unique) | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2016 | |
| 35815 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 2017 | lemma neg_zdiv_mult_2: | 
| 
10e723e54076
tuned proofs (to avoid linarith error message caused by bootstrapping of HOL)
 boehmes parents: 
35673diff
changeset | 2018 | assumes A: "a \<le> (0::int)" shows "(1 + 2*b) div (2*a) = (b+1) div a" | 
| 47166 | 2019 | using neg_divmod_int_rel_mult_2 [OF A divmod_int_rel_div_mod] | 
| 2020 | by (rule div_int_unique) | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2021 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2022 | (* FIXME: add rules for negative numerals *) | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2023 | lemma zdiv_numeral_Bit0 [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2024 | "numeral (Num.Bit0 v) div numeral (Num.Bit0 w) = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2025 | numeral v div (numeral w :: int)" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2026 | unfolding numeral.simps unfolding mult_2 [symmetric] | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2027 | by (rule div_mult_mult1, simp) | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2028 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2029 | lemma zdiv_numeral_Bit1 [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2030 | "numeral (Num.Bit1 v) div numeral (Num.Bit0 w) = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2031 | (numeral v div (numeral w :: int))" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2032 | unfolding numeral.simps | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2033 | unfolding mult_2 [symmetric] add_commute [of _ 1] | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2034 | by (rule pos_zdiv_mult_2, simp) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2035 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2036 | lemma pos_zmod_mult_2: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2037 | fixes a b :: int | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2038 | assumes "0 \<le> a" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2039 | shows "(1 + 2 * b) mod (2 * a) = 1 + 2 * (b mod a)" | 
| 47166 | 2040 | using pos_divmod_int_rel_mult_2 [OF assms divmod_int_rel_div_mod] | 
| 2041 | by (rule mod_int_unique) | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2042 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2043 | lemma neg_zmod_mult_2: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2044 | fixes a b :: int | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2045 | assumes "a \<le> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2046 | shows "(1 + 2 * b) mod (2 * a) = 2 * ((b + 1) mod a) - 1" | 
| 47166 | 2047 | using neg_divmod_int_rel_mult_2 [OF assms divmod_int_rel_div_mod] | 
| 2048 | by (rule mod_int_unique) | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2049 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2050 | (* FIXME: add rules for negative numerals *) | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2051 | lemma zmod_numeral_Bit0 [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2052 | "numeral (Num.Bit0 v) mod numeral (Num.Bit0 w) = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2053 | (2::int) * (numeral v mod numeral w)" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2054 | unfolding numeral_Bit0 [of v] numeral_Bit0 [of w] | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2055 | unfolding mult_2 [symmetric] by (rule mod_mult_mult1) | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2056 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2057 | lemma zmod_numeral_Bit1 [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2058 | "numeral (Num.Bit1 v) mod numeral (Num.Bit0 w) = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2059 | 2 * (numeral v mod numeral w) + (1::int)" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2060 | unfolding numeral_Bit1 [of v] numeral_Bit0 [of w] | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2061 | unfolding mult_2 [symmetric] add_commute [of _ 1] | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2062 | by (rule pos_zmod_mult_2, simp) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2063 | |
| 39489 | 2064 | lemma zdiv_eq_0_iff: | 
| 2065 | "(i::int) div k = 0 \<longleftrightarrow> k=0 \<or> 0\<le>i \<and> i<k \<or> i\<le>0 \<and> k<i" (is "?L = ?R") | |
| 2066 | proof | |
| 2067 | assume ?L | |
| 2068 | have "?L \<longrightarrow> ?R" by (rule split_zdiv[THEN iffD2]) simp | |
| 2069 | with `?L` show ?R by blast | |
| 2070 | next | |
| 2071 | assume ?R thus ?L | |
| 2072 | by(auto simp: div_pos_pos_trivial div_neg_neg_trivial) | |
| 2073 | qed | |
| 2074 | ||
| 2075 | ||
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 2076 | subsubsection {* Quotients of Signs *}
 | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2077 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2078 | lemma div_neg_pos_less0: "[| a < (0::int); 0 < b |] ==> a div b < 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2079 | apply (subgoal_tac "a div b \<le> -1", force) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2080 | apply (rule order_trans) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2081 | apply (rule_tac a' = "-1" in zdiv_mono1) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2082 | apply (auto simp add: div_eq_minus1) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2083 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2084 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2085 | lemma div_nonneg_neg_le0: "[| (0::int) \<le> a; b < 0 |] ==> a div b \<le> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2086 | by (drule zdiv_mono1_neg, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2087 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2088 | lemma div_nonpos_pos_le0: "[| (a::int) \<le> 0; b > 0 |] ==> a div b \<le> 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2089 | by (drule zdiv_mono1, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2090 | |
| 33804 | 2091 | text{* Now for some equivalences of the form @{text"a div b >=< 0 \<longleftrightarrow> \<dots>"}
 | 
| 2092 | conditional upon the sign of @{text a} or @{text b}. There are many more.
 | |
| 2093 | They should all be simp rules unless that causes too much search. *} | |
| 2094 | ||
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2095 | lemma pos_imp_zdiv_nonneg_iff: "(0::int) < b ==> (0 \<le> a div b) = (0 \<le> a)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2096 | apply auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2097 | apply (drule_tac [2] zdiv_mono1) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2098 | apply (auto simp add: linorder_neq_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2099 | apply (simp (no_asm_use) add: linorder_not_less [symmetric]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2100 | apply (blast intro: div_neg_pos_less0) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2101 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2102 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2103 | lemma neg_imp_zdiv_nonneg_iff: | 
| 33804 | 2104 | "b < (0::int) ==> (0 \<le> a div b) = (a \<le> (0::int))" | 
| 47159 | 2105 | apply (subst div_minus_minus [symmetric]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2106 | apply (subst pos_imp_zdiv_nonneg_iff, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2107 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2108 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2109 | (*But not (a div b \<le> 0 iff a\<le>0); consider a=1, b=2 when a div b = 0.*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2110 | lemma pos_imp_zdiv_neg_iff: "(0::int) < b ==> (a div b < 0) = (a < 0)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2111 | by (simp add: linorder_not_le [symmetric] pos_imp_zdiv_nonneg_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2112 | |
| 39489 | 2113 | lemma pos_imp_zdiv_pos_iff: | 
| 2114 | "0<k \<Longrightarrow> 0 < (i::int) div k \<longleftrightarrow> k \<le> i" | |
| 2115 | using pos_imp_zdiv_nonneg_iff[of k i] zdiv_eq_0_iff[of i k] | |
| 2116 | by arith | |
| 2117 | ||
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2118 | (*Again the law fails for \<le>: consider a = -1, b = -2 when a div b = 0*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2119 | lemma neg_imp_zdiv_neg_iff: "b < (0::int) ==> (a div b < 0) = (0 < a)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2120 | by (simp add: linorder_not_le [symmetric] neg_imp_zdiv_nonneg_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2121 | |
| 33804 | 2122 | lemma nonneg1_imp_zdiv_pos_iff: | 
| 2123 | "(0::int) <= a \<Longrightarrow> (a div b > 0) = (a >= b & b>0)" | |
| 2124 | apply rule | |
| 2125 | apply rule | |
| 2126 | using div_pos_pos_trivial[of a b]apply arith | |
| 2127 | apply(cases "b=0")apply simp | |
| 2128 | using div_nonneg_neg_le0[of a b]apply arith | |
| 2129 | using int_one_le_iff_zero_less[of "a div b"] zdiv_mono1[of b a b]apply simp | |
| 2130 | done | |
| 2131 | ||
| 39489 | 2132 | lemma zmod_le_nonneg_dividend: "(m::int) \<ge> 0 ==> m mod k \<le> m" | 
| 2133 | apply (rule split_zmod[THEN iffD2]) | |
| 44890 
22f665a2e91c
new fastforce replacing fastsimp - less confusing name
 nipkow parents: 
44766diff
changeset | 2134 | apply(fastforce dest: q_pos_lemma intro: split_mult_pos_le) | 
| 39489 | 2135 | done | 
| 2136 | ||
| 2137 | ||
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2138 | subsubsection {* The Divides Relation *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2139 | |
| 47268 | 2140 | lemma dvd_neg_numeral_left [simp]: | 
| 2141 | fixes y :: "'a::comm_ring_1" | |
| 2142 | shows "(neg_numeral k) dvd y \<longleftrightarrow> (numeral k) dvd y" | |
| 2143 | unfolding neg_numeral_def minus_dvd_iff .. | |
| 2144 | ||
| 2145 | lemma dvd_neg_numeral_right [simp]: | |
| 2146 | fixes x :: "'a::comm_ring_1" | |
| 2147 | shows "x dvd (neg_numeral k) \<longleftrightarrow> x dvd (numeral k)" | |
| 2148 | unfolding neg_numeral_def dvd_minus_iff .. | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2149 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2150 | lemmas dvd_eq_mod_eq_0_numeral [simp] = | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2151 | dvd_eq_mod_eq_0 [of "numeral x" "numeral y"] for x y | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2152 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2153 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2154 | subsubsection {* Further properties *}
 | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2155 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2156 | lemma zmult_div_cancel: "(n::int) * (m div n) = m - (m mod n)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2157 | using zmod_zdiv_equality[where a="m" and b="n"] | 
| 47142 | 2158 | by (simp add: algebra_simps) (* FIXME: generalize *) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2159 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2160 | lemma zdiv_int: "int (a div b) = (int a) div (int b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2161 | apply (subst split_div, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2162 | apply (subst split_zdiv, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2163 | apply (rule_tac a="int (b * i) + int j" and b="int b" and r="int j" and r'=ja in unique_quotient) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2164 | apply (auto simp add: divmod_int_rel_def of_nat_mult) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2165 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2166 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2167 | lemma zmod_int: "int (a mod b) = (int a) mod (int b)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2168 | apply (subst split_mod, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2169 | apply (subst split_zmod, auto) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2170 | apply (rule_tac a="int (b * i) + int j" and b="int b" and q="int i" and q'=ia | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2171 | in unique_remainder) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2172 | apply (auto simp add: divmod_int_rel_def of_nat_mult) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2173 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2174 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2175 | lemma abs_div: "(y::int) dvd x \<Longrightarrow> abs (x div y) = abs x div abs y" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2176 | by (unfold dvd_def, cases "y=0", auto simp add: abs_mult) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2177 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2178 | text{*Suggested by Matthias Daum*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2179 | lemma int_power_div_base: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2180 | "\<lbrakk>0 < m; 0 < k\<rbrakk> \<Longrightarrow> k ^ m div k = (k::int) ^ (m - Suc 0)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2181 | apply (subgoal_tac "k ^ m = k ^ ((m - Suc 0) + Suc 0)") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2182 | apply (erule ssubst) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2183 | apply (simp only: power_add) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2184 | apply simp_all | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2185 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2186 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2187 | text {* by Brian Huffman *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2188 | lemma zminus_zmod: "- ((x::int) mod m) mod m = - x mod m" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2189 | by (rule mod_minus_eq [symmetric]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2190 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2191 | lemma zdiff_zmod_left: "(x mod m - y) mod m = (x - y) mod (m::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2192 | by (rule mod_diff_left_eq [symmetric]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2193 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2194 | lemma zdiff_zmod_right: "(x - y mod m) mod m = (x - y) mod (m::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2195 | by (rule mod_diff_right_eq [symmetric]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2196 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2197 | lemmas zmod_simps = | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2198 | mod_add_left_eq [symmetric] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2199 | mod_add_right_eq [symmetric] | 
| 47142 | 2200 | mod_mult_right_eq[symmetric] | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2201 | mod_mult_left_eq [symmetric] | 
| 47164 | 2202 | power_mod | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2203 | zminus_zmod zdiff_zmod_left zdiff_zmod_right | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2204 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2205 | text {* Distributive laws for function @{text nat}. *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2206 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2207 | lemma nat_div_distrib: "0 \<le> x \<Longrightarrow> nat (x div y) = nat x div nat y" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2208 | apply (rule linorder_cases [of y 0]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2209 | apply (simp add: div_nonneg_neg_le0) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2210 | apply simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2211 | apply (simp add: nat_eq_iff pos_imp_zdiv_nonneg_iff zdiv_int) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2212 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2213 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2214 | (*Fails if y<0: the LHS collapses to (nat z) but the RHS doesn't*) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2215 | lemma nat_mod_distrib: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2216 | "\<lbrakk>0 \<le> x; 0 \<le> y\<rbrakk> \<Longrightarrow> nat (x mod y) = nat x mod nat y" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2217 | apply (case_tac "y = 0", simp) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2218 | apply (simp add: nat_eq_iff zmod_int) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2219 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2220 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2221 | text  {* transfer setup *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2222 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2223 | lemma transfer_nat_int_functions: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2224 | "(x::int) >= 0 \<Longrightarrow> y >= 0 \<Longrightarrow> (nat x) div (nat y) = nat (x div y)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2225 | "(x::int) >= 0 \<Longrightarrow> y >= 0 \<Longrightarrow> (nat x) mod (nat y) = nat (x mod y)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2226 | by (auto simp add: nat_div_distrib nat_mod_distrib) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2227 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2228 | lemma transfer_nat_int_function_closures: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2229 | "(x::int) >= 0 \<Longrightarrow> y >= 0 \<Longrightarrow> x div y >= 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2230 | "(x::int) >= 0 \<Longrightarrow> y >= 0 \<Longrightarrow> x mod y >= 0" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2231 | apply (cases "y = 0") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2232 | apply (auto simp add: pos_imp_zdiv_nonneg_iff) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2233 | apply (cases "y = 0") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2234 | apply auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2235 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2236 | |
| 35644 | 2237 | declare transfer_morphism_nat_int [transfer add return: | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2238 | transfer_nat_int_functions | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2239 | transfer_nat_int_function_closures | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2240 | ] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2241 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2242 | lemma transfer_int_nat_functions: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2243 | "(int x) div (int y) = int (x div y)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2244 | "(int x) mod (int y) = int (x mod y)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2245 | by (auto simp add: zdiv_int zmod_int) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2246 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2247 | lemma transfer_int_nat_function_closures: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2248 | "is_nat x \<Longrightarrow> is_nat y \<Longrightarrow> is_nat (x div y)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2249 | "is_nat x \<Longrightarrow> is_nat y \<Longrightarrow> is_nat (x mod y)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2250 | by (simp_all only: is_nat_def transfer_nat_int_function_closures) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2251 | |
| 35644 | 2252 | declare transfer_morphism_int_nat [transfer add return: | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2253 | transfer_int_nat_functions | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2254 | transfer_int_nat_function_closures | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2255 | ] | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2256 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2257 | text{*Suggested by Matthias Daum*}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2258 | lemma int_div_less_self: "\<lbrakk>0 < x; 1 < k\<rbrakk> \<Longrightarrow> x div k < (x::int)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2259 | apply (subgoal_tac "nat x div nat k < nat x") | 
| 34225 | 2260 | apply (simp add: nat_div_distrib [symmetric]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2261 | apply (rule Divides.div_less_dividend, simp_all) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2262 | done | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2263 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2264 | lemma zmod_eq_dvd_iff: "(x::int) mod n = y mod n \<longleftrightarrow> n dvd x - y" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2265 | proof | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2266 | assume H: "x mod n = y mod n" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2267 | hence "x mod n - y mod n = 0" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2268 | hence "(x mod n - y mod n) mod n = 0" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2269 | hence "(x - y) mod n = 0" by (simp add: mod_diff_eq[symmetric]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2270 | thus "n dvd x - y" by (simp add: dvd_eq_mod_eq_0) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2271 | next | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2272 | assume H: "n dvd x - y" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2273 | then obtain k where k: "x-y = n*k" unfolding dvd_def by blast | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2274 | hence "x = n*k + y" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2275 | hence "x mod n = (n*k + y) mod n" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2276 | thus "x mod n = y mod n" by (simp add: mod_add_left_eq) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2277 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2278 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2279 | lemma nat_mod_eq_lemma: assumes xyn: "(x::nat) mod n = y mod n" and xy:"y \<le> x" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2280 | shows "\<exists>q. x = y + n * q" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2281 | proof- | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2282 | from xy have th: "int x - int y = int (x - y)" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2283 | from xyn have "int x mod int n = int y mod int n" | 
| 46551 
866bce5442a3
simplify projections on simultaneous computations of div and mod; tuned structure (from Florian Haftmann)
 huffman parents: 
46026diff
changeset | 2284 | by (simp add: zmod_int [symmetric]) | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2285 | hence "int n dvd int x - int y" by (simp only: zmod_eq_dvd_iff[symmetric]) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2286 | hence "n dvd x - y" by (simp add: th zdvd_int) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2287 | then show ?thesis using xy unfolding dvd_def apply clarsimp apply (rule_tac x="k" in exI) by arith | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2288 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2289 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2290 | lemma nat_mod_eq_iff: "(x::nat) mod n = y mod n \<longleftrightarrow> (\<exists>q1 q2. x + n * q1 = y + n * q2)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2291 | (is "?lhs = ?rhs") | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2292 | proof | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2293 | assume H: "x mod n = y mod n" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2294 |   {assume xy: "x \<le> y"
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2295 | from H have th: "y mod n = x mod n" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2296 | from nat_mod_eq_lemma[OF th xy] have ?rhs | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2297 | apply clarify apply (rule_tac x="q" in exI) by (rule exI[where x="0"], simp)} | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2298 | moreover | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2299 |   {assume xy: "y \<le> x"
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2300 | from nat_mod_eq_lemma[OF H xy] have ?rhs | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2301 | apply clarify apply (rule_tac x="0" in exI) by (rule_tac x="q" in exI, simp)} | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2302 | ultimately show ?rhs using linear[of x y] by blast | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2303 | next | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2304 | assume ?rhs then obtain q1 q2 where q12: "x + n * q1 = y + n * q2" by blast | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2305 | hence "(x + n * q1) mod n = (y + n * q2) mod n" by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2306 | thus ?lhs by simp | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2307 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2308 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2309 | lemma div_nat_numeral [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2310 | "(numeral v :: nat) div numeral v' = nat (numeral v div numeral v')" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2311 | by (simp add: nat_div_distrib) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2312 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2313 | lemma one_div_nat_numeral [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2314 | "Suc 0 div numeral v' = nat (1 div numeral v')" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2315 | by (subst nat_div_distrib, simp_all) | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2316 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2317 | lemma mod_nat_numeral [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2318 | "(numeral v :: nat) mod numeral v' = nat (numeral v mod numeral v')" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2319 | by (simp add: nat_mod_distrib) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2320 | |
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2321 | lemma one_mod_nat_numeral [simp]: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2322 | "Suc 0 mod numeral v' = nat (1 mod numeral v')" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2323 | by (subst nat_mod_distrib) simp_all | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2324 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2325 | lemma mod_2_not_eq_zero_eq_one_int: | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2326 | fixes k :: int | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2327 | shows "k mod 2 \<noteq> 0 \<longleftrightarrow> k mod 2 = 1" | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2328 | by auto | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2329 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2330 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2331 | subsubsection {* Tools setup *}
 | 
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2332 | |
| 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2333 | text {* Nitpick *}
 | 
| 34126 | 2334 | |
| 41792 
ff3cb0c418b7
renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics
 blanchet parents: 
41550diff
changeset | 2335 | lemmas [nitpick_unfold] = dvd_eq_mod_eq_0 mod_div_equality' zmod_zdiv_equality' | 
| 34126 | 2336 | |
| 35673 | 2337 | |
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2338 | subsubsection {* Code generation *}
 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2339 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2340 | definition pdivmod :: "int \<Rightarrow> int \<Rightarrow> int \<times> int" where | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2341 | "pdivmod k l = (\<bar>k\<bar> div \<bar>l\<bar>, \<bar>k\<bar> mod \<bar>l\<bar>)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2342 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2343 | lemma pdivmod_posDivAlg [code]: | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2344 | "pdivmod k l = (if l = 0 then (0, \<bar>k\<bar>) else posDivAlg \<bar>k\<bar> \<bar>l\<bar>)" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2345 | by (subst posDivAlg_div_mod) (simp_all add: pdivmod_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2346 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2347 | lemma divmod_int_pdivmod: "divmod_int k l = (if k = 0 then (0, 0) else if l = 0 then (0, k) else | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2348 | apsnd ((op *) (sgn l)) (if 0 < l \<and> 0 \<le> k \<or> l < 0 \<and> k < 0 | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2349 | then pdivmod k l | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2350 | else (let (r, s) = pdivmod k l in | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46560diff
changeset | 2351 | if s = 0 then (- r, 0) else (- r - 1, \<bar>l\<bar> - s))))" | 
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2352 | proof - | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2353 | have aux: "\<And>q::int. - k = l * q \<longleftrightarrow> k = l * - q" by auto | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2354 | show ?thesis | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2355 | by (simp add: divmod_int_mod_div pdivmod_def) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2356 | (auto simp add: aux not_less not_le zdiv_zminus1_eq_if | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2357 | zmod_zminus1_eq_if zdiv_zminus2_eq_if zmod_zminus2_eq_if) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2358 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2359 | |
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2360 | lemma divmod_int_code [code]: "divmod_int k l = (if k = 0 then (0, 0) else if l = 0 then (0, k) else | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2361 | apsnd ((op *) (sgn l)) (if sgn k = sgn l | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2362 | then pdivmod k l | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2363 | else (let (r, s) = pdivmod k l in | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2364 | if s = 0 then (- r, 0) else (- r - 1, \<bar>l\<bar> - s))))" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2365 | proof - | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2366 | have "k \<noteq> 0 \<Longrightarrow> l \<noteq> 0 \<Longrightarrow> 0 < l \<and> 0 \<le> k \<or> l < 0 \<and> k < 0 \<longleftrightarrow> sgn k = sgn l" | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2367 | by (auto simp add: not_less sgn_if) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2368 | then show ?thesis by (simp add: divmod_int_pdivmod) | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2369 | qed | 
| 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2370 | |
| 33364 | 2371 | code_modulename SML | 
| 2372 | Divides Arith | |
| 2373 | ||
| 2374 | code_modulename OCaml | |
| 2375 | Divides Arith | |
| 2376 | ||
| 2377 | code_modulename Haskell | |
| 2378 | Divides Arith | |
| 2379 | ||
| 33361 
1f18de40b43f
combined former theories Divides and IntDiv to one theory Divides
 haftmann parents: 
33340diff
changeset | 2380 | end |