author | wenzelm |
Sat, 16 Jul 2016 12:11:02 +0200 | |
changeset 63516 | 76492eaf3dc1 |
parent 62390 | 842917225d56 |
child 63540 | f8652d0534fa |
permissions | -rw-r--r-- |
59349 | 1 |
(* Author: Florian Haftmann, TU Muenchen *) |
51174 | 2 |
|
60500 | 3 |
section \<open>Common discrete functions\<close> |
51174 | 4 |
|
5 |
theory Discrete |
|
6 |
imports Main |
|
7 |
begin |
|
8 |
||
60500 | 9 |
subsection \<open>Discrete logarithm\<close> |
51174 | 10 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
60500
diff
changeset
|
11 |
context |
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
60500
diff
changeset
|
12 |
begin |
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
60500
diff
changeset
|
13 |
|
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
60500
diff
changeset
|
14 |
qualified fun log :: "nat \<Rightarrow> nat" |
59349 | 15 |
where [simp del]: "log n = (if n < 2 then 0 else Suc (log (n div 2)))" |
51174 | 16 |
|
61831 | 17 |
lemma log_induct [consumes 1, case_names one double]: |
18 |
fixes n :: nat |
|
19 |
assumes "n > 0" |
|
20 |
assumes one: "P 1" |
|
21 |
assumes double: "\<And>n. n \<ge> 2 \<Longrightarrow> P (n div 2) \<Longrightarrow> P n" |
|
22 |
shows "P n" |
|
61975 | 23 |
using \<open>n > 0\<close> proof (induct n rule: log.induct) |
61831 | 24 |
fix n |
25 |
assume "\<not> n < 2 \<Longrightarrow> |
|
26 |
0 < n div 2 \<Longrightarrow> P (n div 2)" |
|
27 |
then have *: "n \<ge> 2 \<Longrightarrow> P (n div 2)" by simp |
|
28 |
assume "n > 0" |
|
29 |
show "P n" |
|
30 |
proof (cases "n = 1") |
|
31 |
case True with one show ?thesis by simp |
|
32 |
next |
|
61975 | 33 |
case False with \<open>n > 0\<close> have "n \<ge> 2" by auto |
61831 | 34 |
moreover with * have "P (n div 2)" . |
35 |
ultimately show ?thesis by (rule double) |
|
36 |
qed |
|
37 |
qed |
|
38 |
||
59349 | 39 |
lemma log_zero [simp]: "log 0 = 0" |
51174 | 40 |
by (simp add: log.simps) |
41 |
||
59349 | 42 |
lemma log_one [simp]: "log 1 = 0" |
51174 | 43 |
by (simp add: log.simps) |
44 |
||
59349 | 45 |
lemma log_Suc_zero [simp]: "log (Suc 0) = 0" |
51174 | 46 |
using log_one by simp |
47 |
||
59349 | 48 |
lemma log_rec: "n \<ge> 2 \<Longrightarrow> log n = Suc (log (n div 2))" |
51174 | 49 |
by (simp add: log.simps) |
50 |
||
59349 | 51 |
lemma log_twice [simp]: "n \<noteq> 0 \<Longrightarrow> log (2 * n) = Suc (log n)" |
51174 | 52 |
by (simp add: log_rec) |
53 |
||
59349 | 54 |
lemma log_half [simp]: "log (n div 2) = log n - 1" |
51174 | 55 |
proof (cases "n < 2") |
56 |
case True |
|
57 |
then have "n = 0 \<or> n = 1" by arith |
|
58 |
then show ?thesis by (auto simp del: One_nat_def) |
|
59 |
next |
|
59349 | 60 |
case False |
61 |
then show ?thesis by (simp add: log_rec) |
|
51174 | 62 |
qed |
63 |
||
59349 | 64 |
lemma log_exp [simp]: "log (2 ^ n) = n" |
51174 | 65 |
by (induct n) simp_all |
66 |
||
59349 | 67 |
lemma log_mono: "mono log" |
51174 | 68 |
proof |
69 |
fix m n :: nat |
|
70 |
assume "m \<le> n" |
|
71 |
then show "log m \<le> log n" |
|
72 |
proof (induct m arbitrary: n rule: log.induct) |
|
73 |
case (1 m) |
|
74 |
then have mn2: "m div 2 \<le> n div 2" by arith |
|
75 |
show "log m \<le> log n" |
|
61831 | 76 |
proof (cases "m \<ge> 2") |
77 |
case False |
|
51174 | 78 |
then have "m = 0 \<or> m = 1" by arith |
79 |
then show ?thesis by (auto simp del: One_nat_def) |
|
80 |
next |
|
61831 | 81 |
case True then have "\<not> m < 2" by simp |
82 |
with mn2 have "n \<ge> 2" by arith |
|
83 |
from True have m2_0: "m div 2 \<noteq> 0" by arith |
|
51174 | 84 |
with mn2 have n2_0: "n div 2 \<noteq> 0" by arith |
61975 | 85 |
from \<open>\<not> m < 2\<close> "1.hyps" mn2 have "log (m div 2) \<le> log (n div 2)" by blast |
51174 | 86 |
with m2_0 n2_0 have "log (2 * (m div 2)) \<le> log (2 * (n div 2))" by simp |
60500 | 87 |
with m2_0 n2_0 \<open>m \<ge> 2\<close> \<open>n \<ge> 2\<close> show ?thesis by (simp only: log_rec [of m] log_rec [of n]) simp |
51174 | 88 |
qed |
89 |
qed |
|
90 |
qed |
|
91 |
||
61831 | 92 |
lemma log_exp2_le: |
93 |
assumes "n > 0" |
|
94 |
shows "2 ^ log n \<le> n" |
|
63516 | 95 |
using assms |
96 |
proof (induct n rule: log_induct) |
|
97 |
case one |
|
98 |
then show ?case by simp |
|
61831 | 99 |
next |
63516 | 100 |
case (double n) |
61831 | 101 |
with log_mono have "log n \<ge> Suc 0" |
102 |
by (simp add: log.simps) |
|
103 |
assume "2 ^ log (n div 2) \<le> n div 2" |
|
61975 | 104 |
with \<open>n \<ge> 2\<close> have "2 ^ (log n - Suc 0) \<le> n div 2" by simp |
61831 | 105 |
then have "2 ^ (log n - Suc 0) * 2 ^ 1 \<le> n div 2 * 2" by simp |
61975 | 106 |
with \<open>log n \<ge> Suc 0\<close> have "2 ^ log n \<le> n div 2 * 2" |
61831 | 107 |
unfolding power_add [symmetric] by simp |
108 |
also have "n div 2 * 2 \<le> n" by (cases "even n") simp_all |
|
63516 | 109 |
finally show ?case . |
61831 | 110 |
qed |
111 |
||
51174 | 112 |
|
60500 | 113 |
subsection \<open>Discrete square root\<close> |
51174 | 114 |
|
61115
3a4400985780
modernized name space management -- more uniform qualification;
wenzelm
parents:
60500
diff
changeset
|
115 |
qualified definition sqrt :: "nat \<Rightarrow> nat" |
59349 | 116 |
where "sqrt n = Max {m. m\<^sup>2 \<le> n}" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
117 |
|
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
118 |
lemma sqrt_aux: |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
119 |
fixes n :: nat |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
120 |
shows "finite {m. m\<^sup>2 \<le> n}" and "{m. m\<^sup>2 \<le> n} \<noteq> {}" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
121 |
proof - |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
122 |
{ fix m |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
123 |
assume "m\<^sup>2 \<le> n" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
124 |
then have "m \<le> n" |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
125 |
by (cases m) (simp_all add: power2_eq_square) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
126 |
} note ** = this |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
127 |
then have "{m. m\<^sup>2 \<le> n} \<subseteq> {m. m \<le> n}" by auto |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
128 |
then show "finite {m. m\<^sup>2 \<le> n}" by (rule finite_subset) rule |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
129 |
have "0\<^sup>2 \<le> n" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
130 |
then show *: "{m. m\<^sup>2 \<le> n} \<noteq> {}" by blast |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
131 |
qed |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
132 |
|
59349 | 133 |
lemma [code]: "sqrt n = Max (Set.filter (\<lambda>m. m\<^sup>2 \<le> n) {0..n})" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
134 |
proof - |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
135 |
from power2_nat_le_imp_le [of _ n] have "{m. m \<le> n \<and> m\<^sup>2 \<le> n} = {m. m\<^sup>2 \<le> n}" by auto |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
136 |
then show ?thesis by (simp add: sqrt_def Set.filter_def) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
137 |
qed |
51174 | 138 |
|
59349 | 139 |
lemma sqrt_inverse_power2 [simp]: "sqrt (n\<^sup>2) = n" |
51174 | 140 |
proof - |
141 |
have "{m. m \<le> n} \<noteq> {}" by auto |
|
142 |
then have "Max {m. m \<le> n} \<le> n" by auto |
|
143 |
then show ?thesis |
|
144 |
by (auto simp add: sqrt_def power2_nat_le_eq_le intro: antisym) |
|
145 |
qed |
|
146 |
||
59349 | 147 |
lemma sqrt_zero [simp]: "sqrt 0 = 0" |
58787 | 148 |
using sqrt_inverse_power2 [of 0] by simp |
149 |
||
59349 | 150 |
lemma sqrt_one [simp]: "sqrt 1 = 1" |
58787 | 151 |
using sqrt_inverse_power2 [of 1] by simp |
152 |
||
59349 | 153 |
lemma mono_sqrt: "mono sqrt" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
154 |
proof |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
155 |
fix m n :: nat |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
156 |
have *: "0 * 0 \<le> m" by simp |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
157 |
assume "m \<le> n" |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
158 |
then show "sqrt m \<le> sqrt n" |
60500 | 159 |
by (auto intro!: Max_mono \<open>0 * 0 \<le> m\<close> finite_less_ub simp add: power2_eq_square sqrt_def) |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
160 |
qed |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
161 |
|
59349 | 162 |
lemma sqrt_greater_zero_iff [simp]: "sqrt n > 0 \<longleftrightarrow> n > 0" |
51174 | 163 |
proof - |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
164 |
have *: "0 < Max {m. m\<^sup>2 \<le> n} \<longleftrightarrow> (\<exists>a\<in>{m. m\<^sup>2 \<le> n}. 0 < a)" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
165 |
by (rule Max_gr_iff) (fact sqrt_aux)+ |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
166 |
show ?thesis |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
167 |
proof |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
168 |
assume "0 < sqrt n" |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
169 |
then have "0 < Max {m. m\<^sup>2 \<le> n}" by (simp add: sqrt_def) |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
170 |
with * show "0 < n" by (auto dest: power2_nat_le_imp_le) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
171 |
next |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
172 |
assume "0 < n" |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
173 |
then have "1\<^sup>2 \<le> n \<and> 0 < (1::nat)" by simp |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
174 |
then have "\<exists>q. q\<^sup>2 \<le> n \<and> 0 < q" .. |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
175 |
with * have "0 < Max {m. m\<^sup>2 \<le> n}" by blast |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
176 |
then show "0 < sqrt n" by (simp add: sqrt_def) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
177 |
qed |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
178 |
qed |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
179 |
|
59349 | 180 |
lemma sqrt_power2_le [simp]: "(sqrt n)\<^sup>2 \<le> n" (* FIXME tune proof *) |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
181 |
proof (cases "n > 0") |
58787 | 182 |
case False then show ?thesis by simp |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
183 |
next |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
184 |
case True then have "sqrt n > 0" by simp |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
185 |
then have "mono (times (Max {m. m\<^sup>2 \<le> n}))" by (auto intro: mono_times_nat simp add: sqrt_def) |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51263
diff
changeset
|
186 |
then have *: "Max {m. m\<^sup>2 \<le> n} * Max {m. m\<^sup>2 \<le> n} = Max (times (Max {m. m\<^sup>2 \<le> n}) ` {m. m\<^sup>2 \<le> n})" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
187 |
using sqrt_aux [of n] by (rule mono_Max_commute) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
188 |
have "Max (op * (Max {m. m * m \<le> n}) ` {m. m * m \<le> n}) \<le> n" |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
189 |
apply (subst Max_le_iff) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
190 |
apply (metis (mono_tags) finite_imageI finite_less_ub le_square) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
191 |
apply simp |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
192 |
apply (metis le0 mult_0_right) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
193 |
apply auto |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
194 |
proof - |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
195 |
fix q |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
196 |
assume "q * q \<le> n" |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
197 |
show "Max {m. m * m \<le> n} * q \<le> n" |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
198 |
proof (cases "q > 0") |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
199 |
case False then show ?thesis by simp |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
200 |
next |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
201 |
case True then have "mono (times q)" by (rule mono_times_nat) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
202 |
then have "q * Max {m. m * m \<le> n} = Max (times q ` {m. m * m \<le> n})" |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
203 |
using sqrt_aux [of n] by (auto simp add: power2_eq_square intro: mono_Max_commute) |
57514
bdc2c6b40bf2
prefer ac_simps collections over separate name bindings for add and mult
haftmann
parents:
53015
diff
changeset
|
204 |
then have "Max {m. m * m \<le> n} * q = Max (times q ` {m. m * m \<le> n})" by (simp add: ac_simps) |
59349 | 205 |
then show ?thesis |
206 |
apply simp |
|
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
207 |
apply (subst Max_le_iff) |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
208 |
apply auto |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
209 |
apply (metis (mono_tags) finite_imageI finite_less_ub le_square) |
60500 | 210 |
apply (metis \<open>q * q \<le> n\<close>) |
211 |
apply (metis \<open>q * q \<le> n\<close> le_cases mult_le_mono1 mult_le_mono2 order_trans) |
|
59349 | 212 |
done |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
213 |
qed |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
214 |
qed |
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
215 |
with * show ?thesis by (simp add: sqrt_def power2_eq_square) |
51174 | 216 |
qed |
217 |
||
59349 | 218 |
lemma sqrt_le: "sqrt n \<le> n" |
51263
31e786e0e6a7
turned example into library for comparing growth of functions
haftmann
parents:
51174
diff
changeset
|
219 |
using sqrt_aux [of n] by (auto simp add: sqrt_def intro: power2_nat_le_imp_le) |
51174 | 220 |
|
221 |
end |
|
222 |
||
62390 | 223 |
end |