| author | blanchet | 
| Tue, 19 Nov 2013 19:42:30 +0100 | |
| changeset 54506 | 8b5caa190054 | 
| parent 54489 | 03ff4d1e6784 | 
| child 55375 | d26d5f988d71 | 
| permissions | -rw-r--r-- | 
| 33366 | 1  | 
(* Author: Various *)  | 
2  | 
||
3  | 
header {* Combination and Cancellation Simprocs for Numeral Expressions *}
 | 
|
4  | 
||
5  | 
theory Numeral_Simprocs  | 
|
6  | 
imports Divides  | 
|
7  | 
begin  | 
|
8  | 
||
| 48891 | 9  | 
ML_file "~~/src/Provers/Arith/assoc_fold.ML"  | 
10  | 
ML_file "~~/src/Provers/Arith/cancel_numerals.ML"  | 
|
11  | 
ML_file "~~/src/Provers/Arith/combine_numerals.ML"  | 
|
12  | 
ML_file "~~/src/Provers/Arith/cancel_numeral_factor.ML"  | 
|
13  | 
ML_file "~~/src/Provers/Arith/extract_common_term.ML"  | 
|
14  | 
||
| 
47255
 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 
huffman 
parents: 
47159 
diff
changeset
 | 
15  | 
lemmas semiring_norm =  | 
| 54249 | 16  | 
Let_def arith_simps diff_nat_numeral rel_simps  | 
| 
47255
 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 
huffman 
parents: 
47159 
diff
changeset
 | 
17  | 
if_False if_True  | 
| 
 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 
huffman 
parents: 
47159 
diff
changeset
 | 
18  | 
add_0 add_Suc add_numeral_left  | 
| 
 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 
huffman 
parents: 
47159 
diff
changeset
 | 
19  | 
add_neg_numeral_left mult_numeral_left  | 
| 
54489
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
20  | 
numeral_One [symmetric] uminus_numeral_One [symmetric] Suc_eq_plus1  | 
| 
47255
 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 
huffman 
parents: 
47159 
diff
changeset
 | 
21  | 
eq_numeral_iff_iszero not_iszero_Numeral1  | 
| 
 
30a1692557b0
removed Nat_Numeral.thy, moving all theorems elsewhere
 
huffman 
parents: 
47159 
diff
changeset
 | 
22  | 
|
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
23  | 
declare split_div [of _ _ "numeral k", arith_split] for k  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
24  | 
declare split_mod [of _ _ "numeral k", arith_split] for k  | 
| 33366 | 25  | 
|
26  | 
text {* For @{text combine_numerals} *}
 | 
|
27  | 
||
28  | 
lemma left_add_mult_distrib: "i*u + (j*u + k) = (i+j)*u + (k::nat)"  | 
|
29  | 
by (simp add: add_mult_distrib)  | 
|
30  | 
||
31  | 
text {* For @{text cancel_numerals} *}
 | 
|
32  | 
||
33  | 
lemma nat_diff_add_eq1:  | 
|
34  | 
"j <= (i::nat) ==> ((i*u + m) - (j*u + n)) = (((i-j)*u + m) - n)"  | 
|
35  | 
by (simp split add: nat_diff_split add: add_mult_distrib)  | 
|
36  | 
||
37  | 
lemma nat_diff_add_eq2:  | 
|
38  | 
"i <= (j::nat) ==> ((i*u + m) - (j*u + n)) = (m - ((j-i)*u + n))"  | 
|
39  | 
by (simp split add: nat_diff_split add: add_mult_distrib)  | 
|
40  | 
||
41  | 
lemma nat_eq_add_iff1:  | 
|
42  | 
"j <= (i::nat) ==> (i*u + m = j*u + n) = ((i-j)*u + m = n)"  | 
|
43  | 
by (auto split add: nat_diff_split simp add: add_mult_distrib)  | 
|
44  | 
||
45  | 
lemma nat_eq_add_iff2:  | 
|
46  | 
"i <= (j::nat) ==> (i*u + m = j*u + n) = (m = (j-i)*u + n)"  | 
|
47  | 
by (auto split add: nat_diff_split simp add: add_mult_distrib)  | 
|
48  | 
||
49  | 
lemma nat_less_add_iff1:  | 
|
50  | 
"j <= (i::nat) ==> (i*u + m < j*u + n) = ((i-j)*u + m < n)"  | 
|
51  | 
by (auto split add: nat_diff_split simp add: add_mult_distrib)  | 
|
52  | 
||
53  | 
lemma nat_less_add_iff2:  | 
|
54  | 
"i <= (j::nat) ==> (i*u + m < j*u + n) = (m < (j-i)*u + n)"  | 
|
55  | 
by (auto split add: nat_diff_split simp add: add_mult_distrib)  | 
|
56  | 
||
57  | 
lemma nat_le_add_iff1:  | 
|
58  | 
"j <= (i::nat) ==> (i*u + m <= j*u + n) = ((i-j)*u + m <= n)"  | 
|
59  | 
by (auto split add: nat_diff_split simp add: add_mult_distrib)  | 
|
60  | 
||
61  | 
lemma nat_le_add_iff2:  | 
|
62  | 
"i <= (j::nat) ==> (i*u + m <= j*u + n) = (m <= (j-i)*u + n)"  | 
|
63  | 
by (auto split add: nat_diff_split simp add: add_mult_distrib)  | 
|
64  | 
||
65  | 
text {* For @{text cancel_numeral_factors} *}
 | 
|
66  | 
||
67  | 
lemma nat_mult_le_cancel1: "(0::nat) < k ==> (k*m <= k*n) = (m<=n)"  | 
|
68  | 
by auto  | 
|
69  | 
||
70  | 
lemma nat_mult_less_cancel1: "(0::nat) < k ==> (k*m < k*n) = (m<n)"  | 
|
71  | 
by auto  | 
|
72  | 
||
73  | 
lemma nat_mult_eq_cancel1: "(0::nat) < k ==> (k*m = k*n) = (m=n)"  | 
|
74  | 
by auto  | 
|
75  | 
||
76  | 
lemma nat_mult_div_cancel1: "(0::nat) < k ==> (k*m) div (k*n) = (m div n)"  | 
|
77  | 
by auto  | 
|
78  | 
||
79  | 
lemma nat_mult_dvd_cancel_disj[simp]:  | 
|
80  | 
"(k*m) dvd (k*n) = (k=0 | m dvd (n::nat))"  | 
|
| 47159 | 81  | 
by (auto simp: dvd_eq_mod_eq_0 mod_mult_mult1)  | 
| 33366 | 82  | 
|
83  | 
lemma nat_mult_dvd_cancel1: "0 < k \<Longrightarrow> (k*m) dvd (k*n::nat) = (m dvd n)"  | 
|
84  | 
by(auto)  | 
|
85  | 
||
86  | 
text {* For @{text cancel_factor} *}
 | 
|
87  | 
||
| 
54489
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
88  | 
lemmas nat_mult_le_cancel_disj = mult_le_cancel1  | 
| 33366 | 89  | 
|
| 
54489
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
90  | 
lemmas nat_mult_less_cancel_disj = mult_less_cancel1  | 
| 33366 | 91  | 
|
| 
54489
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
92  | 
lemma nat_mult_eq_cancel_disj:  | 
| 
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
93  | 
fixes k m n :: nat  | 
| 
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
94  | 
shows "k * m = k * n \<longleftrightarrow> k = 0 \<or> m = n"  | 
| 
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
95  | 
by auto  | 
| 33366 | 96  | 
|
| 
54489
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
97  | 
lemma nat_mult_div_cancel_disj [simp]:  | 
| 
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
98  | 
fixes k m n :: nat  | 
| 
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
99  | 
shows "(k * m) div (k * n) = (if k = 0 then 0 else m div n)"  | 
| 
 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 
haftmann 
parents: 
54249 
diff
changeset
 | 
100  | 
by (fact div_mult_mult1_if)  | 
| 33366 | 101  | 
|
| 48891 | 102  | 
ML_file "Tools/numeral_simprocs.ML"  | 
| 33366 | 103  | 
|
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
104  | 
simproc_setup semiring_assoc_fold  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
105  | 
  ("(a::'a::comm_semiring_1_cancel) * b") =
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
106  | 
  {* fn phi => Numeral_Simprocs.assoc_fold *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
107  | 
|
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
108  | 
(* TODO: see whether the type class can be generalized further *)  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
109  | 
simproc_setup int_combine_numerals  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
110  | 
  ("(i::'a::comm_ring_1) + j" | "(i::'a::comm_ring_1) - j") =
 | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
111  | 
  {* fn phi => Numeral_Simprocs.combine_numerals *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
112  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
113  | 
simproc_setup field_combine_numerals  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
114  | 
  ("(i::'a::{field_inverse_zero,ring_char_0}) + j"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
115  | 
  |"(i::'a::{field_inverse_zero,ring_char_0}) - j") =
 | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
116  | 
  {* fn phi => Numeral_Simprocs.field_combine_numerals *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
117  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
118  | 
simproc_setup inteq_cancel_numerals  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
119  | 
  ("(l::'a::comm_ring_1) + m = n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
120  | 
|"(l::'a::comm_ring_1) = m + n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
121  | 
|"(l::'a::comm_ring_1) - m = n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
122  | 
|"(l::'a::comm_ring_1) = m - n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
123  | 
|"(l::'a::comm_ring_1) * m = n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
124  | 
|"(l::'a::comm_ring_1) = m * n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
125  | 
|"- (l::'a::comm_ring_1) = m"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
126  | 
|"(l::'a::comm_ring_1) = - m") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
127  | 
  {* fn phi => Numeral_Simprocs.eq_cancel_numerals *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
128  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
129  | 
simproc_setup intless_cancel_numerals  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
130  | 
  ("(l::'a::linordered_idom) + m < n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
131  | 
|"(l::'a::linordered_idom) < m + n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
132  | 
|"(l::'a::linordered_idom) - m < n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
133  | 
|"(l::'a::linordered_idom) < m - n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
134  | 
|"(l::'a::linordered_idom) * m < n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
135  | 
|"(l::'a::linordered_idom) < m * n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
136  | 
|"- (l::'a::linordered_idom) < m"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
137  | 
|"(l::'a::linordered_idom) < - m") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
138  | 
  {* fn phi => Numeral_Simprocs.less_cancel_numerals *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
139  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
140  | 
simproc_setup intle_cancel_numerals  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
141  | 
  ("(l::'a::linordered_idom) + m \<le> n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
142  | 
|"(l::'a::linordered_idom) \<le> m + n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
143  | 
|"(l::'a::linordered_idom) - m \<le> n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
144  | 
|"(l::'a::linordered_idom) \<le> m - n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
145  | 
|"(l::'a::linordered_idom) * m \<le> n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
146  | 
|"(l::'a::linordered_idom) \<le> m * n"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
147  | 
|"- (l::'a::linordered_idom) \<le> m"  | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
148  | 
|"(l::'a::linordered_idom) \<le> - m") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
149  | 
  {* fn phi => Numeral_Simprocs.le_cancel_numerals *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
150  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
151  | 
simproc_setup ring_eq_cancel_numeral_factor  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
152  | 
  ("(l::'a::{idom,ring_char_0}) * m = n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
153  | 
  |"(l::'a::{idom,ring_char_0}) = m * n") =
 | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
154  | 
  {* fn phi => Numeral_Simprocs.eq_cancel_numeral_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
155  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
156  | 
simproc_setup ring_less_cancel_numeral_factor  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
157  | 
  ("(l::'a::linordered_idom) * m < n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
158  | 
|"(l::'a::linordered_idom) < m * n") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
159  | 
  {* fn phi => Numeral_Simprocs.less_cancel_numeral_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
160  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
161  | 
simproc_setup ring_le_cancel_numeral_factor  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
162  | 
  ("(l::'a::linordered_idom) * m <= n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
163  | 
|"(l::'a::linordered_idom) <= m * n") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
164  | 
  {* fn phi => Numeral_Simprocs.le_cancel_numeral_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
165  | 
|
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
166  | 
(* TODO: remove comm_ring_1 constraint if possible *)  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
167  | 
simproc_setup int_div_cancel_numeral_factors  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
168  | 
  ("((l::'a::{semiring_div,comm_ring_1,ring_char_0}) * m) div n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
169  | 
  |"(l::'a::{semiring_div,comm_ring_1,ring_char_0}) div (m * n)") =
 | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
170  | 
  {* fn phi => Numeral_Simprocs.div_cancel_numeral_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
171  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
172  | 
simproc_setup divide_cancel_numeral_factor  | 
| 
47108
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
173  | 
  ("((l::'a::{field_inverse_zero,ring_char_0}) * m) / n"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
174  | 
  |"(l::'a::{field_inverse_zero,ring_char_0}) / (m * n)"
 | 
| 
 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 
huffman 
parents: 
45607 
diff
changeset
 | 
175  | 
  |"((numeral v)::'a::{field_inverse_zero,ring_char_0}) / (numeral w)") =
 | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
176  | 
  {* fn phi => Numeral_Simprocs.divide_cancel_numeral_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
177  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
178  | 
simproc_setup ring_eq_cancel_factor  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
179  | 
  ("(l::'a::idom) * m = n" | "(l::'a::idom) = m * n") =
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
180  | 
  {* fn phi => Numeral_Simprocs.eq_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
181  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
182  | 
simproc_setup linordered_ring_le_cancel_factor  | 
| 
45296
 
7a97b2bda137
more accurate class constraints on cancellation simproc patterns
 
huffman 
parents: 
45284 
diff
changeset
 | 
183  | 
  ("(l::'a::linordered_idom) * m <= n"
 | 
| 
 
7a97b2bda137
more accurate class constraints on cancellation simproc patterns
 
huffman 
parents: 
45284 
diff
changeset
 | 
184  | 
|"(l::'a::linordered_idom) <= m * n") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
185  | 
  {* fn phi => Numeral_Simprocs.le_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
186  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
187  | 
simproc_setup linordered_ring_less_cancel_factor  | 
| 
45296
 
7a97b2bda137
more accurate class constraints on cancellation simproc patterns
 
huffman 
parents: 
45284 
diff
changeset
 | 
188  | 
  ("(l::'a::linordered_idom) * m < n"
 | 
| 
 
7a97b2bda137
more accurate class constraints on cancellation simproc patterns
 
huffman 
parents: 
45284 
diff
changeset
 | 
189  | 
|"(l::'a::linordered_idom) < m * n") =  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
190  | 
  {* fn phi => Numeral_Simprocs.less_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
191  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
192  | 
simproc_setup int_div_cancel_factor  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
193  | 
  ("((l::'a::semiring_div) * m) div n"
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
194  | 
|"(l::'a::semiring_div) div (m * n)") =  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
195  | 
  {* fn phi => Numeral_Simprocs.div_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
196  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
197  | 
simproc_setup int_mod_cancel_factor  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
198  | 
  ("((l::'a::semiring_div) * m) mod n"
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
199  | 
|"(l::'a::semiring_div) mod (m * n)") =  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
200  | 
  {* fn phi => Numeral_Simprocs.mod_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
201  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
202  | 
simproc_setup dvd_cancel_factor  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
203  | 
  ("((l::'a::idom) * m) dvd n"
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
204  | 
|"(l::'a::idom) dvd (m * n)") =  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
205  | 
  {* fn phi => Numeral_Simprocs.dvd_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
206  | 
|
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
207  | 
simproc_setup divide_cancel_factor  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
208  | 
  ("((l::'a::field_inverse_zero) * m) / n"
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
209  | 
|"(l::'a::field_inverse_zero) / (m * n)") =  | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
210  | 
  {* fn phi => Numeral_Simprocs.divide_cancel_factor *}
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
211  | 
|
| 48891 | 212  | 
ML_file "Tools/nat_numeral_simprocs.ML"  | 
| 33366 | 213  | 
|
| 
45462
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
214  | 
simproc_setup nat_combine_numerals  | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
215  | 
  ("(i::nat) + j" | "Suc (i + j)") =
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
216  | 
  {* fn phi => Nat_Numeral_Simprocs.combine_numerals *}
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
217  | 
|
| 
45436
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
218  | 
simproc_setup nateq_cancel_numerals  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
219  | 
  ("(l::nat) + m = n" | "(l::nat) = m + n" |
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
220  | 
"(l::nat) * m = n" | "(l::nat) = m * n" |  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
221  | 
"Suc m = n" | "m = Suc n") =  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
222  | 
  {* fn phi => Nat_Numeral_Simprocs.eq_cancel_numerals *}
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
223  | 
|
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
224  | 
simproc_setup natless_cancel_numerals  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
225  | 
  ("(l::nat) + m < n" | "(l::nat) < m + n" |
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
226  | 
"(l::nat) * m < n" | "(l::nat) < m * n" |  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
227  | 
"Suc m < n" | "m < Suc n") =  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
228  | 
  {* fn phi => Nat_Numeral_Simprocs.less_cancel_numerals *}
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
229  | 
|
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
230  | 
simproc_setup natle_cancel_numerals  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
231  | 
  ("(l::nat) + m \<le> n" | "(l::nat) \<le> m + n" |
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
232  | 
"(l::nat) * m \<le> n" | "(l::nat) \<le> m * n" |  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
233  | 
"Suc m \<le> n" | "m \<le> Suc n") =  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
234  | 
  {* fn phi => Nat_Numeral_Simprocs.le_cancel_numerals *}
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
235  | 
|
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
236  | 
simproc_setup natdiff_cancel_numerals  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
237  | 
  ("((l::nat) + m) - n" | "(l::nat) - (m + n)" |
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
238  | 
"(l::nat) * m - n" | "(l::nat) - m * n" |  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
239  | 
"Suc m - n" | "m - Suc n") =  | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
240  | 
  {* fn phi => Nat_Numeral_Simprocs.diff_cancel_numerals *}
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
241  | 
|
| 
45463
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
242  | 
simproc_setup nat_eq_cancel_numeral_factor  | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
243  | 
  ("(l::nat) * m = n" | "(l::nat) = m * n") =
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
244  | 
  {* fn phi => Nat_Numeral_Simprocs.eq_cancel_numeral_factor *}
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
245  | 
|
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
246  | 
simproc_setup nat_less_cancel_numeral_factor  | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
247  | 
  ("(l::nat) * m < n" | "(l::nat) < m * n") =
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
248  | 
  {* fn phi => Nat_Numeral_Simprocs.less_cancel_numeral_factor *}
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
249  | 
|
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
250  | 
simproc_setup nat_le_cancel_numeral_factor  | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
251  | 
  ("(l::nat) * m <= n" | "(l::nat) <= m * n") =
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
252  | 
  {* fn phi => Nat_Numeral_Simprocs.le_cancel_numeral_factor *}
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
253  | 
|
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
254  | 
simproc_setup nat_div_cancel_numeral_factor  | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
255  | 
  ("((l::nat) * m) div n" | "(l::nat) div (m * n)") =
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
256  | 
  {* fn phi => Nat_Numeral_Simprocs.div_cancel_numeral_factor *}
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
257  | 
|
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
258  | 
simproc_setup nat_dvd_cancel_numeral_factor  | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
259  | 
  ("((l::nat) * m) dvd n" | "(l::nat) dvd (m * n)") =
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
260  | 
  {* fn phi => Nat_Numeral_Simprocs.dvd_cancel_numeral_factor *}
 | 
| 
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
261  | 
|
| 
45462
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
262  | 
simproc_setup nat_eq_cancel_factor  | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
263  | 
  ("(l::nat) * m = n" | "(l::nat) = m * n") =
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
264  | 
  {* fn phi => Nat_Numeral_Simprocs.eq_cancel_factor *}
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
265  | 
|
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
266  | 
simproc_setup nat_less_cancel_factor  | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
267  | 
  ("(l::nat) * m < n" | "(l::nat) < m * n") =
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
268  | 
  {* fn phi => Nat_Numeral_Simprocs.less_cancel_factor *}
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
269  | 
|
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
270  | 
simproc_setup nat_le_cancel_factor  | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
271  | 
  ("(l::nat) * m <= n" | "(l::nat) <= m * n") =
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
272  | 
  {* fn phi => Nat_Numeral_Simprocs.le_cancel_factor *}
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
273  | 
|
| 
45463
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
274  | 
simproc_setup nat_div_cancel_factor  | 
| 
45462
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
275  | 
  ("((l::nat) * m) div n" | "(l::nat) div (m * n)") =
 | 
| 
45463
 
9a588a835c1e
use simproc_setup for the remaining nat_numeral simprocs
 
huffman 
parents: 
45462 
diff
changeset
 | 
276  | 
  {* fn phi => Nat_Numeral_Simprocs.div_cancel_factor *}
 | 
| 
45462
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
277  | 
|
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
278  | 
simproc_setup nat_dvd_cancel_factor  | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
279  | 
  ("((l::nat) * m) dvd n" | "(l::nat) dvd (m * n)") =
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
280  | 
  {* fn phi => Nat_Numeral_Simprocs.dvd_cancel_factor *}
 | 
| 
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
281  | 
|
| 33366 | 282  | 
declaration {* 
 | 
| 54249 | 283  | 
K (Lin_Arith.add_simprocs  | 
| 
45284
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
284  | 
      [@{simproc semiring_assoc_fold},
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
285  | 
       @{simproc int_combine_numerals},
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
286  | 
       @{simproc inteq_cancel_numerals},
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
287  | 
       @{simproc intless_cancel_numerals},
 | 
| 
 
ae78a4ffa81d
use simproc_setup for cancellation simprocs, to get proper name bindings
 
huffman 
parents: 
37886 
diff
changeset
 | 
288  | 
       @{simproc intle_cancel_numerals}]
 | 
| 
45436
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
289  | 
#> Lin_Arith.add_simprocs  | 
| 
45462
 
aba629d6cee5
use simproc_setup for more nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45436 
diff
changeset
 | 
290  | 
      [@{simproc nat_combine_numerals},
 | 
| 
45436
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
291  | 
       @{simproc nateq_cancel_numerals},
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
292  | 
       @{simproc natless_cancel_numerals},
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
293  | 
       @{simproc natle_cancel_numerals},
 | 
| 
 
62bc9474d04b
use simproc_setup for some nat_numeral simprocs; add simproc tests
 
huffman 
parents: 
45435 
diff
changeset
 | 
294  | 
       @{simproc natdiff_cancel_numerals}])
 | 
| 33366 | 295  | 
*}  | 
296  | 
||
| 37886 | 297  | 
end  |