author | wenzelm |
Sun, 12 Jan 2025 16:03:43 +0100 | |
changeset 81790 | 134880dc4df2 |
parent 81595 | ed264056f5dc |
permissions | -rw-r--r-- |
58101 | 1 |
(* Author: Tobias Nipkow, TU Muenchen *) |
2 |
||
60758 | 3 |
section \<open>Sum and product over lists\<close> |
58101 | 4 |
|
5 |
theory Groups_List |
|
6 |
imports List |
|
7 |
begin |
|
8 |
||
58320 | 9 |
locale monoid_list = monoid |
10 |
begin |
|
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
11 |
|
58320 | 12 |
definition F :: "'a list \<Rightarrow> 'a" |
13 |
where |
|
63290
9ac558ab0906
boldify syntax in abstract algebraic structures, to avoid clashes with concrete syntax in corresponding type classes
haftmann
parents:
63101
diff
changeset
|
14 |
eq_foldr [code]: "F xs = foldr f xs \<^bold>1" |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
15 |
|
58320 | 16 |
lemma Nil [simp]: |
63290
9ac558ab0906
boldify syntax in abstract algebraic structures, to avoid clashes with concrete syntax in corresponding type classes
haftmann
parents:
63101
diff
changeset
|
17 |
"F [] = \<^bold>1" |
58320 | 18 |
by (simp add: eq_foldr) |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
19 |
|
58320 | 20 |
lemma Cons [simp]: |
63290
9ac558ab0906
boldify syntax in abstract algebraic structures, to avoid clashes with concrete syntax in corresponding type classes
haftmann
parents:
63101
diff
changeset
|
21 |
"F (x # xs) = x \<^bold>* F xs" |
58320 | 22 |
by (simp add: eq_foldr) |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
23 |
|
58320 | 24 |
lemma append [simp]: |
63290
9ac558ab0906
boldify syntax in abstract algebraic structures, to avoid clashes with concrete syntax in corresponding type classes
haftmann
parents:
63101
diff
changeset
|
25 |
"F (xs @ ys) = F xs \<^bold>* F ys" |
58320 | 26 |
by (induct xs) (simp_all add: assoc) |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
27 |
|
58320 | 28 |
end |
58101 | 29 |
|
58320 | 30 |
locale comm_monoid_list = comm_monoid + monoid_list |
31 |
begin |
|
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
32 |
|
58320 | 33 |
lemma rev [simp]: |
34 |
"F (rev xs) = F xs" |
|
35 |
by (simp add: eq_foldr foldr_fold fold_rev fun_eq_iff assoc left_commute) |
|
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
36 |
|
58320 | 37 |
end |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
38 |
|
58320 | 39 |
locale comm_monoid_list_set = list: comm_monoid_list + set: comm_monoid_set |
40 |
begin |
|
58101 | 41 |
|
58320 | 42 |
lemma distinct_set_conv_list: |
43 |
"distinct xs \<Longrightarrow> set.F g (set xs) = list.F (map g xs)" |
|
44 |
by (induct xs) simp_all |
|
58101 | 45 |
|
58320 | 46 |
lemma set_conv_list [code]: |
47 |
"set.F g (set xs) = list.F (map g (remdups xs))" |
|
48 |
by (simp add: distinct_set_conv_list [symmetric]) |
|
49 |
||
80061
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
50 |
lemma list_conv_set_nth: |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
51 |
"list.F xs = set.F (\<lambda>i. xs ! i) {0..<length xs}" |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
52 |
proof - |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
53 |
have "xs = map (\<lambda>i. xs ! i) [0..<length xs]" |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
54 |
by (simp add: map_nth) |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
55 |
also have "list.F \<dots> = set.F (\<lambda>i. xs ! i) {0..<length xs}" |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
56 |
by (subst distinct_set_conv_list [symmetric]) auto |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
57 |
finally show ?thesis . |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
58 |
qed |
4c1347e172b1
moved over material from AFP; most importantly on algebraic numbers and algebraically closed fields
Manuel Eberl <eberlm@in.tum.de>
parents:
79017
diff
changeset
|
59 |
|
58320 | 60 |
end |
61 |
||
62 |
||
60758 | 63 |
subsection \<open>List summation\<close> |
58320 | 64 |
|
65 |
context monoid_add |
|
66 |
begin |
|
67 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
68 |
sublocale sum_list: monoid_list plus 0 |
61776 | 69 |
defines |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
70 |
sum_list = sum_list.F .. |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
71 |
|
58320 | 72 |
end |
73 |
||
74 |
context comm_monoid_add |
|
75 |
begin |
|
76 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
77 |
sublocale sum_list: comm_monoid_list plus 0 |
61566
c3d6e570ccef
Keyword 'rewrites' identifies rewrite morphisms.
ballarin
parents:
61378
diff
changeset
|
78 |
rewrites |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
79 |
"monoid_list.F plus 0 = sum_list" |
58320 | 80 |
proof - |
81 |
show "comm_monoid_list plus 0" .. |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
82 |
then interpret sum_list: comm_monoid_list plus 0 . |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
83 |
from sum_list_def show "monoid_list.F plus 0 = sum_list" by simp |
58101 | 84 |
qed |
85 |
||
64267 | 86 |
sublocale sum: comm_monoid_list_set plus 0 |
61566
c3d6e570ccef
Keyword 'rewrites' identifies rewrite morphisms.
ballarin
parents:
61378
diff
changeset
|
87 |
rewrites |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
88 |
"monoid_list.F plus 0 = sum_list" |
64267 | 89 |
and "comm_monoid_set.F plus 0 = sum" |
58320 | 90 |
proof - |
91 |
show "comm_monoid_list_set plus 0" .. |
|
64267 | 92 |
then interpret sum: comm_monoid_list_set plus 0 . |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
93 |
from sum_list_def show "monoid_list.F plus 0 = sum_list" by simp |
64267 | 94 |
from sum_def show "comm_monoid_set.F plus 0 = sum" by (auto intro: sym) |
58320 | 95 |
qed |
96 |
||
97 |
end |
|
98 |
||
60758 | 99 |
text \<open>Some syntactic sugar for summing a function over a list:\<close> |
81595
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
100 |
|
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
101 |
open_bundle sum_list_syntax |
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
102 |
begin |
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
103 |
|
61955
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61799
diff
changeset
|
104 |
syntax (ASCII) |
80934 | 105 |
"_sum_list" :: "pttrn => 'a list => 'b => 'b" (\<open>(\<open>indent=3 notation=\<open>binder SUM\<close>\<close>SUM _<-_. _)\<close> [0, 51, 10] 10) |
58101 | 106 |
syntax |
80934 | 107 |
"_sum_list" :: "pttrn => 'a list => 'b => 'b" (\<open>(\<open>indent=3 notation=\<open>binder \<Sum>\<close>\<close>\<Sum>_\<leftarrow>_. _)\<close> [0, 51, 10] 10) |
80760 | 108 |
syntax_consts |
109 |
"_sum_list" == sum_list |
|
61799 | 110 |
translations \<comment> \<open>Beware of argument permutation!\<close> |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
111 |
"\<Sum>x\<leftarrow>xs. b" == "CONST sum_list (CONST map (\<lambda>x. b) xs)" |
58101 | 112 |
|
81595
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
113 |
end |
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
114 |
|
70928 | 115 |
context |
116 |
includes lifting_syntax |
|
117 |
begin |
|
118 |
||
119 |
lemma sum_list_transfer [transfer_rule]: |
|
120 |
"(list_all2 A ===> A) sum_list sum_list" |
|
121 |
if [transfer_rule]: "A 0 0" "(A ===> A ===> A) (+) (+)" |
|
122 |
unfolding sum_list.eq_foldr [abs_def] |
|
123 |
by transfer_prover |
|
124 |
||
125 |
end |
|
126 |
||
60758 | 127 |
text \<open>TODO duplicates\<close> |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
128 |
lemmas sum_list_simps = sum_list.Nil sum_list.Cons |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
129 |
lemmas sum_list_append = sum_list.append |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
130 |
lemmas sum_list_rev = sum_list.rev |
58320 | 131 |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
132 |
lemma (in monoid_add) fold_plus_sum_list_rev: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
133 |
"fold plus xs = plus (sum_list (rev xs))" |
58320 | 134 |
proof |
135 |
fix x |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
136 |
have "fold plus xs x = sum_list (rev xs @ [x])" |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
137 |
by (simp add: foldr_conv_fold sum_list.eq_foldr) |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
138 |
also have "\<dots> = sum_list (rev xs) + x" |
58320 | 139 |
by simp |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
140 |
finally show "fold plus xs x = sum_list (rev xs) + x" |
58320 | 141 |
. |
142 |
qed |
|
143 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
144 |
lemma (in comm_monoid_add) sum_list_map_remove1: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
145 |
"x \<in> set xs \<Longrightarrow> sum_list (map f xs) = f x + sum_list (map f (remove1 x xs))" |
58101 | 146 |
by (induct xs) (auto simp add: ac_simps) |
147 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
148 |
lemma (in monoid_add) size_list_conv_sum_list: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
149 |
"size_list f xs = sum_list (map f xs) + size xs" |
58101 | 150 |
by (induct xs) auto |
151 |
||
152 |
lemma (in monoid_add) length_concat: |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
153 |
"length (concat xss) = sum_list (map length xss)" |
58101 | 154 |
by (induct xss) simp_all |
155 |
||
156 |
lemma (in monoid_add) length_product_lists: |
|
69064
5840724b1d71
Prefix form of infix with * on either side no longer needs special treatment
nipkow
parents:
67489
diff
changeset
|
157 |
"length (product_lists xss) = foldr (*) (map length xss) 1" |
58101 | 158 |
proof (induct xss) |
159 |
case (Cons xs xss) then show ?case by (induct xs) (auto simp: length_concat o_def) |
|
160 |
qed simp |
|
161 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
162 |
lemma (in monoid_add) sum_list_map_filter: |
58101 | 163 |
assumes "\<And>x. x \<in> set xs \<Longrightarrow> \<not> P x \<Longrightarrow> f x = 0" |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
164 |
shows "sum_list (map f (filter P xs)) = sum_list (map f xs)" |
58101 | 165 |
using assms by (induct xs) auto |
166 |
||
69231 | 167 |
lemma sum_list_filter_le_nat: |
168 |
fixes f :: "'a \<Rightarrow> nat" |
|
169 |
shows "sum_list (map f (filter P xs)) \<le> sum_list (map f xs)" |
|
170 |
by(induction xs; simp) |
|
171 |
||
64267 | 172 |
lemma (in comm_monoid_add) distinct_sum_list_conv_Sum: |
173 |
"distinct xs \<Longrightarrow> sum_list xs = Sum (set xs)" |
|
58101 | 174 |
by (induct xs) simp_all |
175 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
176 |
lemma sum_list_upt[simp]: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
177 |
"m \<le> n \<Longrightarrow> sum_list [m..<n] = \<Sum> {m..<n}" |
64267 | 178 |
by(simp add: distinct_sum_list_conv_Sum) |
58995 | 179 |
|
66311 | 180 |
context ordered_comm_monoid_add |
181 |
begin |
|
182 |
||
183 |
lemma sum_list_nonneg: "(\<And>x. x \<in> set xs \<Longrightarrow> 0 \<le> x) \<Longrightarrow> 0 \<le> sum_list xs" |
|
184 |
by (induction xs) auto |
|
185 |
||
186 |
lemma sum_list_nonpos: "(\<And>x. x \<in> set xs \<Longrightarrow> x \<le> 0) \<Longrightarrow> sum_list xs \<le> 0" |
|
187 |
by (induction xs) (auto simp: add_nonpos_nonpos) |
|
58101 | 188 |
|
66311 | 189 |
lemma sum_list_nonneg_eq_0_iff: |
190 |
"(\<And>x. x \<in> set xs \<Longrightarrow> 0 \<le> x) \<Longrightarrow> sum_list xs = 0 \<longleftrightarrow> (\<forall>x\<in> set xs. x = 0)" |
|
191 |
by (induction xs) (simp_all add: add_nonneg_eq_0_iff sum_list_nonneg) |
|
192 |
||
193 |
end |
|
194 |
||
195 |
context canonically_ordered_monoid_add |
|
196 |
begin |
|
58101 | 197 |
|
66311 | 198 |
lemma sum_list_eq_0_iff [simp]: |
199 |
"sum_list ns = 0 \<longleftrightarrow> (\<forall>n \<in> set ns. n = 0)" |
|
200 |
by (simp add: sum_list_nonneg_eq_0_iff) |
|
201 |
||
202 |
lemma member_le_sum_list: |
|
203 |
"x \<in> set xs \<Longrightarrow> x \<le> sum_list xs" |
|
204 |
by (induction xs) (auto simp: add_increasing add_increasing2) |
|
58101 | 205 |
|
66311 | 206 |
lemma elem_le_sum_list: |
207 |
"k < size ns \<Longrightarrow> ns ! k \<le> sum_list (ns)" |
|
208 |
by (rule member_le_sum_list) simp |
|
209 |
||
210 |
end |
|
211 |
||
212 |
lemma (in ordered_cancel_comm_monoid_diff) sum_list_update: |
|
213 |
"k < size xs \<Longrightarrow> sum_list (xs[k := x]) = sum_list xs + x - xs ! k" |
|
214 |
apply(induction xs arbitrary:k) |
|
215 |
apply (auto simp: add_ac split: nat.split) |
|
216 |
apply(drule elem_le_sum_list) |
|
217 |
by (simp add: local.add_diff_assoc local.add_increasing) |
|
58101 | 218 |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
219 |
lemma (in monoid_add) sum_list_triv: |
58101 | 220 |
"(\<Sum>x\<leftarrow>xs. r) = of_nat (length xs) * r" |
221 |
by (induct xs) (simp_all add: distrib_right) |
|
222 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
223 |
lemma (in monoid_add) sum_list_0 [simp]: |
58101 | 224 |
"(\<Sum>x\<leftarrow>xs. 0) = 0" |
225 |
by (induct xs) (simp_all add: distrib_right) |
|
226 |
||
61799 | 227 |
text\<open>For non-Abelian groups \<open>xs\<close> needs to be reversed on one side:\<close> |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
228 |
lemma (in ab_group_add) uminus_sum_list_map: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
229 |
"- sum_list (map f xs) = sum_list (map (uminus \<circ> f) xs)" |
58101 | 230 |
by (induct xs) simp_all |
231 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
232 |
lemma (in comm_monoid_add) sum_list_addf: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
233 |
"(\<Sum>x\<leftarrow>xs. f x + g x) = sum_list (map f xs) + sum_list (map g xs)" |
58101 | 234 |
by (induct xs) (simp_all add: algebra_simps) |
235 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
236 |
lemma (in ab_group_add) sum_list_subtractf: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
237 |
"(\<Sum>x\<leftarrow>xs. f x - g x) = sum_list (map f xs) - sum_list (map g xs)" |
58101 | 238 |
by (induct xs) (simp_all add: algebra_simps) |
239 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
240 |
lemma (in semiring_0) sum_list_const_mult: |
58101 | 241 |
"(\<Sum>x\<leftarrow>xs. c * f x) = c * (\<Sum>x\<leftarrow>xs. f x)" |
242 |
by (induct xs) (simp_all add: algebra_simps) |
|
243 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
244 |
lemma (in semiring_0) sum_list_mult_const: |
58101 | 245 |
"(\<Sum>x\<leftarrow>xs. f x * c) = (\<Sum>x\<leftarrow>xs. f x) * c" |
246 |
by (induct xs) (simp_all add: algebra_simps) |
|
247 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
248 |
lemma (in ordered_ab_group_add_abs) sum_list_abs: |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
249 |
"\<bar>sum_list xs\<bar> \<le> sum_list (map abs xs)" |
58101 | 250 |
by (induct xs) (simp_all add: order_trans [OF abs_triangle_ineq]) |
251 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
252 |
lemma sum_list_mono: |
58101 | 253 |
fixes f g :: "'a \<Rightarrow> 'b::{monoid_add, ordered_ab_semigroup_add}" |
254 |
shows "(\<And>x. x \<in> set xs \<Longrightarrow> f x \<le> g x) \<Longrightarrow> (\<Sum>x\<leftarrow>xs. f x) \<le> (\<Sum>x\<leftarrow>xs. g x)" |
|
69231 | 255 |
by (induct xs) (simp, simp add: add_mono) |
256 |
||
257 |
lemma sum_list_strict_mono: |
|
258 |
fixes f g :: "'a \<Rightarrow> 'b::{monoid_add, strict_ordered_ab_semigroup_add}" |
|
259 |
shows "\<lbrakk> xs \<noteq> []; \<And>x. x \<in> set xs \<Longrightarrow> f x < g x \<rbrakk> |
|
260 |
\<Longrightarrow> sum_list (map f xs) < sum_list (map g xs)" |
|
261 |
proof (induction xs) |
|
262 |
case Nil thus ?case by simp |
|
263 |
next |
|
264 |
case C: (Cons _ xs) |
|
265 |
show ?case |
|
266 |
proof (cases xs) |
|
267 |
case Nil thus ?thesis using C.prems by simp |
|
268 |
next |
|
269 |
case Cons thus ?thesis using C by(simp add: add_strict_mono) |
|
270 |
qed |
|
271 |
qed |
|
58101 | 272 |
|
75693 | 273 |
text \<open>A much more general version of this monotonicity lemma |
274 |
can be formulated with multisets and the multiset order\<close> |
|
275 |
||
276 |
lemma sum_list_mono2: fixes xs :: "'a ::ordered_comm_monoid_add list" |
|
277 |
shows "\<lbrakk> length xs = length ys; \<And>i. i < length xs \<longrightarrow> xs!i \<le> ys!i \<rbrakk> |
|
278 |
\<Longrightarrow> sum_list xs \<le> sum_list ys" |
|
279 |
apply(induction xs ys rule: list_induct2) |
|
280 |
by(auto simp: nth_Cons' less_Suc_eq_0_disj imp_ex add_mono) |
|
281 |
||
64267 | 282 |
lemma (in monoid_add) sum_list_distinct_conv_sum_set: |
283 |
"distinct xs \<Longrightarrow> sum_list (map f xs) = sum f (set xs)" |
|
58101 | 284 |
by (induct xs) simp_all |
285 |
||
64267 | 286 |
lemma (in monoid_add) interv_sum_list_conv_sum_set_nat: |
287 |
"sum_list (map f [m..<n]) = sum f (set [m..<n])" |
|
288 |
by (simp add: sum_list_distinct_conv_sum_set) |
|
58101 | 289 |
|
64267 | 290 |
lemma (in monoid_add) interv_sum_list_conv_sum_set_int: |
291 |
"sum_list (map f [k..l]) = sum f (set [k..l])" |
|
292 |
by (simp add: sum_list_distinct_conv_sum_set) |
|
58101 | 293 |
|
69593 | 294 |
text \<open>General equivalence between \<^const>\<open>sum_list\<close> and \<^const>\<open>sum\<close>\<close> |
64267 | 295 |
lemma (in monoid_add) sum_list_sum_nth: |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
296 |
"sum_list xs = (\<Sum> i = 0 ..< length xs. xs ! i)" |
67399 | 297 |
using interv_sum_list_conv_sum_set_nat [of "(!) xs" 0 "length xs"] by (simp add: map_nth) |
58101 | 298 |
|
64267 | 299 |
lemma sum_list_map_eq_sum_count: |
300 |
"sum_list (map f xs) = sum (\<lambda>x. count_list xs x * f x) (set xs)" |
|
59728 | 301 |
proof(induction xs) |
302 |
case (Cons x xs) |
|
303 |
show ?case (is "?l = ?r") |
|
304 |
proof cases |
|
305 |
assume "x \<in> set xs" |
|
60541 | 306 |
have "?l = f x + (\<Sum>x\<in>set xs. count_list xs x * f x)" by (simp add: Cons.IH) |
60758 | 307 |
also have "set xs = insert x (set xs - {x})" using \<open>x \<in> set xs\<close>by blast |
60541 | 308 |
also have "f x + (\<Sum>x\<in>insert x (set xs - {x}). count_list xs x * f x) = ?r" |
64267 | 309 |
by (simp add: sum.insert_remove eq_commute) |
59728 | 310 |
finally show ?thesis . |
311 |
next |
|
312 |
assume "x \<notin> set xs" |
|
313 |
hence "\<And>xa. xa \<in> set xs \<Longrightarrow> x \<noteq> xa" by blast |
|
60758 | 314 |
thus ?thesis by (simp add: Cons.IH \<open>x \<notin> set xs\<close>) |
59728 | 315 |
qed |
316 |
qed simp |
|
317 |
||
64267 | 318 |
lemma sum_list_map_eq_sum_count2: |
59728 | 319 |
assumes "set xs \<subseteq> X" "finite X" |
64267 | 320 |
shows "sum_list (map f xs) = sum (\<lambda>x. count_list xs x * f x) X" |
59728 | 321 |
proof- |
60541 | 322 |
let ?F = "\<lambda>x. count_list xs x * f x" |
64267 | 323 |
have "sum ?F X = sum ?F (set xs \<union> (X - set xs))" |
59728 | 324 |
using Un_absorb1[OF assms(1)] by(simp) |
64267 | 325 |
also have "\<dots> = sum ?F (set xs)" |
59728 | 326 |
using assms(2) |
64267 | 327 |
by(simp add: sum.union_disjoint[OF _ _ Diff_disjoint] del: Un_Diff_cancel) |
328 |
finally show ?thesis by(simp add:sum_list_map_eq_sum_count) |
|
59728 | 329 |
qed |
330 |
||
72545 | 331 |
lemma sum_list_replicate: "sum_list (replicate n c) = of_nat n * c" |
332 |
by(induction n)(auto simp add: distrib_right) |
|
333 |
||
334 |
||
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
335 |
lemma sum_list_nonneg: |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
336 |
"(\<And>x. x \<in> set xs \<Longrightarrow> (x :: 'a :: ordered_comm_monoid_add) \<ge> 0) \<Longrightarrow> sum_list xs \<ge> 0" |
63099
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
61955
diff
changeset
|
337 |
by (induction xs) simp_all |
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
61955
diff
changeset
|
338 |
|
69231 | 339 |
lemma sum_list_Suc: |
340 |
"sum_list (map (\<lambda>x. Suc(f x)) xs) = sum_list (map f xs) + length xs" |
|
341 |
by(induction xs; simp) |
|
342 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
343 |
lemma (in monoid_add) sum_list_map_filter': |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
344 |
"sum_list (map f (filter P xs)) = sum_list (map (\<lambda>x. if P x then f x else 0) xs)" |
63099
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
61955
diff
changeset
|
345 |
by (induction xs) simp_all |
af0e964aad7b
Moved material from AFP/Randomised_Social_Choice to distribution
eberlm
parents:
61955
diff
changeset
|
346 |
|
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
347 |
text \<open>Summation of a strictly ascending sequence with length \<open>n\<close> |
66434
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
348 |
can be upper-bounded by summation over \<open>{0..<n}\<close>.\<close> |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
349 |
|
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
350 |
lemma sorted_wrt_less_sum_mono_lowerbound: |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
351 |
fixes f :: "nat \<Rightarrow> ('b::ordered_comm_monoid_add)" |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
352 |
assumes mono: "\<And>x y. x\<le>y \<Longrightarrow> f x \<le> f y" |
67399 | 353 |
shows "sorted_wrt (<) ns \<Longrightarrow> |
66434
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
354 |
(\<Sum>i\<in>{0..<length ns}. f i) \<le> (\<Sum>i\<leftarrow>ns. f i)" |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
355 |
proof (induction ns rule: rev_induct) |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
356 |
case Nil |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
357 |
then show ?case by simp |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
358 |
next |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
359 |
case (snoc n ns) |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
360 |
have "sum f {0..<length (ns @ [n])} |
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
361 |
= sum f {0..<length ns} + f (length ns)" |
66434
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
362 |
by simp |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
363 |
also have "sum f {0..<length ns} \<le> sum_list (map f ns)" |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
364 |
using snoc by (auto simp: sorted_wrt_append) |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
365 |
also have "length ns \<le> n" |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
366 |
using sorted_wrt_less_idx[OF snoc.prems(1), of "length ns"] by auto |
66434
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
367 |
finally have "sum f {0..<length (ns @ [n])} \<le> sum_list (map f ns) + f n" |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
368 |
using mono add_mono by blast |
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
369 |
thus ?case by simp |
67489
f1ba59ddd9a6
drop redundant cong rules
Lars Hupel <lars.hupel@mytum.de>
parents:
67399
diff
changeset
|
370 |
qed |
66434
5d7e770c7d5d
added sorted_wrt to List; added Data_Structures/Binomial_Heap.thy
nipkow
parents:
66311
diff
changeset
|
371 |
|
58101 | 372 |
|
72024 | 373 |
subsection \<open>Horner sums\<close> |
374 |
||
375 |
context comm_semiring_0 |
|
376 |
begin |
|
377 |
||
378 |
definition horner_sum :: \<open>('b \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'b list \<Rightarrow> 'a\<close> |
|
379 |
where horner_sum_foldr: \<open>horner_sum f a xs = foldr (\<lambda>x b. f x + a * b) xs 0\<close> |
|
380 |
||
381 |
lemma horner_sum_simps [simp]: |
|
382 |
\<open>horner_sum f a [] = 0\<close> |
|
383 |
\<open>horner_sum f a (x # xs) = f x + a * horner_sum f a xs\<close> |
|
384 |
by (simp_all add: horner_sum_foldr) |
|
385 |
||
386 |
lemma horner_sum_eq_sum_funpow: |
|
387 |
\<open>horner_sum f a xs = (\<Sum>n = 0..<length xs. ((*) a ^^ n) (f (xs ! n)))\<close> |
|
388 |
proof (induction xs) |
|
389 |
case Nil |
|
390 |
then show ?case |
|
391 |
by simp |
|
392 |
next |
|
393 |
case (Cons x xs) |
|
394 |
then show ?case |
|
395 |
by (simp add: sum.atLeast0_lessThan_Suc_shift sum_distrib_left del: sum.op_ivl_Suc) |
|
396 |
qed |
|
397 |
||
398 |
end |
|
399 |
||
400 |
context |
|
401 |
includes lifting_syntax |
|
402 |
begin |
|
403 |
||
404 |
lemma horner_sum_transfer [transfer_rule]: |
|
405 |
\<open>((B ===> A) ===> A ===> list_all2 B ===> A) horner_sum horner_sum\<close> |
|
406 |
if [transfer_rule]: \<open>A 0 0\<close> |
|
407 |
and [transfer_rule]: \<open>(A ===> A ===> A) (+) (+)\<close> |
|
408 |
and [transfer_rule]: \<open>(A ===> A ===> A) (*) (*)\<close> |
|
409 |
by (unfold horner_sum_foldr) transfer_prover |
|
410 |
||
411 |
end |
|
412 |
||
413 |
context comm_semiring_1 |
|
414 |
begin |
|
415 |
||
416 |
lemma horner_sum_eq_sum: |
|
417 |
\<open>horner_sum f a xs = (\<Sum>n = 0..<length xs. f (xs ! n) * a ^ n)\<close> |
|
418 |
proof - |
|
419 |
have \<open>(*) a ^^ n = (*) (a ^ n)\<close> for n |
|
420 |
by (induction n) (simp_all add: ac_simps) |
|
421 |
then show ?thesis |
|
422 |
by (simp add: horner_sum_eq_sum_funpow ac_simps) |
|
423 |
qed |
|
424 |
||
72619 | 425 |
lemma horner_sum_append: |
426 |
\<open>horner_sum f a (xs @ ys) = horner_sum f a xs + a ^ length xs * horner_sum f a ys\<close> |
|
427 |
using sum.atLeastLessThan_shift_bounds [of _ 0 \<open>length xs\<close> \<open>length ys\<close>] |
|
428 |
atLeastLessThan_add_Un [of 0 \<open>length xs\<close> \<open>length ys\<close>] |
|
429 |
by (simp add: horner_sum_eq_sum sum_distrib_left sum.union_disjoint ac_simps nth_append power_add) |
|
430 |
||
72024 | 431 |
end |
432 |
||
75662 | 433 |
context linordered_semidom |
434 |
begin |
|
435 |
||
436 |
lemma horner_sum_nonnegative: |
|
437 |
\<open>0 \<le> horner_sum of_bool 2 bs\<close> |
|
438 |
by (induction bs) simp_all |
|
439 |
||
440 |
end |
|
441 |
||
78935
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
442 |
context discrete_linordered_semidom |
75662 | 443 |
begin |
444 |
||
445 |
lemma horner_sum_bound: |
|
446 |
\<open>horner_sum of_bool 2 bs < 2 ^ length bs\<close> |
|
447 |
proof (induction bs) |
|
448 |
case Nil |
|
449 |
then show ?case |
|
450 |
by simp |
|
451 |
next |
|
452 |
case (Cons b bs) |
|
453 |
moreover define a where \<open>a = 2 ^ length bs - horner_sum of_bool 2 bs\<close> |
|
454 |
ultimately have *: \<open>2 ^ length bs = horner_sum of_bool 2 bs + a\<close> |
|
455 |
by simp |
|
78935
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
456 |
have \<open>0 < a\<close> |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
457 |
using Cons * by simp |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
458 |
moreover have \<open>1 \<le> a\<close> |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
459 |
using \<open>0 < a\<close> by (simp add: less_eq_iff_succ_less) |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
460 |
ultimately have \<open>0 + 1 < a + a\<close> |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
461 |
by (rule add_less_le_mono) |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
462 |
then have \<open>1 < a * 2\<close> |
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
463 |
by (simp add: mult_2_right) |
75662 | 464 |
with Cons show ?case |
78935
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
465 |
by (simp add: * algebra_simps) |
75662 | 466 |
qed |
467 |
||
79017 | 468 |
lemma horner_sum_of_bool_2_less: |
469 |
\<open>(horner_sum of_bool 2 bs) < 2 ^ length bs\<close> |
|
470 |
by (fact horner_sum_bound) |
|
471 |
||
75662 | 472 |
end |
473 |
||
474 |
lemma nat_horner_sum [simp]: |
|
475 |
\<open>nat (horner_sum of_bool 2 bs) = horner_sum of_bool 2 bs\<close> |
|
476 |
by (induction bs) (auto simp add: nat_add_distrib horner_sum_nonnegative) |
|
477 |
||
78935
5e788ff7a489
explicit type class for discrete linordered semidoms
haftmann
parents:
75693
diff
changeset
|
478 |
context discrete_linordered_semidom |
75662 | 479 |
begin |
480 |
||
481 |
lemma horner_sum_less_eq_iff_lexordp_eq: |
|
482 |
\<open>horner_sum of_bool 2 bs \<le> horner_sum of_bool 2 cs \<longleftrightarrow> lexordp_eq (rev bs) (rev cs)\<close> |
|
483 |
if \<open>length bs = length cs\<close> |
|
484 |
proof - |
|
485 |
have \<open>horner_sum of_bool 2 (rev bs) \<le> horner_sum of_bool 2 (rev cs) \<longleftrightarrow> lexordp_eq bs cs\<close> |
|
486 |
if \<open>length bs = length cs\<close> for bs cs |
|
487 |
using that proof (induction bs cs rule: list_induct2) |
|
488 |
case Nil |
|
489 |
then show ?case |
|
490 |
by simp |
|
491 |
next |
|
492 |
case (Cons b bs c cs) |
|
493 |
with horner_sum_nonnegative [of \<open>rev bs\<close>] horner_sum_nonnegative [of \<open>rev cs\<close>] |
|
494 |
horner_sum_bound [of \<open>rev bs\<close>] horner_sum_bound [of \<open>rev cs\<close>] |
|
495 |
show ?case |
|
496 |
by (auto simp add: horner_sum_append not_le Cons intro: add_strict_increasing2 add_increasing) |
|
497 |
qed |
|
498 |
from that this [of \<open>rev bs\<close> \<open>rev cs\<close>] show ?thesis |
|
499 |
by simp |
|
500 |
qed |
|
501 |
||
502 |
lemma horner_sum_less_iff_lexordp: |
|
503 |
\<open>horner_sum of_bool 2 bs < horner_sum of_bool 2 cs \<longleftrightarrow> ord_class.lexordp (rev bs) (rev cs)\<close> |
|
504 |
if \<open>length bs = length cs\<close> |
|
505 |
proof - |
|
506 |
have \<open>horner_sum of_bool 2 (rev bs) < horner_sum of_bool 2 (rev cs) \<longleftrightarrow> ord_class.lexordp bs cs\<close> |
|
507 |
if \<open>length bs = length cs\<close> for bs cs |
|
508 |
using that proof (induction bs cs rule: list_induct2) |
|
509 |
case Nil |
|
510 |
then show ?case |
|
511 |
by simp |
|
512 |
next |
|
513 |
case (Cons b bs c cs) |
|
514 |
with horner_sum_nonnegative [of \<open>rev bs\<close>] horner_sum_nonnegative [of \<open>rev cs\<close>] |
|
515 |
horner_sum_bound [of \<open>rev bs\<close>] horner_sum_bound [of \<open>rev cs\<close>] |
|
516 |
show ?case |
|
517 |
by (auto simp add: horner_sum_append not_less Cons intro: add_strict_increasing2 add_increasing) |
|
518 |
qed |
|
519 |
from that this [of \<open>rev bs\<close> \<open>rev cs\<close>] show ?thesis |
|
520 |
by simp |
|
521 |
qed |
|
522 |
||
523 |
end |
|
524 |
||
72024 | 525 |
|
69593 | 526 |
subsection \<open>Further facts about \<^const>\<open>List.n_lists\<close>\<close> |
58101 | 527 |
|
528 |
lemma length_n_lists: "length (List.n_lists n xs) = length xs ^ n" |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
529 |
by (induct n) (auto simp add: comp_def length_concat sum_list_triv) |
58101 | 530 |
|
531 |
lemma distinct_n_lists: |
|
532 |
assumes "distinct xs" |
|
533 |
shows "distinct (List.n_lists n xs)" |
|
534 |
proof (rule card_distinct) |
|
535 |
from assms have card_length: "card (set xs) = length xs" by (rule distinct_card) |
|
536 |
have "card (set (List.n_lists n xs)) = card (set xs) ^ n" |
|
537 |
proof (induct n) |
|
538 |
case 0 then show ?case by simp |
|
539 |
next |
|
540 |
case (Suc n) |
|
541 |
moreover have "card (\<Union>ys\<in>set (List.n_lists n xs). (\<lambda>y. y # ys) ` set xs) |
|
542 |
= (\<Sum>ys\<in>set (List.n_lists n xs). card ((\<lambda>y. y # ys) ` set xs))" |
|
543 |
by (rule card_UN_disjoint) auto |
|
544 |
moreover have "\<And>ys. card ((\<lambda>y. y # ys) ` set xs) = card (set xs)" |
|
545 |
by (rule card_image) (simp add: inj_on_def) |
|
546 |
ultimately show ?case by auto |
|
547 |
qed |
|
548 |
also have "\<dots> = length xs ^ n" by (simp add: card_length) |
|
549 |
finally show "card (set (List.n_lists n xs)) = length (List.n_lists n xs)" |
|
550 |
by (simp add: length_n_lists) |
|
551 |
qed |
|
552 |
||
553 |
||
60758 | 554 |
subsection \<open>Tools setup\<close> |
58101 | 555 |
|
64267 | 556 |
lemmas sum_code = sum.set_conv_list |
58320 | 557 |
|
64267 | 558 |
lemma sum_set_upto_conv_sum_list_int [code_unfold]: |
559 |
"sum f (set [i..j::int]) = sum_list (map f [i..j])" |
|
560 |
by (simp add: interv_sum_list_conv_sum_set_int) |
|
58101 | 561 |
|
64267 | 562 |
lemma sum_set_upt_conv_sum_list_nat [code_unfold]: |
563 |
"sum f (set [m..<n]) = sum_list (map f [m..<n])" |
|
564 |
by (simp add: interv_sum_list_conv_sum_set_nat) |
|
58101 | 565 |
|
58368 | 566 |
|
60758 | 567 |
subsection \<open>List product\<close> |
58368 | 568 |
|
569 |
context monoid_mult |
|
570 |
begin |
|
571 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
572 |
sublocale prod_list: monoid_list times 1 |
61776 | 573 |
defines |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
574 |
prod_list = prod_list.F .. |
58368 | 575 |
|
58320 | 576 |
end |
58368 | 577 |
|
578 |
context comm_monoid_mult |
|
579 |
begin |
|
580 |
||
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
581 |
sublocale prod_list: comm_monoid_list times 1 |
61566
c3d6e570ccef
Keyword 'rewrites' identifies rewrite morphisms.
ballarin
parents:
61378
diff
changeset
|
582 |
rewrites |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
583 |
"monoid_list.F times 1 = prod_list" |
58368 | 584 |
proof - |
585 |
show "comm_monoid_list times 1" .. |
|
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
586 |
then interpret prod_list: comm_monoid_list times 1 . |
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
587 |
from prod_list_def show "monoid_list.F times 1 = prod_list" by simp |
58368 | 588 |
qed |
589 |
||
64272 | 590 |
sublocale prod: comm_monoid_list_set times 1 |
61566
c3d6e570ccef
Keyword 'rewrites' identifies rewrite morphisms.
ballarin
parents:
61378
diff
changeset
|
591 |
rewrites |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
592 |
"monoid_list.F times 1 = prod_list" |
64272 | 593 |
and "comm_monoid_set.F times 1 = prod" |
58368 | 594 |
proof - |
595 |
show "comm_monoid_list_set times 1" .. |
|
64272 | 596 |
then interpret prod: comm_monoid_list_set times 1 . |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
597 |
from prod_list_def show "monoid_list.F times 1 = prod_list" by simp |
64272 | 598 |
from prod_def show "comm_monoid_set.F times 1 = prod" by (auto intro: sym) |
58368 | 599 |
qed |
600 |
||
601 |
end |
|
602 |
||
60758 | 603 |
text \<open>Some syntactic sugar:\<close> |
58368 | 604 |
|
81595
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
605 |
open_bundle prod_list_syntax |
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
606 |
begin |
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
607 |
|
61955
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61799
diff
changeset
|
608 |
syntax (ASCII) |
80934 | 609 |
"_prod_list" :: "pttrn => 'a list => 'b => 'b" (\<open>(\<open>indent=3 notation=\<open>binder PROD\<close>\<close>PROD _<-_. _)\<close> [0, 51, 10] 10) |
61955
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61799
diff
changeset
|
610 |
syntax |
80934 | 611 |
"_prod_list" :: "pttrn => 'a list => 'b => 'b" (\<open>(\<open>indent=3 notation=\<open>binder \<Prod>\<close>\<close>\<Prod>_\<leftarrow>_. _)\<close> [0, 51, 10] 10) |
80760 | 612 |
syntax_consts |
613 |
"_prod_list" \<rightleftharpoons> prod_list |
|
61799 | 614 |
translations \<comment> \<open>Beware of argument permutation!\<close> |
63882
018998c00003
renamed listsum -> sum_list, listprod ~> prod_list
nipkow
parents:
63343
diff
changeset
|
615 |
"\<Prod>x\<leftarrow>xs. b" \<rightleftharpoons> "CONST prod_list (CONST map (\<lambda>x. b) xs)" |
58368 | 616 |
|
81595
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
617 |
end |
ed264056f5dc
more syntax bundles, e.g. to explore terms without notation;
wenzelm
parents:
80934
diff
changeset
|
618 |
|
70928 | 619 |
context |
620 |
includes lifting_syntax |
|
621 |
begin |
|
622 |
||
623 |
lemma prod_list_transfer [transfer_rule]: |
|
624 |
"(list_all2 A ===> A) prod_list prod_list" |
|
625 |
if [transfer_rule]: "A 1 1" "(A ===> A ===> A) (*) (*)" |
|
626 |
unfolding prod_list.eq_foldr [abs_def] |
|
627 |
by transfer_prover |
|
628 |
||
58368 | 629 |
end |
70928 | 630 |
|
631 |
lemma prod_list_zero_iff: |
|
632 |
"prod_list xs = 0 \<longleftrightarrow> (0 :: 'a :: {semiring_no_zero_divisors, semiring_1}) \<in> set xs" |
|
633 |
by (induction xs) simp_all |
|
634 |
||
635 |
end |