| author | wenzelm | 
| Wed, 05 Jul 2023 15:01:46 +0200 | |
| changeset 78255 | 3e11f510b3f6 | 
| parent 78131 | 1cadc477f644 | 
| child 82338 | 1eb12389c499 | 
| permissions | -rw-r--r-- | 
| 52265 | 1 | (* Title: HOL/Limits.thy | 
| 51526 | 2 | Author: Brian Huffman | 
| 3 | Author: Jacques D. Fleuriot, University of Cambridge | |
| 4 | Author: Lawrence C Paulson | |
| 5 | Author: Jeremy Avigad | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 6 | *) | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 7 | |
| 60758 | 8 | section \<open>Limits on Real Vector Spaces\<close> | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 9 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 10 | theory Limits | 
| 63546 | 11 | imports Real_Vector_Spaces | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 12 | begin | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 13 | |
| 73795 | 14 | lemma range_mult [simp]: | 
| 15 |   fixes a::"real" shows "range ((*) a) = (if a=0 then {0} else UNIV)"
 | |
| 16 | by (simp add: surj_def) (meson dvdE dvd_field_iff) | |
| 17 | ||
| 18 | ||
| 60758 | 19 | subsection \<open>Filter going to infinity norm\<close> | 
| 51526 | 20 | |
| 63546 | 21 | definition at_infinity :: "'a::real_normed_vector filter" | 
| 22 |   where "at_infinity = (INF r. principal {x. r \<le> norm x})"
 | |
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 23 | |
| 57276 | 24 | lemma eventually_at_infinity: "eventually P at_infinity \<longleftrightarrow> (\<exists>b. \<forall>x. b \<le> norm x \<longrightarrow> P x)" | 
| 25 | unfolding at_infinity_def | |
| 26 | by (subst eventually_INF_base) | |
| 27 | (auto simp: subset_eq eventually_principal intro!: exI[of _ "max a b" for a b]) | |
| 31392 | 28 | |
| 62379 
340738057c8c
An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!
 paulson <lp15@cam.ac.uk> parents: 
62369diff
changeset | 29 | corollary eventually_at_infinity_pos: | 
| 63546 | 30 | "eventually p at_infinity \<longleftrightarrow> (\<exists>b. 0 < b \<and> (\<forall>x. norm x \<ge> b \<longrightarrow> p x))" | 
| 68614 | 31 | unfolding eventually_at_infinity | 
| 32 | by (meson le_less_trans norm_ge_zero not_le zero_less_one) | |
| 63546 | 33 | |
| 34 | lemma at_infinity_eq_at_top_bot: "(at_infinity :: real filter) = sup at_top at_bot" | |
| 68614 | 35 | proof - | 
| 36 | have 1: "\<lbrakk>\<forall>n\<ge>u. A n; \<forall>n\<le>v. A n\<rbrakk> | |
| 37 | \<Longrightarrow> \<exists>b. \<forall>x. b \<le> \<bar>x\<bar> \<longrightarrow> A x" for A and u v::real | |
| 38 | by (rule_tac x="max (- v) u" in exI) (auto simp: abs_real_def) | |
| 39 | have 2: "\<forall>x. u \<le> \<bar>x\<bar> \<longrightarrow> A x \<Longrightarrow> \<exists>N. \<forall>n\<ge>N. A n" for A and u::real | |
| 40 | by (meson abs_less_iff le_cases less_le_not_le) | |
| 41 | have 3: "\<forall>x. u \<le> \<bar>x\<bar> \<longrightarrow> A x \<Longrightarrow> \<exists>N. \<forall>n\<le>N. A n" for A and u::real | |
| 42 | by (metis (full_types) abs_ge_self abs_minus_cancel le_minus_iff order_trans) | |
| 43 | show ?thesis | |
| 68615 | 44 | by (auto simp: filter_eq_iff eventually_sup eventually_at_infinity | 
| 68614 | 45 | eventually_at_top_linorder eventually_at_bot_linorder intro: 1 2 3) | 
| 46 | qed | |
| 50325 | 47 | |
| 57276 | 48 | lemma at_top_le_at_infinity: "at_top \<le> (at_infinity :: real filter)" | 
| 50325 | 49 | unfolding at_infinity_eq_at_top_bot by simp | 
| 50 | ||
| 57276 | 51 | lemma at_bot_le_at_infinity: "at_bot \<le> (at_infinity :: real filter)" | 
| 50325 | 52 | unfolding at_infinity_eq_at_top_bot by simp | 
| 53 | ||
| 63546 | 54 | lemma filterlim_at_top_imp_at_infinity: "filterlim f at_top F \<Longrightarrow> filterlim f at_infinity F" | 
| 55 | for f :: "_ \<Rightarrow> real" | |
| 57275 
0ddb5b755cdc
moved lemmas from the proof of the Central Limit Theorem by Jeremy Avigad and Luke Serafin
 hoelzl parents: 
56541diff
changeset | 56 | by (rule filterlim_mono[OF _ at_top_le_at_infinity order_refl]) | 
| 
0ddb5b755cdc
moved lemmas from the proof of the Central Limit Theorem by Jeremy Avigad and Luke Serafin
 hoelzl parents: 
56541diff
changeset | 57 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 58 | lemma filterlim_real_at_infinity_sequentially: "filterlim real at_infinity sequentially" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 59 | by (simp add: filterlim_at_top_imp_at_infinity filterlim_real_sequentially) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 60 | |
| 63546 | 61 | lemma lim_infinity_imp_sequentially: "(f \<longlongrightarrow> l) at_infinity \<Longrightarrow> ((\<lambda>n. f(n)) \<longlongrightarrow> l) sequentially" | 
| 62 | by (simp add: filterlim_at_top_imp_at_infinity filterlim_compose filterlim_real_sequentially) | |
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 63 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 64 | |
| 60758 | 65 | subsubsection \<open>Boundedness\<close> | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 66 | |
| 63546 | 67 | definition Bfun :: "('a \<Rightarrow> 'b::metric_space) \<Rightarrow> 'a filter \<Rightarrow> bool"
 | 
| 68 | where Bfun_metric_def: "Bfun f F = (\<exists>y. \<exists>K>0. eventually (\<lambda>x. dist (f x) y \<le> K) F)" | |
| 69 | ||
| 70 | abbreviation Bseq :: "(nat \<Rightarrow> 'a::metric_space) \<Rightarrow> bool" | |
| 71 | where "Bseq X \<equiv> Bfun X sequentially" | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 72 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 73 | lemma Bseq_conv_Bfun: "Bseq X \<longleftrightarrow> Bfun X sequentially" .. | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 74 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 75 | lemma Bseq_ignore_initial_segment: "Bseq X \<Longrightarrow> Bseq (\<lambda>n. X (n + k))" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 76 | unfolding Bfun_metric_def by (subst eventually_sequentially_seg) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 77 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 78 | lemma Bseq_offset: "Bseq (\<lambda>n. X (n + k)) \<Longrightarrow> Bseq X" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 79 | unfolding Bfun_metric_def by (subst (asm) eventually_sequentially_seg) | 
| 31355 | 80 | |
| 63546 | 81 | lemma Bfun_def: "Bfun f F \<longleftrightarrow> (\<exists>K>0. eventually (\<lambda>x. norm (f x) \<le> K) F)" | 
| 51474 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 82 | unfolding Bfun_metric_def norm_conv_dist | 
| 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 83 | proof safe | 
| 63546 | 84 | fix y K | 
| 85 | assume K: "0 < K" and *: "eventually (\<lambda>x. dist (f x) y \<le> K) F" | |
| 51474 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 86 | moreover have "eventually (\<lambda>x. dist (f x) 0 \<le> dist (f x) y + dist 0 y) F" | 
| 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 87 | by (intro always_eventually) (metis dist_commute dist_triangle) | 
| 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 88 | with * have "eventually (\<lambda>x. dist (f x) 0 \<le> K + dist 0 y) F" | 
| 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 89 | by eventually_elim auto | 
| 60758 | 90 | with \<open>0 < K\<close> show "\<exists>K>0. eventually (\<lambda>x. dist (f x) 0 \<le> K) F" | 
| 51474 
1e9e68247ad1
generalize Bfun and Bseq to metric spaces; Bseq is an abbreviation for Bfun
 hoelzl parents: 
51472diff
changeset | 91 | by (intro exI[of _ "K + dist 0 y"] add_pos_nonneg conjI zero_le_dist) auto | 
| 62379 
340738057c8c
An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!
 paulson <lp15@cam.ac.uk> parents: 
62369diff
changeset | 92 | qed (force simp del: norm_conv_dist [symmetric]) | 
| 31355 | 93 | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 94 | lemma BfunI: | 
| 63546 | 95 | assumes K: "eventually (\<lambda>x. norm (f x) \<le> K) F" | 
| 96 | shows "Bfun f F" | |
| 97 | unfolding Bfun_def | |
| 31355 | 98 | proof (intro exI conjI allI) | 
| 99 | show "0 < max K 1" by simp | |
| 44195 | 100 | show "eventually (\<lambda>x. norm (f x) \<le> max K 1) F" | 
| 63546 | 101 | using K by (rule eventually_mono) simp | 
| 31355 | 102 | qed | 
| 103 | ||
| 104 | lemma BfunE: | |
| 44195 | 105 | assumes "Bfun f F" | 
| 106 | obtains B where "0 < B" and "eventually (\<lambda>x. norm (f x) \<le> B) F" | |
| 63546 | 107 | using assms unfolding Bfun_def by blast | 
| 31355 | 108 | |
| 68614 | 109 | lemma Cauchy_Bseq: | 
| 110 | assumes "Cauchy X" shows "Bseq X" | |
| 111 | proof - | |
| 112 | have "\<exists>y K. 0 < K \<and> (\<exists>N. \<forall>n\<ge>N. dist (X n) y \<le> K)" | |
| 113 | if "\<And>m n. \<lbrakk>m \<ge> M; n \<ge> M\<rbrakk> \<Longrightarrow> dist (X m) (X n) < 1" for M | |
| 114 | by (meson order.order_iff_strict that zero_less_one) | |
| 115 | with assms show ?thesis | |
| 116 | by (force simp: Cauchy_def Bfun_metric_def eventually_sequentially) | |
| 117 | qed | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 118 | |
| 60758 | 119 | subsubsection \<open>Bounded Sequences\<close> | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 120 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 121 | lemma BseqI': "(\<And>n. norm (X n) \<le> K) \<Longrightarrow> Bseq X" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 122 | by (intro BfunI) (auto simp: eventually_sequentially) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 123 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 124 | lemma Bseq_def: "Bseq X \<longleftrightarrow> (\<exists>K>0. \<forall>n. norm (X n) \<le> K)" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 125 | unfolding Bfun_def eventually_sequentially | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 126 | proof safe | 
| 63546 | 127 | fix N K | 
| 128 | assume "0 < K" "\<forall>n\<ge>N. norm (X n) \<le> K" | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 129 | then show "\<exists>K>0. \<forall>n. norm (X n) \<le> K" | 
| 54863 
82acc20ded73
prefer more canonical names for lemmas on min/max
 haftmann parents: 
54263diff
changeset | 130 |     by (intro exI[of _ "max (Max (norm ` X ` {..N})) K"] max.strict_coboundedI2)
 | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 131 | (auto intro!: imageI not_less[where 'a=nat, THEN iffD1] Max_ge simp: le_max_iff_disj) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 132 | qed auto | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 133 | |
| 63546 | 134 | lemma BseqE: "Bseq X \<Longrightarrow> (\<And>K. 0 < K \<Longrightarrow> \<forall>n. norm (X n) \<le> K \<Longrightarrow> Q) \<Longrightarrow> Q" | 
| 135 | unfolding Bseq_def by auto | |
| 136 | ||
| 137 | lemma BseqD: "Bseq X \<Longrightarrow> \<exists>K. 0 < K \<and> (\<forall>n. norm (X n) \<le> K)" | |
| 138 | by (simp add: Bseq_def) | |
| 139 | ||
| 140 | lemma BseqI: "0 < K \<Longrightarrow> \<forall>n. norm (X n) \<le> K \<Longrightarrow> Bseq X" | |
| 68615 | 141 | by (auto simp: Bseq_def) | 
| 63546 | 142 | |
| 143 | lemma Bseq_bdd_above: "Bseq X \<Longrightarrow> bdd_above (range X)" | |
| 144 | for X :: "nat \<Rightarrow> real" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 145 | proof (elim BseqE, intro bdd_aboveI2) | 
| 63546 | 146 | fix K n | 
| 147 | assume "0 < K" "\<forall>n. norm (X n) \<le> K" | |
| 148 | then show "X n \<le> K" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 149 | by (auto elim!: allE[of _ n]) | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 150 | qed | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 151 | |
| 63546 | 152 | lemma Bseq_bdd_above': "Bseq X \<Longrightarrow> bdd_above (range (\<lambda>n. norm (X n)))" | 
| 153 | for X :: "nat \<Rightarrow> 'a :: real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 154 | proof (elim BseqE, intro bdd_aboveI2) | 
| 63546 | 155 | fix K n | 
| 156 | assume "0 < K" "\<forall>n. norm (X n) \<le> K" | |
| 157 | then show "norm (X n) \<le> K" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 158 | by (auto elim!: allE[of _ n]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 159 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 160 | |
| 63546 | 161 | lemma Bseq_bdd_below: "Bseq X \<Longrightarrow> bdd_below (range X)" | 
| 162 | for X :: "nat \<Rightarrow> real" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 163 | proof (elim BseqE, intro bdd_belowI2) | 
| 63546 | 164 | fix K n | 
| 165 | assume "0 < K" "\<forall>n. norm (X n) \<le> K" | |
| 166 | then show "- K \<le> X n" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 167 | by (auto elim!: allE[of _ n]) | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 168 | qed | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 169 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 170 | lemma Bseq_eventually_mono: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 171 | assumes "eventually (\<lambda>n. norm (f n) \<le> norm (g n)) sequentially" "Bseq g" | 
| 63546 | 172 | shows "Bseq f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 173 | proof - | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 174 | from assms(2) obtain K where "0 < K" and "eventually (\<lambda>n. norm (g n) \<le> K) sequentially" | 
| 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 175 | unfolding Bfun_def by fast | 
| 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 176 | with assms(1) have "eventually (\<lambda>n. norm (f n) \<le> K) sequentially" | 
| 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 177 | by (fast elim: eventually_elim2 order_trans) | 
| 69272 | 178 | with \<open>0 < K\<close> show "Bseq f" | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 179 | unfolding Bfun_def by fast | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 180 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 181 | |
| 63546 | 182 | lemma lemma_NBseq_def: "(\<exists>K > 0. \<forall>n. norm (X n) \<le> K) \<longleftrightarrow> (\<exists>N. \<forall>n. norm (X n) \<le> real(Suc N))" | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 183 | proof safe | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 184 | fix K :: real | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 185 | from reals_Archimedean2 obtain n :: nat where "K < real n" .. | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 186 | then have "K \<le> real (Suc n)" by auto | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 187 | moreover assume "\<forall>m. norm (X m) \<le> K" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 188 | ultimately have "\<forall>m. norm (X m) \<le> real (Suc n)" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 189 | by (blast intro: order_trans) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 190 | then show "\<exists>N. \<forall>n. norm (X n) \<le> real (Suc N)" .. | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 191 | next | 
| 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 192 | show "\<And>N. \<forall>n. norm (X n) \<le> real (Suc N) \<Longrightarrow> \<exists>K>0. \<forall>n. norm (X n) \<le> K" | 
| 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 193 | using of_nat_0_less_iff by blast | 
| 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 194 | qed | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 195 | |
| 63546 | 196 | text \<open>Alternative definition for \<open>Bseq\<close>.\<close> | 
| 197 | lemma Bseq_iff: "Bseq X \<longleftrightarrow> (\<exists>N. \<forall>n. norm (X n) \<le> real(Suc N))" | |
| 198 | by (simp add: Bseq_def) (simp add: lemma_NBseq_def) | |
| 199 | ||
| 200 | lemma lemma_NBseq_def2: "(\<exists>K > 0. \<forall>n. norm (X n) \<le> K) = (\<exists>N. \<forall>n. norm (X n) < real(Suc N))" | |
| 68614 | 201 | proof - | 
| 202 | have *: "\<And>N. \<forall>n. norm (X n) \<le> 1 + real N \<Longrightarrow> | |
| 203 | \<exists>N. \<forall>n. norm (X n) < 1 + real N" | |
| 204 | by (metis add.commute le_less_trans less_add_one of_nat_Suc) | |
| 205 | then show ?thesis | |
| 206 | unfolding lemma_NBseq_def | |
| 207 | by (metis less_le_not_le not_less_iff_gr_or_eq of_nat_Suc) | |
| 208 | qed | |
| 63546 | 209 | |
| 210 | text \<open>Yet another definition for Bseq.\<close> | |
| 211 | lemma Bseq_iff1a: "Bseq X \<longleftrightarrow> (\<exists>N. \<forall>n. norm (X n) < real (Suc N))" | |
| 212 | by (simp add: Bseq_def lemma_NBseq_def2) | |
| 213 | ||
| 214 | subsubsection \<open>A Few More Equivalence Theorems for Boundedness\<close> | |
| 215 | ||
| 216 | text \<open>Alternative formulation for boundedness.\<close> | |
| 217 | lemma Bseq_iff2: "Bseq X \<longleftrightarrow> (\<exists>k > 0. \<exists>x. \<forall>n. norm (X n + - x) \<le> k)" | |
| 68614 | 218 | by (metis BseqE BseqI' add.commute add_cancel_right_left add_uminus_conv_diff norm_add_leD | 
| 219 | norm_minus_cancel norm_minus_commute) | |
| 63546 | 220 | |
| 221 | text \<open>Alternative formulation for boundedness.\<close> | |
| 222 | lemma Bseq_iff3: "Bseq X \<longleftrightarrow> (\<exists>k>0. \<exists>N. \<forall>n. norm (X n + - X N) \<le> k)" | |
| 223 | (is "?P \<longleftrightarrow> ?Q") | |
| 53602 | 224 | proof | 
| 225 | assume ?P | |
| 63546 | 226 | then obtain K where *: "0 < K" and **: "\<And>n. norm (X n) \<le> K" | 
| 68615 | 227 | by (auto simp: Bseq_def) | 
| 53602 | 228 | from * have "0 < K + norm (X 0)" by (rule order_less_le_trans) simp | 
| 54230 
b1d955791529
more simplification rules on unary and binary minus
 haftmann parents: 
53602diff
changeset | 229 | from ** have "\<forall>n. norm (X n - X 0) \<le> K + norm (X 0)" | 
| 
b1d955791529
more simplification rules on unary and binary minus
 haftmann parents: 
53602diff
changeset | 230 | by (auto intro: order_trans norm_triangle_ineq4) | 
| 
b1d955791529
more simplification rules on unary and binary minus
 haftmann parents: 
53602diff
changeset | 231 | then have "\<forall>n. norm (X n + - X 0) \<le> K + norm (X 0)" | 
| 
b1d955791529
more simplification rules on unary and binary minus
 haftmann parents: 
53602diff
changeset | 232 | by simp | 
| 60758 | 233 | with \<open>0 < K + norm (X 0)\<close> show ?Q by blast | 
| 53602 | 234 | next | 
| 63546 | 235 | assume ?Q | 
| 68615 | 236 | then show ?P by (auto simp: Bseq_iff2) | 
| 53602 | 237 | qed | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 238 | |
| 63546 | 239 | |
| 240 | subsubsection \<open>Upper Bounds and Lubs of Bounded Sequences\<close> | |
| 241 | ||
| 242 | lemma Bseq_minus_iff: "Bseq (\<lambda>n. - (X n) :: 'a::real_normed_vector) \<longleftrightarrow> Bseq X" | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 243 | by (simp add: Bseq_def) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 244 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 245 | lemma Bseq_add: | 
| 63546 | 246 | fixes f :: "nat \<Rightarrow> 'a::real_normed_vector" | 
| 247 | assumes "Bseq f" | |
| 248 | shows "Bseq (\<lambda>x. f x + c)" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 249 | proof - | 
| 63546 | 250 | from assms obtain K where K: "\<And>x. norm (f x) \<le> K" | 
| 251 | unfolding Bseq_def by blast | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 252 |   {
 | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 253 | fix x :: nat | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 254 | have "norm (f x + c) \<le> norm (f x) + norm c" by (rule norm_triangle_ineq) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 255 | also have "norm (f x) \<le> K" by (rule K) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 256 | finally have "norm (f x + c) \<le> K + norm c" by simp | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 257 | } | 
| 63546 | 258 | then show ?thesis by (rule BseqI') | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 259 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 260 | |
| 63546 | 261 | lemma Bseq_add_iff: "Bseq (\<lambda>x. f x + c) \<longleftrightarrow> Bseq f" | 
| 262 | for f :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 263 | using Bseq_add[of f c] Bseq_add[of "\<lambda>x. f x + c" "-c"] by auto | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 264 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 265 | lemma Bseq_mult: | 
| 63546 | 266 | fixes f g :: "nat \<Rightarrow> 'a::real_normed_field" | 
| 267 | assumes "Bseq f" and "Bseq g" | |
| 268 | shows "Bseq (\<lambda>x. f x * g x)" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 269 | proof - | 
| 63546 | 270 | from assms obtain K1 K2 where K: "norm (f x) \<le> K1" "K1 > 0" "norm (g x) \<le> K2" "K2 > 0" | 
| 271 | for x | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 272 | unfolding Bseq_def by blast | 
| 63546 | 273 | then have "norm (f x * g x) \<le> K1 * K2" for x | 
| 274 | by (auto simp: norm_mult intro!: mult_mono) | |
| 275 | then show ?thesis by (rule BseqI') | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 276 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 277 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 278 | lemma Bfun_const [simp]: "Bfun (\<lambda>_. c) F" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 279 | unfolding Bfun_metric_def by (auto intro!: exI[of _ c] exI[of _ "1::real"]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 280 | |
| 63546 | 281 | lemma Bseq_cmult_iff: | 
| 282 | fixes c :: "'a::real_normed_field" | |
| 283 | assumes "c \<noteq> 0" | |
| 284 | shows "Bseq (\<lambda>x. c * f x) \<longleftrightarrow> Bseq f" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 285 | proof | 
| 63546 | 286 | assume "Bseq (\<lambda>x. c * f x)" | 
| 287 | with Bfun_const have "Bseq (\<lambda>x. inverse c * (c * f x))" | |
| 288 | by (rule Bseq_mult) | |
| 289 | with \<open>c \<noteq> 0\<close> show "Bseq f" | |
| 70817 
dd675800469d
dedicated fact collections for algebraic simplification rules potentially splitting goals
 haftmann parents: 
70804diff
changeset | 290 | by (simp add: field_split_simps) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 291 | qed (intro Bseq_mult Bfun_const) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 292 | |
| 63546 | 293 | lemma Bseq_subseq: "Bseq f \<Longrightarrow> Bseq (\<lambda>x. f (g x))" | 
| 294 | for f :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 295 | unfolding Bseq_def by auto | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 296 | |
| 63546 | 297 | lemma Bseq_Suc_iff: "Bseq (\<lambda>n. f (Suc n)) \<longleftrightarrow> Bseq f" | 
| 298 | for f :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 299 | using Bseq_offset[of f 1] by (auto intro: Bseq_subseq) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 300 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 301 | lemma increasing_Bseq_subseq_iff: | 
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 302 | assumes "\<And>x y. x \<le> y \<Longrightarrow> norm (f x :: 'a::real_normed_vector) \<le> norm (f y)" "strict_mono g" | 
| 63546 | 303 | shows "Bseq (\<lambda>x. f (g x)) \<longleftrightarrow> Bseq f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 304 | proof | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 305 | assume "Bseq (\<lambda>x. f (g x))" | 
| 63546 | 306 | then obtain K where K: "\<And>x. norm (f (g x)) \<le> K" | 
| 307 | unfolding Bseq_def by auto | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 308 |   {
 | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 309 | fix x :: nat | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 310 | from filterlim_subseq[OF assms(2)] obtain y where "g y \<ge> x" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 311 | by (auto simp: filterlim_at_top eventually_at_top_linorder) | 
| 63546 | 312 | then have "norm (f x) \<le> norm (f (g y))" | 
| 313 | using assms(1) by blast | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 314 | also have "norm (f (g y)) \<le> K" by (rule K) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 315 | finally have "norm (f x) \<le> K" . | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 316 | } | 
| 63546 | 317 | then show "Bseq f" by (rule BseqI') | 
| 318 | qed (use Bseq_subseq[of f g] in simp_all) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 319 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 320 | lemma nonneg_incseq_Bseq_subseq_iff: | 
| 63546 | 321 | fixes f :: "nat \<Rightarrow> real" | 
| 322 | and g :: "nat \<Rightarrow> nat" | |
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 323 | assumes "\<And>x. f x \<ge> 0" "incseq f" "strict_mono g" | 
| 63546 | 324 | shows "Bseq (\<lambda>x. f (g x)) \<longleftrightarrow> Bseq f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 325 | using assms by (intro increasing_Bseq_subseq_iff) (auto simp: incseq_def) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 326 | |
| 63546 | 327 | lemma Bseq_eq_bounded: "range f \<subseteq> {a..b} \<Longrightarrow> Bseq f"
 | 
| 328 | for a b :: real | |
| 68614 | 329 | proof (rule BseqI'[where K="max (norm a) (norm b)"]) | 
| 330 |   fix n assume "range f \<subseteq> {a..b}"
 | |
| 331 |   then have "f n \<in> {a..b}"
 | |
| 332 | by blast | |
| 333 | then show "norm (f n) \<le> max (norm a) (norm b)" | |
| 334 | by auto | |
| 335 | qed | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 336 | |
| 63546 | 337 | lemma incseq_bounded: "incseq X \<Longrightarrow> \<forall>i. X i \<le> B \<Longrightarrow> Bseq X" | 
| 338 | for B :: real | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 339 | by (intro Bseq_eq_bounded[of X "X 0" B]) (auto simp: incseq_def) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 340 | |
| 63546 | 341 | lemma decseq_bounded: "decseq X \<Longrightarrow> \<forall>i. B \<le> X i \<Longrightarrow> Bseq X" | 
| 342 | for B :: real | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 343 | by (intro Bseq_eq_bounded[of X B "X 0"]) (auto simp: decseq_def) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 344 | |
| 63546 | 345 | |
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 346 | subsubsection\<^marker>\<open>tag unimportant\<close> \<open>Polynomal function extremal theorem, from HOL Light\<close> | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 347 | |
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 348 | lemma polyfun_extremal_lemma: | 
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 349 | fixes c :: "nat \<Rightarrow> 'a::real_normed_div_algebra" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 350 | assumes "0 < e" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 351 | shows "\<exists>M. \<forall>z. M \<le> norm(z) \<longrightarrow> norm (\<Sum>i\<le>n. c(i) * z^i) \<le> e * norm(z) ^ (Suc n)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 352 | proof (induct n) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 353 | case 0 with assms | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 354 | show ?case | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 355 | apply (rule_tac x="norm (c 0) / e" in exI) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 356 | apply (auto simp: field_simps) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 357 | done | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 358 | next | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 359 | case (Suc n) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 360 | obtain M where M: "\<And>z. M \<le> norm z \<Longrightarrow> norm (\<Sum>i\<le>n. c i * z^i) \<le> e * norm z ^ Suc n" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 361 | using Suc assms by blast | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 362 | show ?case | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 363 | proof (rule exI [where x= "max M (1 + norm(c(Suc n)) / e)"], clarsimp simp del: power_Suc) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 364 | fix z::'a | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 365 | assume z1: "M \<le> norm z" and "1 + norm (c (Suc n)) / e \<le> norm z" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 366 | then have z2: "e + norm (c (Suc n)) \<le> e * norm z" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 367 | using assms by (simp add: field_simps) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 368 | have "norm (\<Sum>i\<le>n. c i * z^i) \<le> e * norm z ^ Suc n" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 369 | using M [OF z1] by simp | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 370 | then have "norm (\<Sum>i\<le>n. c i * z^i) + norm (c (Suc n) * z ^ Suc n) \<le> e * norm z ^ Suc n + norm (c (Suc n) * z ^ Suc n)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 371 | by simp | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 372 | then have "norm ((\<Sum>i\<le>n. c i * z^i) + c (Suc n) * z ^ Suc n) \<le> e * norm z ^ Suc n + norm (c (Suc n) * z ^ Suc n)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 373 | by (blast intro: norm_triangle_le elim: ) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 374 | also have "... \<le> (e + norm (c (Suc n))) * norm z ^ Suc n" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 375 | by (simp add: norm_power norm_mult algebra_simps) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 376 | also have "... \<le> (e * norm z) * norm z ^ Suc n" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 377 | by (metis z2 mult.commute mult_left_mono norm_ge_zero norm_power) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 378 | finally show "norm ((\<Sum>i\<le>n. c i * z^i) + c (Suc n) * z ^ Suc n) \<le> e * norm z ^ Suc (Suc n)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 379 | by simp | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 380 | qed | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 381 | qed | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 382 | |
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 383 | lemma polyfun_extremal: (*COMPLEX_POLYFUN_EXTREMAL in HOL Light*) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 384 | fixes c :: "nat \<Rightarrow> 'a::real_normed_div_algebra" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 385 | assumes k: "c k \<noteq> 0" "1\<le>k" and kn: "k\<le>n" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 386 | shows "eventually (\<lambda>z. norm (\<Sum>i\<le>n. c(i) * z^i) \<ge> B) at_infinity" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 387 | using kn | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 388 | proof (induction n) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 389 | case 0 | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 390 | then show ?case | 
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 391 | using k by simp | 
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 392 | next | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 393 | case (Suc m) | 
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 394 | show ?case | 
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 395 | proof (cases "c (Suc m) = 0") | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 396 | case True | 
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 397 | then show ?thesis using Suc k | 
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 398 | by auto (metis antisym_conv less_eq_Suc_le not_le) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 399 | next | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 400 | case False | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 401 | then obtain M where M: | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 402 | "\<And>z. M \<le> norm z \<Longrightarrow> norm (\<Sum>i\<le>m. c i * z^i) \<le> norm (c (Suc m)) / 2 * norm z ^ Suc m" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 403 | using polyfun_extremal_lemma [of "norm(c (Suc m)) / 2" c m] Suc | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 404 | by auto | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 405 | have "\<exists>b. \<forall>z. b \<le> norm z \<longrightarrow> B \<le> norm (\<Sum>i\<le>Suc m. c i * z^i)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 406 | proof (rule exI [where x="max M (max 1 (\<bar>B\<bar> / (norm(c (Suc m)) / 2)))"], clarsimp simp del: power_Suc) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 407 | fix z::'a | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 408 | assume z1: "M \<le> norm z" "1 \<le> norm z" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 409 | and "\<bar>B\<bar> * 2 / norm (c (Suc m)) \<le> norm z" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 410 | then have z2: "\<bar>B\<bar> \<le> norm (c (Suc m)) * norm z / 2" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 411 | using False by (simp add: field_simps) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 412 | have nz: "norm z \<le> norm z ^ Suc m" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 413 | by (metis \<open>1 \<le> norm z\<close> One_nat_def less_eq_Suc_le power_increasing power_one_right zero_less_Suc) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 414 | have *: "\<And>y x. norm (c (Suc m)) * norm z / 2 \<le> norm y - norm x \<Longrightarrow> B \<le> norm (x + y)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 415 | by (metis abs_le_iff add.commute norm_diff_ineq order_trans z2) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 416 | have "norm z * norm (c (Suc m)) + 2 * norm (\<Sum>i\<le>m. c i * z^i) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 417 | \<le> norm (c (Suc m)) * norm z + norm (c (Suc m)) * norm z ^ Suc m" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 418 | using M [of z] Suc z1 by auto | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 419 | also have "... \<le> 2 * (norm (c (Suc m)) * norm z ^ Suc m)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 420 | using nz by (simp add: mult_mono del: power_Suc) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 421 | finally show "B \<le> norm ((\<Sum>i\<le>m. c i * z^i) + c (Suc m) * z ^ Suc m)" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 422 | using Suc.IH | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 423 | apply (auto simp: eventually_at_infinity) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 424 | apply (rule *) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 425 | apply (simp add: field_simps norm_mult norm_power) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 426 | done | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 427 | qed | 
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 428 | then show ?thesis | 
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 429 | by (simp add: eventually_at_infinity) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 430 | qed | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 431 | qed | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 432 | |
| 60758 | 433 | subsection \<open>Convergence to Zero\<close> | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 434 | |
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 435 | definition Zfun :: "('a \<Rightarrow> 'b::real_normed_vector) \<Rightarrow> 'a filter \<Rightarrow> bool"
 | 
| 44195 | 436 | where "Zfun f F = (\<forall>r>0. eventually (\<lambda>x. norm (f x) < r) F)" | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 437 | |
| 63546 | 438 | lemma ZfunI: "(\<And>r. 0 < r \<Longrightarrow> eventually (\<lambda>x. norm (f x) < r) F) \<Longrightarrow> Zfun f F" | 
| 439 | by (simp add: Zfun_def) | |
| 440 | ||
| 441 | lemma ZfunD: "Zfun f F \<Longrightarrow> 0 < r \<Longrightarrow> eventually (\<lambda>x. norm (f x) < r) F" | |
| 442 | by (simp add: Zfun_def) | |
| 443 | ||
| 444 | lemma Zfun_ssubst: "eventually (\<lambda>x. f x = g x) F \<Longrightarrow> Zfun g F \<Longrightarrow> Zfun f F" | |
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 445 | unfolding Zfun_def by (auto elim!: eventually_rev_mp) | 
| 31355 | 446 | |
| 44195 | 447 | lemma Zfun_zero: "Zfun (\<lambda>x. 0) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 448 | unfolding Zfun_def by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 449 | |
| 44195 | 450 | lemma Zfun_norm_iff: "Zfun (\<lambda>x. norm (f x)) F = Zfun (\<lambda>x. f x) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 451 | unfolding Zfun_def by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 452 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 453 | lemma Zfun_imp_Zfun: | 
| 44195 | 454 | assumes f: "Zfun f F" | 
| 63546 | 455 | and g: "eventually (\<lambda>x. norm (g x) \<le> norm (f x) * K) F" | 
| 44195 | 456 | shows "Zfun (\<lambda>x. g x) F" | 
| 63546 | 457 | proof (cases "0 < K") | 
| 458 | case K: True | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 459 | show ?thesis | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 460 | proof (rule ZfunI) | 
| 63546 | 461 | fix r :: real | 
| 462 | assume "0 < r" | |
| 463 | then have "0 < r / K" using K by simp | |
| 44195 | 464 | then have "eventually (\<lambda>x. norm (f x) < r / K) F" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 465 | using ZfunD [OF f] by blast | 
| 44195 | 466 | with g show "eventually (\<lambda>x. norm (g x) < r) F" | 
| 46887 | 467 | proof eventually_elim | 
| 468 | case (elim x) | |
| 63546 | 469 | then have "norm (f x) * K < r" | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 470 | by (simp add: pos_less_divide_eq K) | 
| 63546 | 471 | then show ?case | 
| 46887 | 472 | by (simp add: order_le_less_trans [OF elim(1)]) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 473 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 474 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 475 | next | 
| 63546 | 476 | case False | 
| 477 | then have K: "K \<le> 0" by (simp only: not_less) | |
| 31355 | 478 | show ?thesis | 
| 479 | proof (rule ZfunI) | |
| 480 | fix r :: real | |
| 481 | assume "0 < r" | |
| 44195 | 482 | from g show "eventually (\<lambda>x. norm (g x) < r) F" | 
| 46887 | 483 | proof eventually_elim | 
| 484 | case (elim x) | |
| 485 | also have "norm (f x) * K \<le> norm (f x) * 0" | |
| 31355 | 486 | using K norm_ge_zero by (rule mult_left_mono) | 
| 46887 | 487 | finally show ?case | 
| 60758 | 488 | using \<open>0 < r\<close> by simp | 
| 31355 | 489 | qed | 
| 490 | qed | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 491 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 492 | |
| 63546 | 493 | lemma Zfun_le: "Zfun g F \<Longrightarrow> \<forall>x. norm (f x) \<le> norm (g x) \<Longrightarrow> Zfun f F" | 
| 494 | by (erule Zfun_imp_Zfun [where K = 1]) simp | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 495 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 496 | lemma Zfun_add: | 
| 63546 | 497 | assumes f: "Zfun f F" | 
| 498 | and g: "Zfun g F" | |
| 44195 | 499 | shows "Zfun (\<lambda>x. f x + g x) F" | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 500 | proof (rule ZfunI) | 
| 63546 | 501 | fix r :: real | 
| 502 | assume "0 < r" | |
| 503 | then have r: "0 < r / 2" by simp | |
| 44195 | 504 | have "eventually (\<lambda>x. norm (f x) < r/2) F" | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 505 | using f r by (rule ZfunD) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 506 | moreover | 
| 44195 | 507 | have "eventually (\<lambda>x. norm (g x) < r/2) F" | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 508 | using g r by (rule ZfunD) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 509 | ultimately | 
| 44195 | 510 | show "eventually (\<lambda>x. norm (f x + g x) < r) F" | 
| 46887 | 511 | proof eventually_elim | 
| 512 | case (elim x) | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 513 | have "norm (f x + g x) \<le> norm (f x) + norm (g x)" | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 514 | by (rule norm_triangle_ineq) | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 515 | also have "\<dots> < r/2 + r/2" | 
| 46887 | 516 | using elim by (rule add_strict_mono) | 
| 517 | finally show ?case | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 518 | by simp | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 519 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 520 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 521 | |
| 44195 | 522 | lemma Zfun_minus: "Zfun f F \<Longrightarrow> Zfun (\<lambda>x. - f x) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 523 | unfolding Zfun_def by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 524 | |
| 63546 | 525 | lemma Zfun_diff: "Zfun f F \<Longrightarrow> Zfun g F \<Longrightarrow> Zfun (\<lambda>x. f x - g x) F" | 
| 54230 
b1d955791529
more simplification rules on unary and binary minus
 haftmann parents: 
53602diff
changeset | 526 | using Zfun_add [of f F "\<lambda>x. - g x"] by (simp add: Zfun_minus) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 527 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 528 | lemma (in bounded_linear) Zfun: | 
| 44195 | 529 | assumes g: "Zfun g F" | 
| 530 | shows "Zfun (\<lambda>x. f (g x)) F" | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 531 | proof - | 
| 63546 | 532 | obtain K where "norm (f x) \<le> norm x * K" for x | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 533 | using bounded by blast | 
| 44195 | 534 | then have "eventually (\<lambda>x. norm (f (g x)) \<le> norm (g x) * K) F" | 
| 31355 | 535 | by simp | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 536 | with g show ?thesis | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 537 | by (rule Zfun_imp_Zfun) | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 538 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 539 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 540 | lemma (in bounded_bilinear) Zfun: | 
| 44195 | 541 | assumes f: "Zfun f F" | 
| 63546 | 542 | and g: "Zfun g F" | 
| 44195 | 543 | shows "Zfun (\<lambda>x. f x ** g x) F" | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 544 | proof (rule ZfunI) | 
| 63546 | 545 | fix r :: real | 
| 546 | assume r: "0 < r" | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 547 | obtain K where K: "0 < K" | 
| 63546 | 548 | and norm_le: "norm (x ** y) \<le> norm x * norm y * K" for x y | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 549 | using pos_bounded by blast | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 550 | from K have K': "0 < inverse K" | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 551 | by (rule positive_imp_inverse_positive) | 
| 44195 | 552 | have "eventually (\<lambda>x. norm (f x) < r) F" | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 553 | using f r by (rule ZfunD) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 554 | moreover | 
| 44195 | 555 | have "eventually (\<lambda>x. norm (g x) < inverse K) F" | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 556 | using g K' by (rule ZfunD) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 557 | ultimately | 
| 44195 | 558 | show "eventually (\<lambda>x. norm (f x ** g x) < r) F" | 
| 46887 | 559 | proof eventually_elim | 
| 560 | case (elim x) | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 561 | have "norm (f x ** g x) \<le> norm (f x) * norm (g x) * K" | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 562 | by (rule norm_le) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 563 | also have "norm (f x) * norm (g x) * K < r * inverse K * K" | 
| 46887 | 564 | by (intro mult_strict_right_mono mult_strict_mono' norm_ge_zero elim K) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 565 | also from K have "r * inverse K * K = r" | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 566 | by simp | 
| 46887 | 567 | finally show ?case . | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 568 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 569 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 570 | |
| 63546 | 571 | lemma (in bounded_bilinear) Zfun_left: "Zfun f F \<Longrightarrow> Zfun (\<lambda>x. f x ** a) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 572 | by (rule bounded_linear_left [THEN bounded_linear.Zfun]) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 573 | |
| 63546 | 574 | lemma (in bounded_bilinear) Zfun_right: "Zfun f F \<Longrightarrow> Zfun (\<lambda>x. a ** f x) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 575 | by (rule bounded_linear_right [THEN bounded_linear.Zfun]) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 576 | |
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 577 | lemmas Zfun_mult = bounded_bilinear.Zfun [OF bounded_bilinear_mult] | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 578 | lemmas Zfun_mult_right = bounded_bilinear.Zfun_right [OF bounded_bilinear_mult] | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 579 | lemmas Zfun_mult_left = bounded_bilinear.Zfun_left [OF bounded_bilinear_mult] | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 580 | |
| 61973 | 581 | lemma tendsto_Zfun_iff: "(f \<longlongrightarrow> a) F = Zfun (\<lambda>x. f x - a) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 582 | by (simp only: tendsto_iff Zfun_def dist_norm) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 583 | |
| 63546 | 584 | lemma tendsto_0_le: | 
| 585 | "(f \<longlongrightarrow> 0) F \<Longrightarrow> eventually (\<lambda>x. norm (g x) \<le> norm (f x) * K) F \<Longrightarrow> (g \<longlongrightarrow> 0) F" | |
| 56366 | 586 | by (simp add: Zfun_imp_Zfun tendsto_Zfun_iff) | 
| 587 | ||
| 63546 | 588 | |
| 60758 | 589 | subsubsection \<open>Distance and norms\<close> | 
| 36662 
621122eeb138
generalize types of LIMSEQ and LIM; generalize many lemmas
 huffman parents: 
36656diff
changeset | 590 | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 591 | lemma tendsto_dist [tendsto_intros]: | 
| 63546 | 592 | fixes l m :: "'a::metric_space" | 
| 593 | assumes f: "(f \<longlongrightarrow> l) F" | |
| 594 | and g: "(g \<longlongrightarrow> m) F" | |
| 61973 | 595 | shows "((\<lambda>x. dist (f x) (g x)) \<longlongrightarrow> dist l m) F" | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 596 | proof (rule tendstoI) | 
| 63546 | 597 | fix e :: real | 
| 598 | assume "0 < e" | |
| 599 | then have e2: "0 < e/2" by simp | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 600 | from tendstoD [OF f e2] tendstoD [OF g e2] | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 601 | show "eventually (\<lambda>x. dist (dist (f x) (g x)) (dist l m) < e) F" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 602 | proof (eventually_elim) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 603 | case (elim x) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 604 | then show "dist (dist (f x) (g x)) (dist l m) < e" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 605 | unfolding dist_real_def | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 606 | using dist_triangle2 [of "f x" "g x" "l"] | 
| 63546 | 607 | and dist_triangle2 [of "g x" "l" "m"] | 
| 608 | and dist_triangle3 [of "l" "m" "f x"] | |
| 609 | and dist_triangle [of "f x" "m" "g x"] | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 610 | by arith | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 611 | qed | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 612 | qed | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 613 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 614 | lemma continuous_dist[continuous_intros]: | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 615 | fixes f g :: "_ \<Rightarrow> 'a :: metric_space" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 616 | shows "continuous F f \<Longrightarrow> continuous F g \<Longrightarrow> continuous F (\<lambda>x. dist (f x) (g x))" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 617 | unfolding continuous_def by (rule tendsto_dist) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 618 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 619 | lemma continuous_on_dist[continuous_intros]: | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 620 | fixes f g :: "_ \<Rightarrow> 'a :: metric_space" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 621 | shows "continuous_on s f \<Longrightarrow> continuous_on s g \<Longrightarrow> continuous_on s (\<lambda>x. dist (f x) (g x))" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 622 | unfolding continuous_on_def by (auto intro: tendsto_dist) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 623 | |
| 69918 
eddcc7c726f3
new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
 paulson <lp15@cam.ac.uk> parents: 
69593diff
changeset | 624 | lemma continuous_at_dist: "isCont (dist a) b" | 
| 
eddcc7c726f3
new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
 paulson <lp15@cam.ac.uk> parents: 
69593diff
changeset | 625 | using continuous_on_dist [OF continuous_on_const continuous_on_id] continuous_on_eq_continuous_within by blast | 
| 
eddcc7c726f3
new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
 paulson <lp15@cam.ac.uk> parents: 
69593diff
changeset | 626 | |
| 63546 | 627 | lemma tendsto_norm [tendsto_intros]: "(f \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. norm (f x)) \<longlongrightarrow> norm a) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 628 | unfolding norm_conv_dist by (intro tendsto_intros) | 
| 36662 
621122eeb138
generalize types of LIMSEQ and LIM; generalize many lemmas
 huffman parents: 
36656diff
changeset | 629 | |
| 63546 | 630 | lemma continuous_norm [continuous_intros]: "continuous F f \<Longrightarrow> continuous F (\<lambda>x. norm (f x))" | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 631 | unfolding continuous_def by (rule tendsto_norm) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 632 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 633 | lemma continuous_on_norm [continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 634 | "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. norm (f x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 635 | unfolding continuous_on_def by (auto intro: tendsto_norm) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 636 | |
| 71167 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 637 | lemma continuous_on_norm_id [continuous_intros]: "continuous_on S norm" | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 638 | by (intro continuous_on_id continuous_on_norm) | 
| 
b4d409c65a76
Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
 paulson <lp15@cam.ac.uk> parents: 
70999diff
changeset | 639 | |
| 63546 | 640 | lemma tendsto_norm_zero: "(f \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. norm (f x)) \<longlongrightarrow> 0) F" | 
| 641 | by (drule tendsto_norm) simp | |
| 642 | ||
| 643 | lemma tendsto_norm_zero_cancel: "((\<lambda>x. norm (f x)) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> 0) F" | |
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 644 | unfolding tendsto_iff dist_norm by simp | 
| 36662 
621122eeb138
generalize types of LIMSEQ and LIM; generalize many lemmas
 huffman parents: 
36656diff
changeset | 645 | |
| 63546 | 646 | lemma tendsto_norm_zero_iff: "((\<lambda>x. norm (f x)) \<longlongrightarrow> 0) F \<longleftrightarrow> (f \<longlongrightarrow> 0) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 647 | unfolding tendsto_iff dist_norm by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 648 | |
| 63546 | 649 | lemma tendsto_rabs [tendsto_intros]: "(f \<longlongrightarrow> l) F \<Longrightarrow> ((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> \<bar>l\<bar>) F" | 
| 650 | for l :: real | |
| 651 | by (fold real_norm_def) (rule tendsto_norm) | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 652 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 653 | lemma continuous_rabs [continuous_intros]: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 654 | "continuous F f \<Longrightarrow> continuous F (\<lambda>x. \<bar>f x :: real\<bar>)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 655 | unfolding real_norm_def[symmetric] by (rule continuous_norm) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 656 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 657 | lemma continuous_on_rabs [continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 658 | "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. \<bar>f x :: real\<bar>)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 659 | unfolding real_norm_def[symmetric] by (rule continuous_on_norm) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 660 | |
| 63546 | 661 | lemma tendsto_rabs_zero: "(f \<longlongrightarrow> (0::real)) F \<Longrightarrow> ((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> 0) F" | 
| 662 | by (fold real_norm_def) (rule tendsto_norm_zero) | |
| 663 | ||
| 664 | lemma tendsto_rabs_zero_cancel: "((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> (0::real)) F \<Longrightarrow> (f \<longlongrightarrow> 0) F" | |
| 665 | by (fold real_norm_def) (rule tendsto_norm_zero_cancel) | |
| 666 | ||
| 667 | lemma tendsto_rabs_zero_iff: "((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> (0::real)) F \<longleftrightarrow> (f \<longlongrightarrow> 0) F" | |
| 668 | by (fold real_norm_def) (rule tendsto_norm_zero_iff) | |
| 669 | ||
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 670 | |
| 62368 | 671 | subsection \<open>Topological Monoid\<close> | 
| 672 | ||
| 673 | class topological_monoid_add = topological_space + monoid_add + | |
| 674 | assumes tendsto_add_Pair: "LIM x (nhds a \<times>\<^sub>F nhds b). fst x + snd x :> nhds (a + b)" | |
| 675 | ||
| 676 | class topological_comm_monoid_add = topological_monoid_add + comm_monoid_add | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 677 | |
| 31565 | 678 | lemma tendsto_add [tendsto_intros]: | 
| 62368 | 679 | fixes a b :: "'a::topological_monoid_add" | 
| 680 | shows "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. f x + g x) \<longlongrightarrow> a + b) F" | |
| 681 | using filterlim_compose[OF tendsto_add_Pair, of "\<lambda>x. (f x, g x)" a b F] | |
| 682 | by (simp add: nhds_prod[symmetric] tendsto_Pair) | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 683 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 684 | lemma continuous_add [continuous_intros]: | 
| 62368 | 685 | fixes f g :: "_ \<Rightarrow> 'b::topological_monoid_add" | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 686 | shows "continuous F f \<Longrightarrow> continuous F g \<Longrightarrow> continuous F (\<lambda>x. f x + g x)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 687 | unfolding continuous_def by (rule tendsto_add) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 688 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 689 | lemma continuous_on_add [continuous_intros]: | 
| 62368 | 690 | fixes f g :: "_ \<Rightarrow> 'b::topological_monoid_add" | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 691 | shows "continuous_on s f \<Longrightarrow> continuous_on s g \<Longrightarrow> continuous_on s (\<lambda>x. f x + g x)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 692 | unfolding continuous_on_def by (auto intro: tendsto_add) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 693 | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 694 | lemma tendsto_add_zero: | 
| 62368 | 695 | fixes f g :: "_ \<Rightarrow> 'b::topological_monoid_add" | 
| 63546 | 696 | shows "(f \<longlongrightarrow> 0) F \<Longrightarrow> (g \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. f x + g x) \<longlongrightarrow> 0) F" | 
| 697 | by (drule (1) tendsto_add) simp | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 698 | |
| 64267 | 699 | lemma tendsto_sum [tendsto_intros]: | 
| 62368 | 700 | fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 63915 | 701 | shows "(\<And>i. i \<in> I \<Longrightarrow> (f i \<longlongrightarrow> a i) F) \<Longrightarrow> ((\<lambda>x. \<Sum>i\<in>I. f i x) \<longlongrightarrow> (\<Sum>i\<in>I. a i)) F" | 
| 702 | by (induct I rule: infinite_finite_induct) (simp_all add: tendsto_add) | |
| 62368 | 703 | |
| 67673 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 704 | lemma tendsto_null_sum: | 
| 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 705 | fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 706 | assumes "\<And>i. i \<in> I \<Longrightarrow> ((\<lambda>x. f x i) \<longlongrightarrow> 0) F" | 
| 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 707 | shows "((\<lambda>i. sum (f i) I) \<longlongrightarrow> 0) F" | 
| 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 708 | using tendsto_sum [of I "\<lambda>x y. f y x" "\<lambda>x. 0"] assms by simp | 
| 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 709 | |
| 64267 | 710 | lemma continuous_sum [continuous_intros]: | 
| 62368 | 711 | fixes f :: "'a \<Rightarrow> 'b::t2_space \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 63301 | 712 | shows "(\<And>i. i \<in> I \<Longrightarrow> continuous F (f i)) \<Longrightarrow> continuous F (\<lambda>x. \<Sum>i\<in>I. f i x)" | 
| 64267 | 713 | unfolding continuous_def by (rule tendsto_sum) | 
| 714 | ||
| 715 | lemma continuous_on_sum [continuous_intros]: | |
| 62368 | 716 | fixes f :: "'a \<Rightarrow> 'b::topological_space \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 63301 | 717 | shows "(\<And>i. i \<in> I \<Longrightarrow> continuous_on S (f i)) \<Longrightarrow> continuous_on S (\<lambda>x. \<Sum>i\<in>I. f i x)" | 
| 64267 | 718 | unfolding continuous_on_def by (auto intro: tendsto_sum) | 
| 62368 | 719 | |
| 62369 | 720 | instance nat :: topological_comm_monoid_add | 
| 63546 | 721 | by standard | 
| 722 | (simp add: nhds_discrete principal_prod_principal filterlim_principal eventually_principal) | |
| 62369 | 723 | |
| 724 | instance int :: topological_comm_monoid_add | |
| 63546 | 725 | by standard | 
| 726 | (simp add: nhds_discrete principal_prod_principal filterlim_principal eventually_principal) | |
| 727 | ||
| 62369 | 728 | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 729 | subsubsection \<open>Topological group\<close> | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 730 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 731 | class topological_group_add = topological_monoid_add + group_add + | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 732 | assumes tendsto_uminus_nhds: "(uminus \<longlongrightarrow> - a) (nhds a)" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 733 | begin | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 734 | |
| 63546 | 735 | lemma tendsto_minus [tendsto_intros]: "(f \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. - f x) \<longlongrightarrow> - a) F" | 
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 736 | by (rule filterlim_compose[OF tendsto_uminus_nhds]) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 737 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 738 | end | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 739 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 740 | class topological_ab_group_add = topological_group_add + ab_group_add | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 741 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 742 | instance topological_ab_group_add < topological_comm_monoid_add .. | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 743 | |
| 63546 | 744 | lemma continuous_minus [continuous_intros]: "continuous F f \<Longrightarrow> continuous F (\<lambda>x. - f x)" | 
| 745 | for f :: "'a::t2_space \<Rightarrow> 'b::topological_group_add" | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 746 | unfolding continuous_def by (rule tendsto_minus) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 747 | |
| 63546 | 748 | lemma continuous_on_minus [continuous_intros]: "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. - f x)" | 
| 749 | for f :: "_ \<Rightarrow> 'b::topological_group_add" | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 750 | unfolding continuous_on_def by (auto intro: tendsto_minus) | 
| 62368 | 751 | |
| 63546 | 752 | lemma tendsto_minus_cancel: "((\<lambda>x. - f x) \<longlongrightarrow> - a) F \<Longrightarrow> (f \<longlongrightarrow> a) F" | 
| 753 | for a :: "'a::topological_group_add" | |
| 754 | by (drule tendsto_minus) simp | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 755 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 756 | lemma tendsto_minus_cancel_left: | 
| 63546 | 757 | "(f \<longlongrightarrow> - (y::_::topological_group_add)) F \<longleftrightarrow> ((\<lambda>x. - f x) \<longlongrightarrow> y) F" | 
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 758 | using tendsto_minus_cancel[of f "- y" F] tendsto_minus[of f "- y" F] | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 759 | by auto | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 760 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 761 | lemma tendsto_diff [tendsto_intros]: | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 762 | fixes a b :: "'a::topological_group_add" | 
| 63546 | 763 | shows "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. f x - g x) \<longlongrightarrow> a - b) F" | 
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 764 | using tendsto_add [of f a F "\<lambda>x. - g x" "- b"] by (simp add: tendsto_minus) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 765 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 766 | lemma continuous_diff [continuous_intros]: | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 767 | fixes f g :: "'a::t2_space \<Rightarrow> 'b::topological_group_add" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 768 | shows "continuous F f \<Longrightarrow> continuous F g \<Longrightarrow> continuous F (\<lambda>x. f x - g x)" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 769 | unfolding continuous_def by (rule tendsto_diff) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 770 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 771 | lemma continuous_on_diff [continuous_intros]: | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 772 | fixes f g :: "_ \<Rightarrow> 'b::topological_group_add" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 773 | shows "continuous_on s f \<Longrightarrow> continuous_on s g \<Longrightarrow> continuous_on s (\<lambda>x. f x - g x)" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 774 | unfolding continuous_on_def by (auto intro: tendsto_diff) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 775 | |
| 67399 | 776 | lemma continuous_on_op_minus: "continuous_on (s::'a::topological_group_add set) ((-) x)" | 
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 777 | by (rule continuous_intros | simp)+ | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 778 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 779 | instance real_normed_vector < topological_ab_group_add | 
| 62368 | 780 | proof | 
| 63546 | 781 | fix a b :: 'a | 
| 782 | show "((\<lambda>x. fst x + snd x) \<longlongrightarrow> a + b) (nhds a \<times>\<^sub>F nhds b)" | |
| 62368 | 783 | unfolding tendsto_Zfun_iff add_diff_add | 
| 784 | using tendsto_fst[OF filterlim_ident, of "(a,b)"] tendsto_snd[OF filterlim_ident, of "(a,b)"] | |
| 785 | by (intro Zfun_add) | |
| 68615 | 786 | (auto simp: tendsto_Zfun_iff[symmetric] nhds_prod[symmetric] intro!: tendsto_fst) | 
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 787 | show "(uminus \<longlongrightarrow> - a) (nhds a)" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 788 | unfolding tendsto_Zfun_iff minus_diff_minus | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 789 | using filterlim_ident[of "nhds a"] | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 790 | by (intro Zfun_minus) (simp add: tendsto_Zfun_iff) | 
| 62368 | 791 | qed | 
| 792 | ||
| 65204 
d23eded35a33
modernized construction of type bcontfun; base explicit theorems on Uniform_Limit.thy; added some lemmas
 immler parents: 
65036diff
changeset | 793 | lemmas real_tendsto_sandwich = tendsto_sandwich[where 'a=real] | 
| 50999 | 794 | |
| 63546 | 795 | |
| 60758 | 796 | subsubsection \<open>Linear operators and multiplication\<close> | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 797 | |
| 70999 
5b753486c075
Inverse function theorem + lemmas
 paulson <lp15@cam.ac.uk> parents: 
70817diff
changeset | 798 | lemma linear_times [simp]: "linear (\<lambda>x. c * x)" | 
| 63546 | 799 | for c :: "'a::real_algebra" | 
| 61806 
d2e62ae01cd8
Cauchy's integral formula for circles.  Starting to fix eventually_mono.
 paulson <lp15@cam.ac.uk> parents: 
61799diff
changeset | 800 | by (auto simp: linearI distrib_left) | 
| 
d2e62ae01cd8
Cauchy's integral formula for circles.  Starting to fix eventually_mono.
 paulson <lp15@cam.ac.uk> parents: 
61799diff
changeset | 801 | |
| 63546 | 802 | lemma (in bounded_linear) tendsto: "(g \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f (g x)) \<longlongrightarrow> f a) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 803 | by (simp only: tendsto_Zfun_iff diff [symmetric] Zfun) | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 804 | |
| 63546 | 805 | lemma (in bounded_linear) continuous: "continuous F g \<Longrightarrow> continuous F (\<lambda>x. f (g x))" | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 806 | using tendsto[of g _ F] by (auto simp: continuous_def) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 807 | |
| 63546 | 808 | lemma (in bounded_linear) continuous_on: "continuous_on s g \<Longrightarrow> continuous_on s (\<lambda>x. f (g x))" | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 809 | using tendsto[of g] by (auto simp: continuous_on_def) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 810 | |
| 63546 | 811 | lemma (in bounded_linear) tendsto_zero: "(g \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. f (g x)) \<longlongrightarrow> 0) F" | 
| 812 | by (drule tendsto) (simp only: zero) | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 813 | |
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 814 | lemma (in bounded_bilinear) tendsto: | 
| 63546 | 815 | "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. f x ** g x) \<longlongrightarrow> a ** b) F" | 
| 816 | by (simp only: tendsto_Zfun_iff prod_diff_prod Zfun_add Zfun Zfun_left Zfun_right) | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 817 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 818 | lemma (in bounded_bilinear) continuous: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 819 | "continuous F f \<Longrightarrow> continuous F g \<Longrightarrow> continuous F (\<lambda>x. f x ** g x)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 820 | using tendsto[of f _ F g] by (auto simp: continuous_def) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 821 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 822 | lemma (in bounded_bilinear) continuous_on: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 823 | "continuous_on s f \<Longrightarrow> continuous_on s g \<Longrightarrow> continuous_on s (\<lambda>x. f x ** g x)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 824 | using tendsto[of f _ _ g] by (auto simp: continuous_on_def) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 825 | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 826 | lemma (in bounded_bilinear) tendsto_zero: | 
| 61973 | 827 | assumes f: "(f \<longlongrightarrow> 0) F" | 
| 63546 | 828 | and g: "(g \<longlongrightarrow> 0) F" | 
| 61973 | 829 | shows "((\<lambda>x. f x ** g x) \<longlongrightarrow> 0) F" | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 830 | using tendsto [OF f g] by (simp add: zero_left) | 
| 31355 | 831 | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 832 | lemma (in bounded_bilinear) tendsto_left_zero: | 
| 61973 | 833 | "(f \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. f x ** c) \<longlongrightarrow> 0) F" | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 834 | by (rule bounded_linear.tendsto_zero [OF bounded_linear_left]) | 
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 835 | |
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 836 | lemma (in bounded_bilinear) tendsto_right_zero: | 
| 61973 | 837 | "(f \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. c ** f x) \<longlongrightarrow> 0) F" | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 838 | by (rule bounded_linear.tendsto_zero [OF bounded_linear_right]) | 
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 839 | |
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 840 | lemmas tendsto_of_real [tendsto_intros] = | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 841 | bounded_linear.tendsto [OF bounded_linear_of_real] | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 842 | |
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 843 | lemmas tendsto_scaleR [tendsto_intros] = | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 844 | bounded_bilinear.tendsto [OF bounded_bilinear_scaleR] | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 845 | |
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 846 | |
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 847 | text\<open>Analogous type class for multiplication\<close> | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 848 | class topological_semigroup_mult = topological_space + semigroup_mult + | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 849 | assumes tendsto_mult_Pair: "LIM x (nhds a \<times>\<^sub>F nhds b). fst x * snd x :> nhds (a * b)" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 850 | |
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 851 | instance real_normed_algebra < topological_semigroup_mult | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 852 | proof | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 853 | fix a b :: 'a | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 854 | show "((\<lambda>x. fst x * snd x) \<longlongrightarrow> a * b) (nhds a \<times>\<^sub>F nhds b)" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 855 | unfolding nhds_prod[symmetric] | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 856 | using tendsto_fst[OF filterlim_ident, of "(a,b)"] tendsto_snd[OF filterlim_ident, of "(a,b)"] | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 857 | by (simp add: bounded_bilinear.tendsto [OF bounded_bilinear_mult]) | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 858 | qed | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 859 | |
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 860 | lemma tendsto_mult [tendsto_intros]: | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 861 | fixes a b :: "'a::topological_semigroup_mult" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 862 | shows "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. f x * g x) \<longlongrightarrow> a * b) F" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 863 | using filterlim_compose[OF tendsto_mult_Pair, of "\<lambda>x. (f x, g x)" a b F] | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 864 | by (simp add: nhds_prod[symmetric] tendsto_Pair) | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 865 | |
| 63546 | 866 | lemma tendsto_mult_left: "(f \<longlongrightarrow> l) F \<Longrightarrow> ((\<lambda>x. c * (f x)) \<longlongrightarrow> c * l) F" | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 867 | for c :: "'a::topological_semigroup_mult" | 
| 63546 | 868 | by (rule tendsto_mult [OF tendsto_const]) | 
| 869 | ||
| 870 | lemma tendsto_mult_right: "(f \<longlongrightarrow> l) F \<Longrightarrow> ((\<lambda>x. (f x) * c) \<longlongrightarrow> l * c) F" | |
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 871 | for c :: "'a::topological_semigroup_mult" | 
| 63546 | 872 | by (rule tendsto_mult [OF _ tendsto_const]) | 
| 61806 
d2e62ae01cd8
Cauchy's integral formula for circles.  Starting to fix eventually_mono.
 paulson <lp15@cam.ac.uk> parents: 
61799diff
changeset | 873 | |
| 70804 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 874 | lemma tendsto_mult_left_iff [simp]: | 
| 70803 
2d658afa1fc0
Generalised two results concerning limits from the real numbers to type classes
 paulson <lp15@cam.ac.uk> parents: 
70723diff
changeset | 875 |    "c \<noteq> 0 \<Longrightarrow> tendsto(\<lambda>x. c * f x) (c * l) F \<longleftrightarrow> tendsto f l F" for c :: "'a::{topological_semigroup_mult,field}"
 | 
| 70688 
3d894e1cfc75
new material on Analysis, plus some rearrangements
 paulson <lp15@cam.ac.uk> parents: 
70532diff
changeset | 876 | by (auto simp: tendsto_mult_left dest: tendsto_mult_left [where c = "1/c"]) | 
| 
3d894e1cfc75
new material on Analysis, plus some rearrangements
 paulson <lp15@cam.ac.uk> parents: 
70532diff
changeset | 877 | |
| 70804 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 878 | lemma tendsto_mult_right_iff [simp]: | 
| 70803 
2d658afa1fc0
Generalised two results concerning limits from the real numbers to type classes
 paulson <lp15@cam.ac.uk> parents: 
70723diff
changeset | 879 |    "c \<noteq> 0 \<Longrightarrow> tendsto(\<lambda>x. f x * c) (l * c) F \<longleftrightarrow> tendsto f l F" for c :: "'a::{topological_semigroup_mult,field}"
 | 
| 
2d658afa1fc0
Generalised two results concerning limits from the real numbers to type classes
 paulson <lp15@cam.ac.uk> parents: 
70723diff
changeset | 880 | by (auto simp: tendsto_mult_right dest: tendsto_mult_left [where c = "1/c"]) | 
| 70688 
3d894e1cfc75
new material on Analysis, plus some rearrangements
 paulson <lp15@cam.ac.uk> parents: 
70532diff
changeset | 881 | |
| 70804 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 882 | lemma tendsto_zero_mult_left_iff [simp]: | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 883 |   fixes c::"'a::{topological_semigroup_mult,field}" assumes "c \<noteq> 0" shows "(\<lambda>n. c * a n)\<longlonglongrightarrow> 0 \<longleftrightarrow> a \<longlonglongrightarrow> 0"
 | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 884 | using assms tendsto_mult_left tendsto_mult_left_iff by fastforce | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 885 | |
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 886 | lemma tendsto_zero_mult_right_iff [simp]: | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 887 |   fixes c::"'a::{topological_semigroup_mult,field}" assumes "c \<noteq> 0" shows "(\<lambda>n. a n * c)\<longlonglongrightarrow> 0 \<longleftrightarrow> a \<longlonglongrightarrow> 0"
 | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 888 | using assms tendsto_mult_right tendsto_mult_right_iff by fastforce | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 889 | |
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 890 | lemma tendsto_zero_divide_iff [simp]: | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 891 |   fixes c::"'a::{topological_semigroup_mult,field}" assumes "c \<noteq> 0" shows "(\<lambda>n. a n / c)\<longlonglongrightarrow> 0 \<longleftrightarrow> a \<longlonglongrightarrow> 0"
 | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 892 | using tendsto_zero_mult_right_iff [of "1/c" a] assms by (simp add: field_simps) | 
| 
4eef7c6ef7bf
More theorems about limits, including cancellation simprules
 paulson <lp15@cam.ac.uk> parents: 
70803diff
changeset | 893 | |
| 70365 
4df0628e8545
a few new lemmas and a bit of tidying
 paulson <lp15@cam.ac.uk> parents: 
69918diff
changeset | 894 | lemma lim_const_over_n [tendsto_intros]: | 
| 
4df0628e8545
a few new lemmas and a bit of tidying
 paulson <lp15@cam.ac.uk> parents: 
69918diff
changeset | 895 | fixes a :: "'a::real_normed_field" | 
| 
4df0628e8545
a few new lemmas and a bit of tidying
 paulson <lp15@cam.ac.uk> parents: 
69918diff
changeset | 896 | shows "(\<lambda>n. a / of_nat n) \<longlonglongrightarrow> 0" | 
| 
4df0628e8545
a few new lemmas and a bit of tidying
 paulson <lp15@cam.ac.uk> parents: 
69918diff
changeset | 897 | using tendsto_mult [OF tendsto_const [of a] lim_1_over_n] by simp | 
| 
4df0628e8545
a few new lemmas and a bit of tidying
 paulson <lp15@cam.ac.uk> parents: 
69918diff
changeset | 898 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 899 | lemmas continuous_of_real [continuous_intros] = | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 900 | bounded_linear.continuous [OF bounded_linear_of_real] | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 901 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 902 | lemmas continuous_scaleR [continuous_intros] = | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 903 | bounded_bilinear.continuous [OF bounded_bilinear_scaleR] | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 904 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 905 | lemmas continuous_mult [continuous_intros] = | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 906 | bounded_bilinear.continuous [OF bounded_bilinear_mult] | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 907 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 908 | lemmas continuous_on_of_real [continuous_intros] = | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 909 | bounded_linear.continuous_on [OF bounded_linear_of_real] | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 910 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 911 | lemmas continuous_on_scaleR [continuous_intros] = | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 912 | bounded_bilinear.continuous_on [OF bounded_bilinear_scaleR] | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 913 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 914 | lemmas continuous_on_mult [continuous_intros] = | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 915 | bounded_bilinear.continuous_on [OF bounded_bilinear_mult] | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 916 | |
| 44568 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 917 | lemmas tendsto_mult_zero = | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 918 | bounded_bilinear.tendsto_zero [OF bounded_bilinear_mult] | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 919 | |
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 920 | lemmas tendsto_mult_left_zero = | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 921 | bounded_bilinear.tendsto_left_zero [OF bounded_bilinear_mult] | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 922 | |
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 923 | lemmas tendsto_mult_right_zero = | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 924 | bounded_bilinear.tendsto_right_zero [OF bounded_bilinear_mult] | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 925 | |
| 68296 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 926 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 927 | lemma continuous_mult_left: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 928 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 929 | shows "continuous F f \<Longrightarrow> continuous F (\<lambda>x. c * f x)" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 930 | by (rule continuous_mult [OF continuous_const]) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 931 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 932 | lemma continuous_mult_right: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 933 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 934 | shows "continuous F f \<Longrightarrow> continuous F (\<lambda>x. f x * c)" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 935 | by (rule continuous_mult [OF _ continuous_const]) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 936 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 937 | lemma continuous_on_mult_left: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 938 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 939 | shows "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. c * f x)" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 940 | by (rule continuous_on_mult [OF continuous_on_const]) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 941 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 942 | lemma continuous_on_mult_right: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 943 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 944 | shows "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. f x * c)" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 945 | by (rule continuous_on_mult [OF _ continuous_on_const]) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 946 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 947 | lemma continuous_on_mult_const [simp]: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 948 | fixes c::"'a::real_normed_algebra" | 
| 69064 
5840724b1d71
Prefix form of infix with * on either side no longer needs special treatment
 nipkow parents: 
68860diff
changeset | 949 | shows "continuous_on s ((*) c)" | 
| 68296 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 950 | by (intro continuous_on_mult_left continuous_on_id) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 951 | |
| 66793 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 952 | lemma tendsto_divide_zero: | 
| 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 953 | fixes c :: "'a::real_normed_field" | 
| 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 954 | shows "(f \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. f x / c) \<longlongrightarrow> 0) F" | 
| 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 955 | by (cases "c=0") (simp_all add: divide_inverse tendsto_mult_left_zero) | 
| 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 956 | |
| 63546 | 957 | lemma tendsto_power [tendsto_intros]: "(f \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f x ^ n) \<longlongrightarrow> a ^ n) F" | 
| 958 |   for f :: "'a \<Rightarrow> 'b::{power,real_normed_algebra}"
 | |
| 58729 
e8ecc79aee43
add tendsto_const and tendsto_ident_at as simp and intro rules
 hoelzl parents: 
57512diff
changeset | 959 | by (induct n) (simp_all add: tendsto_mult) | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 960 | |
| 65680 
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
 paulson <lp15@cam.ac.uk> parents: 
65578diff
changeset | 961 | lemma tendsto_null_power: "\<lbrakk>(f \<longlongrightarrow> 0) F; 0 < n\<rbrakk> \<Longrightarrow> ((\<lambda>x. f x ^ n) \<longlongrightarrow> 0) F" | 
| 
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
 paulson <lp15@cam.ac.uk> parents: 
65578diff
changeset | 962 |     for f :: "'a \<Rightarrow> 'b::{power,real_normed_algebra_1}"
 | 
| 
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
 paulson <lp15@cam.ac.uk> parents: 
65578diff
changeset | 963 | using tendsto_power [of f 0 F n] by (simp add: power_0_left) | 
| 
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
 paulson <lp15@cam.ac.uk> parents: 
65578diff
changeset | 964 | |
| 63546 | 965 | lemma continuous_power [continuous_intros]: "continuous F f \<Longrightarrow> continuous F (\<lambda>x. (f x)^n)" | 
| 966 |   for f :: "'a::t2_space \<Rightarrow> 'b::{power,real_normed_algebra}"
 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 967 | unfolding continuous_def by (rule tendsto_power) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 968 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 969 | lemma continuous_on_power [continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 970 |   fixes f :: "_ \<Rightarrow> 'b::{power,real_normed_algebra}"
 | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 971 | shows "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. (f x)^n)" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 972 | unfolding continuous_on_def by (auto intro: tendsto_power) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 973 | |
| 64272 | 974 | lemma tendsto_prod [tendsto_intros]: | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 975 |   fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::{real_normed_algebra,comm_ring_1}"
 | 
| 63915 | 976 | shows "(\<And>i. i \<in> S \<Longrightarrow> (f i \<longlongrightarrow> L i) F) \<Longrightarrow> ((\<lambda>x. \<Prod>i\<in>S. f i x) \<longlongrightarrow> (\<Prod>i\<in>S. L i)) F" | 
| 977 | by (induct S rule: infinite_finite_induct) (simp_all add: tendsto_mult) | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 978 | |
| 64272 | 979 | lemma continuous_prod [continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 980 |   fixes f :: "'a \<Rightarrow> 'b::t2_space \<Rightarrow> 'c::{real_normed_algebra,comm_ring_1}"
 | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 981 | shows "(\<And>i. i \<in> S \<Longrightarrow> continuous F (f i)) \<Longrightarrow> continuous F (\<lambda>x. \<Prod>i\<in>S. f i x)" | 
| 64272 | 982 | unfolding continuous_def by (rule tendsto_prod) | 
| 983 | ||
| 984 | lemma continuous_on_prod [continuous_intros]: | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 985 |   fixes f :: "'a \<Rightarrow> _ \<Rightarrow> 'c::{real_normed_algebra,comm_ring_1}"
 | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 986 | shows "(\<And>i. i \<in> S \<Longrightarrow> continuous_on s (f i)) \<Longrightarrow> continuous_on s (\<lambda>x. \<Prod>i\<in>S. f i x)" | 
| 64272 | 987 | unfolding continuous_on_def by (auto intro: tendsto_prod) | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 988 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 989 | lemma tendsto_of_real_iff: | 
| 63546 | 990 | "((\<lambda>x. of_real (f x) :: 'a::real_normed_div_algebra) \<longlongrightarrow> of_real c) F \<longleftrightarrow> (f \<longlongrightarrow> c) F" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 991 | unfolding tendsto_iff by simp | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 992 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 993 | lemma tendsto_add_const_iff: | 
| 74475 
409ca22dee4c
new notion of infinite sums in HOL-Analysis, ordering on complex numbers
 eberlm <eberlm@in.tum.de> parents: 
73885diff
changeset | 994 | "((\<lambda>x. c + f x :: 'a::topological_group_add) \<longlongrightarrow> c + d) F \<longleftrightarrow> (f \<longlongrightarrow> d) F" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 995 | using tendsto_add[OF tendsto_const[of c], of f d] | 
| 63546 | 996 | and tendsto_add[OF tendsto_const[of "-c"], of "\<lambda>x. c + f x" "c + d"] by auto | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 997 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 998 | |
| 68860 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 999 | class topological_monoid_mult = topological_semigroup_mult + monoid_mult | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1000 | class topological_comm_monoid_mult = topological_monoid_mult + comm_monoid_mult | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1001 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1002 | lemma tendsto_power_strong [tendsto_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1003 | fixes f :: "_ \<Rightarrow> 'b :: topological_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1004 | assumes "(f \<longlongrightarrow> a) F" "(g \<longlongrightarrow> b) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1005 | shows "((\<lambda>x. f x ^ g x) \<longlongrightarrow> a ^ b) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1006 | proof - | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1007 | have "((\<lambda>x. f x ^ b) \<longlongrightarrow> a ^ b) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1008 | by (induction b) (auto intro: tendsto_intros assms) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1009 | also from assms(2) have "eventually (\<lambda>x. g x = b) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1010 | by (simp add: nhds_discrete filterlim_principal) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1011 | hence "eventually (\<lambda>x. f x ^ b = f x ^ g x) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1012 | by eventually_elim simp | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1013 | hence "((\<lambda>x. f x ^ b) \<longlongrightarrow> a ^ b) F \<longleftrightarrow> ((\<lambda>x. f x ^ g x) \<longlongrightarrow> a ^ b) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1014 | by (intro filterlim_cong refl) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1015 | finally show ?thesis . | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1016 | qed | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1017 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1018 | lemma continuous_mult' [continuous_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1019 | fixes f g :: "_ \<Rightarrow> 'b::topological_semigroup_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1020 | shows "continuous F f \<Longrightarrow> continuous F g \<Longrightarrow> continuous F (\<lambda>x. f x * g x)" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1021 | unfolding continuous_def by (rule tendsto_mult) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1022 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1023 | lemma continuous_power' [continuous_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1024 | fixes f :: "_ \<Rightarrow> 'b::topological_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1025 | shows "continuous F f \<Longrightarrow> continuous F g \<Longrightarrow> continuous F (\<lambda>x. f x ^ g x)" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1026 | unfolding continuous_def by (rule tendsto_power_strong) auto | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1027 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1028 | lemma continuous_on_mult' [continuous_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1029 | fixes f g :: "_ \<Rightarrow> 'b::topological_semigroup_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1030 | shows "continuous_on A f \<Longrightarrow> continuous_on A g \<Longrightarrow> continuous_on A (\<lambda>x. f x * g x)" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1031 | unfolding continuous_on_def by (auto intro: tendsto_mult) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1032 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1033 | lemma continuous_on_power' [continuous_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1034 | fixes f :: "_ \<Rightarrow> 'b::topological_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1035 | shows "continuous_on A f \<Longrightarrow> continuous_on A g \<Longrightarrow> continuous_on A (\<lambda>x. f x ^ g x)" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1036 | unfolding continuous_on_def by (auto intro: tendsto_power_strong) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1037 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1038 | lemma tendsto_mult_one: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1039 | fixes f g :: "_ \<Rightarrow> 'b::topological_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1040 | shows "(f \<longlongrightarrow> 1) F \<Longrightarrow> (g \<longlongrightarrow> 1) F \<Longrightarrow> ((\<lambda>x. f x * g x) \<longlongrightarrow> 1) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1041 | by (drule (1) tendsto_mult) simp | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1042 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1043 | lemma tendsto_prod' [tendsto_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1044 | fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::topological_comm_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1045 | shows "(\<And>i. i \<in> I \<Longrightarrow> (f i \<longlongrightarrow> a i) F) \<Longrightarrow> ((\<lambda>x. \<Prod>i\<in>I. f i x) \<longlongrightarrow> (\<Prod>i\<in>I. a i)) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1046 | by (induct I rule: infinite_finite_induct) (simp_all add: tendsto_mult) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1047 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1048 | lemma tendsto_one_prod': | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1049 | fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::topological_comm_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1050 | assumes "\<And>i. i \<in> I \<Longrightarrow> ((\<lambda>x. f x i) \<longlongrightarrow> 1) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1051 | shows "((\<lambda>i. prod (f i) I) \<longlongrightarrow> 1) F" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1052 | using tendsto_prod' [of I "\<lambda>x y. f y x" "\<lambda>x. 1"] assms by simp | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1053 | |
| 76724 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1054 | lemma LIMSEQ_prod_0: | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1055 |   fixes f :: "nat \<Rightarrow> 'a::{semidom,topological_space}"
 | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1056 | assumes "f i = 0" | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1057 |   shows "(\<lambda>n. prod f {..n}) \<longlonglongrightarrow> 0"
 | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1058 | proof (subst tendsto_cong) | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1059 |   show "\<forall>\<^sub>F n in sequentially. prod f {..n} = 0"
 | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1060 | using assms eventually_at_top_linorder by auto | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1061 | qed auto | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1062 | |
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1063 | lemma LIMSEQ_prod_nonneg: | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1064 |   fixes f :: "nat \<Rightarrow> 'a::{linordered_semidom,linorder_topology}"
 | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1065 |   assumes 0: "\<And>n. 0 \<le> f n" and a: "(\<lambda>n. prod f {..n}) \<longlonglongrightarrow> a"
 | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1066 | shows "a \<ge> 0" | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1067 | by (simp add: "0" prod_nonneg LIMSEQ_le_const [OF a]) | 
| 
7ff71bdcf731
Additional new material about infinite products, etc.
 paulson <lp15@cam.ac.uk> parents: 
74513diff
changeset | 1068 | |
| 68860 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1069 | lemma continuous_prod' [continuous_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1070 | fixes f :: "'a \<Rightarrow> 'b::t2_space \<Rightarrow> 'c::topological_comm_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1071 | shows "(\<And>i. i \<in> I \<Longrightarrow> continuous F (f i)) \<Longrightarrow> continuous F (\<lambda>x. \<Prod>i\<in>I. f i x)" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1072 | unfolding continuous_def by (rule tendsto_prod') | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1073 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1074 | lemma continuous_on_prod' [continuous_intros]: | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1075 | fixes f :: "'a \<Rightarrow> 'b::topological_space \<Rightarrow> 'c::topological_comm_monoid_mult" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1076 | shows "(\<And>i. i \<in> I \<Longrightarrow> continuous_on S (f i)) \<Longrightarrow> continuous_on S (\<lambda>x. \<Prod>i\<in>I. f i x)" | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1077 | unfolding continuous_on_def by (auto intro: tendsto_prod') | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1078 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1079 | instance nat :: topological_comm_monoid_mult | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1080 | by standard | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1081 | (simp add: nhds_discrete principal_prod_principal filterlim_principal eventually_principal) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1082 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1083 | instance int :: topological_comm_monoid_mult | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1084 | by standard | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1085 | (simp add: nhds_discrete principal_prod_principal filterlim_principal eventually_principal) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1086 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1087 | class comm_real_normed_algebra_1 = real_normed_algebra_1 + comm_monoid_mult | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1088 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1089 | context real_normed_field | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1090 | begin | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1091 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1092 | subclass comm_real_normed_algebra_1 | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1093 | proof | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1094 | from norm_mult[of "1 :: 'a" 1] show "norm 1 = 1" by simp | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1095 | qed (simp_all add: norm_mult) | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1096 | |
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1097 | end | 
| 
f443ec10447d
Some basic materials on filters and topology
 Manuel Eberl <eberlm@in.tum.de> parents: 
68721diff
changeset | 1098 | |
| 60758 | 1099 | subsubsection \<open>Inverse and division\<close> | 
| 31355 | 1100 | |
| 1101 | lemma (in bounded_bilinear) Zfun_prod_Bfun: | |
| 44195 | 1102 | assumes f: "Zfun f F" | 
| 63546 | 1103 | and g: "Bfun g F" | 
| 44195 | 1104 | shows "Zfun (\<lambda>x. f x ** g x) F" | 
| 31355 | 1105 | proof - | 
| 1106 | obtain K where K: "0 \<le> K" | |
| 1107 | and norm_le: "\<And>x y. norm (x ** y) \<le> norm x * norm y * K" | |
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 1108 | using nonneg_bounded by blast | 
| 31355 | 1109 | obtain B where B: "0 < B" | 
| 44195 | 1110 | and norm_g: "eventually (\<lambda>x. norm (g x) \<le> B) F" | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1111 | using g by (rule BfunE) | 
| 44195 | 1112 | have "eventually (\<lambda>x. norm (f x ** g x) \<le> norm (f x) * (B * K)) F" | 
| 46887 | 1113 | using norm_g proof eventually_elim | 
| 1114 | case (elim x) | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1115 | have "norm (f x ** g x) \<le> norm (f x) * norm (g x) * K" | 
| 31355 | 1116 | by (rule norm_le) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1117 | also have "\<dots> \<le> norm (f x) * B * K" | 
| 63546 | 1118 | by (intro mult_mono' order_refl norm_g norm_ge_zero mult_nonneg_nonneg K elim) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1119 | also have "\<dots> = norm (f x) * (B * K)" | 
| 57512 
cc97b347b301
reduced name variants for assoc and commute on plus and mult
 haftmann parents: 
57447diff
changeset | 1120 | by (rule mult.assoc) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1121 | finally show "norm (f x ** g x) \<le> norm (f x) * (B * K)" . | 
| 31355 | 1122 | qed | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1123 | with f show ?thesis | 
| 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1124 | by (rule Zfun_imp_Zfun) | 
| 31355 | 1125 | qed | 
| 1126 | ||
| 1127 | lemma (in bounded_bilinear) Bfun_prod_Zfun: | |
| 44195 | 1128 | assumes f: "Bfun f F" | 
| 63546 | 1129 | and g: "Zfun g F" | 
| 44195 | 1130 | shows "Zfun (\<lambda>x. f x ** g x) F" | 
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 1131 | using flip g f by (rule bounded_bilinear.Zfun_prod_Bfun) | 
| 31355 | 1132 | |
| 1133 | lemma Bfun_inverse: | |
| 1134 | fixes a :: "'a::real_normed_div_algebra" | |
| 61973 | 1135 | assumes f: "(f \<longlongrightarrow> a) F" | 
| 31355 | 1136 | assumes a: "a \<noteq> 0" | 
| 44195 | 1137 | shows "Bfun (\<lambda>x. inverse (f x)) F" | 
| 31355 | 1138 | proof - | 
| 1139 | from a have "0 < norm a" by simp | |
| 63546 | 1140 | then have "\<exists>r>0. r < norm a" by (rule dense) | 
| 1141 | then obtain r where r1: "0 < r" and r2: "r < norm a" | |
| 1142 | by blast | |
| 44195 | 1143 | have "eventually (\<lambda>x. dist (f x) a < r) F" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 1144 | using tendstoD [OF f r1] by blast | 
| 63546 | 1145 | then have "eventually (\<lambda>x. norm (inverse (f x)) \<le> inverse (norm a - r)) F" | 
| 46887 | 1146 | proof eventually_elim | 
| 1147 | case (elim x) | |
| 63546 | 1148 | then have 1: "norm (f x - a) < r" | 
| 31355 | 1149 | by (simp add: dist_norm) | 
| 63546 | 1150 | then have 2: "f x \<noteq> 0" using r2 by auto | 
| 1151 | then have "norm (inverse (f x)) = inverse (norm (f x))" | |
| 31355 | 1152 | by (rule nonzero_norm_inverse) | 
| 1153 | also have "\<dots> \<le> inverse (norm a - r)" | |
| 1154 | proof (rule le_imp_inverse_le) | |
| 63546 | 1155 | show "0 < norm a - r" | 
| 1156 | using r2 by simp | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1157 | have "norm a - norm (f x) \<le> norm (a - f x)" | 
| 31355 | 1158 | by (rule norm_triangle_ineq2) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1159 | also have "\<dots> = norm (f x - a)" | 
| 31355 | 1160 | by (rule norm_minus_commute) | 
| 1161 | also have "\<dots> < r" using 1 . | |
| 63546 | 1162 | finally show "norm a - r \<le> norm (f x)" | 
| 1163 | by simp | |
| 31355 | 1164 | qed | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 1165 | finally show "norm (inverse (f x)) \<le> inverse (norm a - r)" . | 
| 31355 | 1166 | qed | 
| 63546 | 1167 | then show ?thesis by (rule BfunI) | 
| 31355 | 1168 | qed | 
| 1169 | ||
| 31565 | 1170 | lemma tendsto_inverse [tendsto_intros]: | 
| 31355 | 1171 | fixes a :: "'a::real_normed_div_algebra" | 
| 61973 | 1172 | assumes f: "(f \<longlongrightarrow> a) F" | 
| 63546 | 1173 | and a: "a \<noteq> 0" | 
| 61973 | 1174 | shows "((\<lambda>x. inverse (f x)) \<longlongrightarrow> inverse a) F" | 
| 31355 | 1175 | proof - | 
| 1176 | from a have "0 < norm a" by simp | |
| 44195 | 1177 | with f have "eventually (\<lambda>x. dist (f x) a < norm a) F" | 
| 31355 | 1178 | by (rule tendstoD) | 
| 44195 | 1179 | then have "eventually (\<lambda>x. f x \<noteq> 0) F" | 
| 61810 | 1180 | unfolding dist_norm by (auto elim!: eventually_mono) | 
| 44627 | 1181 | with a have "eventually (\<lambda>x. inverse (f x) - inverse a = | 
| 1182 | - (inverse (f x) * (f x - a) * inverse a)) F" | |
| 61810 | 1183 | by (auto elim!: eventually_mono simp: inverse_diff_inverse) | 
| 44627 | 1184 | moreover have "Zfun (\<lambda>x. - (inverse (f x) * (f x - a) * inverse a)) F" | 
| 1185 | by (intro Zfun_minus Zfun_mult_left | |
| 1186 | bounded_bilinear.Bfun_prod_Zfun [OF bounded_bilinear_mult] | |
| 1187 | Bfun_inverse [OF f a] f [unfolded tendsto_Zfun_iff]) | |
| 1188 | ultimately show ?thesis | |
| 1189 | unfolding tendsto_Zfun_iff by (rule Zfun_ssubst) | |
| 31355 | 1190 | qed | 
| 1191 | ||
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1192 | lemma continuous_inverse: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1193 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1194 | assumes "continuous F f" | 
| 1195 | and "f (Lim F (\<lambda>x. x)) \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1196 | shows "continuous F (\<lambda>x. inverse (f x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1197 | using assms unfolding continuous_def by (rule tendsto_inverse) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1198 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1199 | lemma continuous_at_within_inverse[continuous_intros]: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1200 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1201 | assumes "continuous (at a within s) f" | 
| 1202 | and "f a \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1203 | shows "continuous (at a within s) (\<lambda>x. inverse (f x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1204 | using assms unfolding continuous_within by (rule tendsto_inverse) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1205 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 1206 | lemma continuous_on_inverse[continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1207 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1208 | assumes "continuous_on s f" | 
| 1209 | and "\<forall>x\<in>s. f x \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1210 | shows "continuous_on s (\<lambda>x. inverse (f x))" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 1211 | using assms unfolding continuous_on_def by (blast intro: tendsto_inverse) | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1212 | |
| 31565 | 1213 | lemma tendsto_divide [tendsto_intros]: | 
| 31355 | 1214 | fixes a b :: "'a::real_normed_field" | 
| 63546 | 1215 | shows "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> b \<noteq> 0 \<Longrightarrow> ((\<lambda>x. f x / g x) \<longlongrightarrow> a / b) F" | 
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 1216 | by (simp add: tendsto_mult tendsto_inverse divide_inverse) | 
| 31355 | 1217 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1218 | lemma continuous_divide: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1219 | fixes f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_field" | 
| 63546 | 1220 | assumes "continuous F f" | 
| 1221 | and "continuous F g" | |
| 1222 | and "g (Lim F (\<lambda>x. x)) \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1223 | shows "continuous F (\<lambda>x. (f x) / (g x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1224 | using assms unfolding continuous_def by (rule tendsto_divide) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1225 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1226 | lemma continuous_at_within_divide[continuous_intros]: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1227 | fixes f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_field" | 
| 63546 | 1228 | assumes "continuous (at a within s) f" "continuous (at a within s) g" | 
| 1229 | and "g a \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1230 | shows "continuous (at a within s) (\<lambda>x. (f x) / (g x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1231 | using assms unfolding continuous_within by (rule tendsto_divide) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1232 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1233 | lemma isCont_divide[continuous_intros, simp]: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1234 | fixes f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_field" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1235 | assumes "isCont f a" "isCont g a" "g a \<noteq> 0" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1236 | shows "isCont (\<lambda>x. (f x) / g x) a" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1237 | using assms unfolding continuous_at by (rule tendsto_divide) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1238 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 1239 | lemma continuous_on_divide[continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1240 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_field" | 
| 63546 | 1241 | assumes "continuous_on s f" "continuous_on s g" | 
| 1242 | and "\<forall>x\<in>s. g x \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1243 | shows "continuous_on s (\<lambda>x. (f x) / (g x))" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 1244 | using assms unfolding continuous_on_def by (blast intro: tendsto_divide) | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1245 | |
| 71837 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1246 | lemma tendsto_power_int [tendsto_intros]: | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1247 | fixes a :: "'a::real_normed_div_algebra" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1248 | assumes f: "(f \<longlongrightarrow> a) F" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1249 | and a: "a \<noteq> 0" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1250 | shows "((\<lambda>x. power_int (f x) n) \<longlongrightarrow> power_int a n) F" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1251 | using assms by (cases n rule: int_cases4) (auto intro!: tendsto_intros simp: power_int_minus) | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1252 | |
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1253 | lemma continuous_power_int: | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1254 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1255 | assumes "continuous F f" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1256 | and "f (Lim F (\<lambda>x. x)) \<noteq> 0" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1257 | shows "continuous F (\<lambda>x. power_int (f x) n)" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1258 | using assms unfolding continuous_def by (rule tendsto_power_int) | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1259 | |
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1260 | lemma continuous_at_within_power_int[continuous_intros]: | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1261 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1262 | assumes "continuous (at a within s) f" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1263 | and "f a \<noteq> 0" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1264 | shows "continuous (at a within s) (\<lambda>x. power_int (f x) n)" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1265 | using assms unfolding continuous_within by (rule tendsto_power_int) | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1266 | |
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1267 | lemma continuous_on_power_int [continuous_intros]: | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1268 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1269 | assumes "continuous_on s f" and "\<forall>x\<in>s. f x \<noteq> 0" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1270 | shows "continuous_on s (\<lambda>x. power_int (f x) n)" | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1271 | using assms unfolding continuous_on_def by (blast intro: tendsto_power_int) | 
| 
dca11678c495
new constant power_int in HOL
 Manuel Eberl <eberlm@in.tum.de> parents: 
71827diff
changeset | 1272 | |
| 77221 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1273 | lemma tendsto_power_int' [tendsto_intros]: | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1274 | fixes a :: "'a::real_normed_div_algebra" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1275 | assumes f: "(f \<longlongrightarrow> a) F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1276 | and a: "a \<noteq> 0 \<or> n \<ge> 0" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1277 | shows "((\<lambda>x. power_int (f x) n) \<longlongrightarrow> power_int a n) F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1278 | using assms by (cases n rule: int_cases4) (auto intro!: tendsto_intros simp: power_int_minus) | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1279 | |
| 63546 | 1280 | lemma tendsto_sgn [tendsto_intros]: "(f \<longlongrightarrow> l) F \<Longrightarrow> l \<noteq> 0 \<Longrightarrow> ((\<lambda>x. sgn (f x)) \<longlongrightarrow> sgn l) F" | 
| 1281 | for l :: "'a::real_normed_vector" | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 1282 | unfolding sgn_div_norm by (simp add: tendsto_intros) | 
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 1283 | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1284 | lemma continuous_sgn: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1285 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1286 | assumes "continuous F f" | 
| 1287 | and "f (Lim F (\<lambda>x. x)) \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1288 | shows "continuous F (\<lambda>x. sgn (f x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1289 | using assms unfolding continuous_def by (rule tendsto_sgn) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1290 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1291 | lemma continuous_at_within_sgn[continuous_intros]: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1292 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1293 | assumes "continuous (at a within s) f" | 
| 1294 | and "f a \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1295 | shows "continuous (at a within s) (\<lambda>x. sgn (f x))" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1296 | using assms unfolding continuous_within by (rule tendsto_sgn) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1297 | |
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1298 | lemma isCont_sgn[continuous_intros]: | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1299 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1300 | assumes "isCont f a" | 
| 1301 | and "f a \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1302 | shows "isCont (\<lambda>x. sgn (f x)) a" | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1303 | using assms unfolding continuous_at by (rule tendsto_sgn) | 
| 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1304 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 1305 | lemma continuous_on_sgn[continuous_intros]: | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1306 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1307 | assumes "continuous_on s f" | 
| 1308 | and "\<forall>x\<in>s. f x \<noteq> 0" | |
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1309 | shows "continuous_on s (\<lambda>x. sgn (f x))" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 1310 | using assms unfolding continuous_on_def by (blast intro: tendsto_sgn) | 
| 51478 
270b21f3ae0a
move continuous and continuous_on to the HOL image; isCont is an abbreviation for continuous (at x) (isCont is now restricted to a T2 space)
 hoelzl parents: 
51474diff
changeset | 1311 | |
| 50325 | 1312 | lemma filterlim_at_infinity: | 
| 61076 | 1313 | fixes f :: "_ \<Rightarrow> 'a::real_normed_vector" | 
| 50325 | 1314 | assumes "0 \<le> c" | 
| 1315 | shows "(LIM x F. f x :> at_infinity) \<longleftrightarrow> (\<forall>r>c. eventually (\<lambda>x. r \<le> norm (f x)) F)" | |
| 1316 | unfolding filterlim_iff eventually_at_infinity | |
| 1317 | proof safe | |
| 63546 | 1318 | fix P :: "'a \<Rightarrow> bool" | 
| 1319 | fix b | |
| 50325 | 1320 | assume *: "\<forall>r>c. eventually (\<lambda>x. r \<le> norm (f x)) F" | 
| 63546 | 1321 | assume P: "\<forall>x. b \<le> norm x \<longrightarrow> P x" | 
| 50325 | 1322 | have "max b (c + 1) > c" by auto | 
| 1323 | with * have "eventually (\<lambda>x. max b (c + 1) \<le> norm (f x)) F" | |
| 1324 | by auto | |
| 1325 | then show "eventually (\<lambda>x. P (f x)) F" | |
| 1326 | proof eventually_elim | |
| 63546 | 1327 | case (elim x) | 
| 50325 | 1328 | with P show "P (f x)" by auto | 
| 1329 | qed | |
| 1330 | qed force | |
| 1331 | ||
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1332 | lemma filterlim_at_infinity_imp_norm_at_top: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1333 | fixes F | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1334 | assumes "filterlim f at_infinity F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1335 | shows "filterlim (\<lambda>x. norm (f x)) at_top F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1336 | proof - | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1337 |   {
 | 
| 68611 | 1338 | fix r :: real | 
| 1339 | have "\<forall>\<^sub>F x in F. r \<le> norm (f x)" using filterlim_at_infinity[of 0 f F] assms | |
| 1340 | by (cases "r > 0") | |
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1341 | (auto simp: not_less intro: always_eventually order.trans[OF _ norm_ge_zero]) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1342 | } | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1343 | thus ?thesis by (auto simp: filterlim_at_top) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1344 | qed | 
| 68611 | 1345 | |
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1346 | lemma filterlim_norm_at_top_imp_at_infinity: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1347 | fixes F | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1348 | assumes "filterlim (\<lambda>x. norm (f x)) at_top F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1349 | shows "filterlim f at_infinity F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1350 | using filterlim_at_infinity[of 0 f F] assms by (auto simp: filterlim_at_top) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1351 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1352 | lemma filterlim_norm_at_top: "filterlim norm at_top at_infinity" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1353 | by (rule filterlim_at_infinity_imp_norm_at_top) (rule filterlim_ident) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1354 | |
| 67950 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1355 | lemma filterlim_at_infinity_conv_norm_at_top: | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1356 | "filterlim f at_infinity G \<longleftrightarrow> filterlim (\<lambda>x. norm (f x)) at_top G" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1357 | by (auto simp: filterlim_at_infinity[OF order.refl] filterlim_at_top_gt[of _ _ 0]) | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1358 | |
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1359 | lemma eventually_not_equal_at_infinity: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1360 |   "eventually (\<lambda>x. x \<noteq> (a :: 'a :: {real_normed_vector})) at_infinity"
 | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1361 | proof - | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1362 | from filterlim_norm_at_top[where 'a = 'a] | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1363 | have "\<forall>\<^sub>F x in at_infinity. norm a < norm (x::'a)" by (auto simp: filterlim_at_top_dense) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1364 | thus ?thesis by eventually_elim auto | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1365 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1366 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1367 | lemma filterlim_int_of_nat_at_topD: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1368 | fixes F | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1369 | assumes "filterlim (\<lambda>x. f (int x)) F at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1370 | shows "filterlim f F at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1371 | proof - | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1372 | have "filterlim (\<lambda>x. f (int (nat x))) F at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1373 | by (rule filterlim_compose[OF assms filterlim_nat_sequentially]) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1374 | also have "?this \<longleftrightarrow> filterlim f F at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1375 | by (intro filterlim_cong refl eventually_mono [OF eventually_ge_at_top[of "0::int"]]) auto | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1376 | finally show ?thesis . | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1377 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1378 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1379 | lemma filterlim_int_sequentially [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1380 | "filterlim int at_top sequentially" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1381 | unfolding filterlim_at_top | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1382 | proof | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1383 | fix C :: int | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1384 | show "eventually (\<lambda>n. int n \<ge> C) at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1385 | using eventually_ge_at_top[of "nat \<lceil>C\<rceil>"] by eventually_elim linarith | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1386 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1387 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1388 | lemma filterlim_real_of_int_at_top [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1389 | "filterlim real_of_int at_top at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1390 | unfolding filterlim_at_top | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1391 | proof | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1392 | fix C :: real | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1393 | show "eventually (\<lambda>n. real_of_int n \<ge> C) at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1394 | using eventually_ge_at_top[of "\<lceil>C\<rceil>"] by eventually_elim linarith | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1395 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1396 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1397 | lemma filterlim_abs_real: "filterlim (abs::real \<Rightarrow> real) at_top at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1398 | proof (subst filterlim_cong[OF refl refl]) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1399 | from eventually_ge_at_top[of "0::real"] show "eventually (\<lambda>x::real. \<bar>x\<bar> = x) at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1400 | by eventually_elim simp | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1401 | qed (simp_all add: filterlim_ident) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1402 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1403 | lemma filterlim_of_real_at_infinity [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1404 | "filterlim (of_real :: real \<Rightarrow> 'a :: real_normed_algebra_1) at_infinity at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1405 | by (intro filterlim_norm_at_top_imp_at_infinity) (auto simp: filterlim_abs_real) | 
| 68611 | 1406 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1407 | lemma not_tendsto_and_filterlim_at_infinity: | 
| 63546 | 1408 | fixes c :: "'a::real_normed_vector" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1409 | assumes "F \<noteq> bot" | 
| 63546 | 1410 | and "(f \<longlongrightarrow> c) F" | 
| 1411 | and "filterlim f at_infinity F" | |
| 1412 | shows False | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1413 | proof - | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 1414 | from tendstoD[OF assms(2), of "1/2"] | 
| 63546 | 1415 | have "eventually (\<lambda>x. dist (f x) c < 1/2) F" | 
| 1416 | by simp | |
| 1417 | moreover | |
| 1418 | from filterlim_at_infinity[of "norm c" f F] assms(3) | |
| 1419 | have "eventually (\<lambda>x. norm (f x) \<ge> norm c + 1) F" by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1420 | ultimately have "eventually (\<lambda>x. False) F" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1421 | proof eventually_elim | 
| 63546 | 1422 | fix x | 
| 1423 | assume A: "dist (f x) c < 1/2" | |
| 1424 | assume "norm (f x) \<ge> norm c + 1" | |
| 62379 
340738057c8c
An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!
 paulson <lp15@cam.ac.uk> parents: 
62369diff
changeset | 1425 | also have "norm (f x) = dist (f x) 0" by simp | 
| 63546 | 1426 | also have "\<dots> \<le> dist (f x) c + dist c 0" by (rule dist_triangle) | 
| 62379 
340738057c8c
An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!
 paulson <lp15@cam.ac.uk> parents: 
62369diff
changeset | 1427 | finally show False using A by simp | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1428 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1429 | with assms show False by simp | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1430 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1431 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1432 | lemma filterlim_at_infinity_imp_not_convergent: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1433 | assumes "filterlim f at_infinity sequentially" | 
| 63546 | 1434 | shows "\<not> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1435 | by (rule notI, rule not_tendsto_and_filterlim_at_infinity[OF _ _ assms]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1436 | (simp_all add: convergent_LIMSEQ_iff) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1437 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1438 | lemma filterlim_at_infinity_imp_eventually_ne: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1439 | assumes "filterlim f at_infinity F" | 
| 63546 | 1440 | shows "eventually (\<lambda>z. f z \<noteq> c) F" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1441 | proof - | 
| 63546 | 1442 | have "norm c + 1 > 0" | 
| 1443 | by (intro add_nonneg_pos) simp_all | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1444 | with filterlim_at_infinity[OF order.refl, of f F] assms | 
| 63546 | 1445 | have "eventually (\<lambda>z. norm (f z) \<ge> norm c + 1) F" | 
| 1446 | by blast | |
| 1447 | then show ?thesis | |
| 1448 | by eventually_elim auto | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1449 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1450 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 1451 | lemma tendsto_of_nat [tendsto_intros]: | 
| 63546 | 1452 | "filterlim (of_nat :: nat \<Rightarrow> 'a::real_normed_algebra_1) at_infinity sequentially" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1453 | proof (subst filterlim_at_infinity[OF order.refl], intro allI impI) | 
| 63040 | 1454 | fix r :: real | 
| 1455 | assume r: "r > 0" | |
| 1456 | define n where "n = nat \<lceil>r\<rceil>" | |
| 63546 | 1457 | from r have n: "\<forall>m\<ge>n. of_nat m \<ge> r" | 
| 1458 | unfolding n_def by linarith | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1459 | from eventually_ge_at_top[of n] show "eventually (\<lambda>m. norm (of_nat m :: 'a) \<ge> r) sequentially" | 
| 63546 | 1460 | by eventually_elim (use n in simp_all) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1461 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1462 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1463 | |
| 69593 | 1464 | subsection \<open>Relate \<^const>\<open>at\<close>, \<^const>\<open>at_left\<close> and \<^const>\<open>at_right\<close>\<close> | 
| 50347 | 1465 | |
| 60758 | 1466 | text \<open> | 
| 69593 | 1467 | This lemmas are useful for conversion between \<^term>\<open>at x\<close> to \<^term>\<open>at_left x\<close> and | 
| 1468 | \<^term>\<open>at_right x\<close> and also \<^term>\<open>at_right 0\<close>. | |
| 60758 | 1469 | \<close> | 
| 50347 | 1470 | |
| 51471 | 1471 | lemmas filterlim_split_at_real = filterlim_split_at[where 'a=real] | 
| 50323 | 1472 | |
| 63546 | 1473 | lemma filtermap_nhds_shift: "filtermap (\<lambda>x. x - d) (nhds a) = nhds (a - d)" | 
| 1474 | for a d :: "'a::real_normed_vector" | |
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1475 | by (rule filtermap_fun_inverse[where g="\<lambda>x. x + d"]) | 
| 63546 | 1476 | (auto intro!: tendsto_eq_intros filterlim_ident) | 
| 1477 | ||
| 1478 | lemma filtermap_nhds_minus: "filtermap (\<lambda>x. - x) (nhds a) = nhds (- a)" | |
| 1479 | for a :: "'a::real_normed_vector" | |
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1480 | by (rule filtermap_fun_inverse[where g=uminus]) | 
| 63546 | 1481 | (auto intro!: tendsto_eq_intros filterlim_ident) | 
| 1482 | ||
| 1483 | lemma filtermap_at_shift: "filtermap (\<lambda>x. x - d) (at a) = at (a - d)" | |
| 1484 | for a d :: "'a::real_normed_vector" | |
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1485 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_shift[symmetric]) | 
| 50347 | 1486 | |
| 63546 | 1487 | lemma filtermap_at_right_shift: "filtermap (\<lambda>x. x - d) (at_right a) = at_right (a - d)" | 
| 1488 | for a d :: "real" | |
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1489 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_shift[symmetric]) | 
| 50323 | 1490 | |
| 73795 | 1491 | lemma filterlim_shift: | 
| 1492 | fixes d :: "'a::real_normed_vector" | |
| 1493 | assumes "filterlim f F (at a)" | |
| 1494 | shows "filterlim (f \<circ> (+) d) F (at (a - d))" | |
| 1495 | unfolding filterlim_iff | |
| 1496 | proof (intro strip) | |
| 1497 | fix P | |
| 1498 | assume "eventually P F" | |
| 1499 | then have "\<forall>\<^sub>F x in filtermap (\<lambda>y. y - d) (at a). P (f (d + x))" | |
| 1500 | using assms by (force simp add: filterlim_iff eventually_filtermap) | |
| 1501 | then show "(\<forall>\<^sub>F x in at (a - d). P ((f \<circ> (+) d) x))" | |
| 1502 | by (force simp add: filtermap_at_shift) | |
| 1503 | qed | |
| 1504 | ||
| 1505 | lemma filterlim_shift_iff: | |
| 1506 | fixes d :: "'a::real_normed_vector" | |
| 1507 | shows "filterlim (f \<circ> (+) d) F (at (a - d)) = filterlim f F (at a)" (is "?lhs = ?rhs") | |
| 1508 | proof | |
| 1509 | assume L: ?lhs show ?rhs | |
| 1510 | using filterlim_shift [OF L, of "-d"] by (simp add: filterlim_iff) | |
| 1511 | qed (metis filterlim_shift) | |
| 1512 | ||
| 63546 | 1513 | lemma at_right_to_0: "at_right a = filtermap (\<lambda>x. x + a) (at_right 0)" | 
| 1514 | for a :: real | |
| 50347 | 1515 | using filtermap_at_right_shift[of "-a" 0] by simp | 
| 1516 | ||
| 1517 | lemma filterlim_at_right_to_0: | |
| 63546 | 1518 | "filterlim f F (at_right a) \<longleftrightarrow> filterlim (\<lambda>x. f (x + a)) F (at_right 0)" | 
| 1519 | for a :: real | |
| 50347 | 1520 | unfolding filterlim_def filtermap_filtermap at_right_to_0[of a] .. | 
| 1521 | ||
| 1522 | lemma eventually_at_right_to_0: | |
| 63546 | 1523 | "eventually P (at_right a) \<longleftrightarrow> eventually (\<lambda>x. P (x + a)) (at_right 0)" | 
| 1524 | for a :: real | |
| 50347 | 1525 | unfolding at_right_to_0[of a] by (simp add: eventually_filtermap) | 
| 1526 | ||
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1527 | lemma at_to_0: "at a = filtermap (\<lambda>x. x + a) (at 0)" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1528 | for a :: "'a::real_normed_vector" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1529 | using filtermap_at_shift[of "-a" 0] by simp | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1530 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1531 | lemma filterlim_at_to_0: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1532 | "filterlim f F (at a) \<longleftrightarrow> filterlim (\<lambda>x. f (x + a)) F (at 0)" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1533 | for a :: "'a::real_normed_vector" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1534 | unfolding filterlim_def filtermap_filtermap at_to_0[of a] .. | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1535 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1536 | lemma eventually_at_to_0: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1537 | "eventually P (at a) \<longleftrightarrow> eventually (\<lambda>x. P (x + a)) (at 0)" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1538 | for a :: "'a::real_normed_vector" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1539 | unfolding at_to_0[of a] by (simp add: eventually_filtermap) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1540 | |
| 63546 | 1541 | lemma filtermap_at_minus: "filtermap (\<lambda>x. - x) (at a) = at (- a)" | 
| 1542 | for a :: "'a::real_normed_vector" | |
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1543 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_minus[symmetric]) | 
| 50347 | 1544 | |
| 63546 | 1545 | lemma at_left_minus: "at_left a = filtermap (\<lambda>x. - x) (at_right (- a))" | 
| 1546 | for a :: real | |
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1547 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_minus[symmetric]) | 
| 50323 | 1548 | |
| 63546 | 1549 | lemma at_right_minus: "at_right a = filtermap (\<lambda>x. - x) (at_left (- a))" | 
| 1550 | for a :: real | |
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1551 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_minus[symmetric]) | 
| 50347 | 1552 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1553 | |
| 50347 | 1554 | lemma filterlim_at_left_to_right: | 
| 63546 | 1555 | "filterlim f F (at_left a) \<longleftrightarrow> filterlim (\<lambda>x. f (- x)) F (at_right (-a))" | 
| 1556 | for a :: real | |
| 50347 | 1557 | unfolding filterlim_def filtermap_filtermap at_left_minus[of a] .. | 
| 1558 | ||
| 1559 | lemma eventually_at_left_to_right: | |
| 63546 | 1560 | "eventually P (at_left a) \<longleftrightarrow> eventually (\<lambda>x. P (- x)) (at_right (-a))" | 
| 1561 | for a :: real | |
| 50347 | 1562 | unfolding at_left_minus[of a] by (simp add: eventually_filtermap) | 
| 1563 | ||
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1564 | lemma filterlim_uminus_at_top_at_bot: "LIM x at_bot. - x :: real :> at_top" | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1565 | unfolding filterlim_at_top eventually_at_bot_dense | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1566 | by (metis leI minus_less_iff order_less_asym) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1567 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1568 | lemma filterlim_uminus_at_bot_at_top: "LIM x at_top. - x :: real :> at_bot" | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1569 | unfolding filterlim_at_bot eventually_at_top_dense | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1570 | by (metis leI less_minus_iff order_less_asym) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1571 | |
| 68611 | 1572 | lemma at_bot_mirror : | 
| 1573 |   shows "(at_bot::('a::{ordered_ab_group_add,linorder} filter)) = filtermap uminus at_top"
 | |
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 1574 | proof (rule filtermap_fun_inverse[symmetric]) | 
| 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 1575 | show "filterlim uminus at_top (at_bot::'a filter)" | 
| 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 1576 | using eventually_at_bot_linorder filterlim_at_top le_minus_iff by force | 
| 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 1577 | show "filterlim uminus (at_bot::'a filter) at_top" | 
| 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 1578 | by (simp add: filterlim_at_bot minus_le_iff) | 
| 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 1579 | qed auto | 
| 68532 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1580 | |
| 68611 | 1581 | lemma at_top_mirror : | 
| 1582 |   shows "(at_top::('a::{ordered_ab_group_add,linorder} filter)) = filtermap uminus at_bot"
 | |
| 68532 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1583 | apply (subst at_bot_mirror) | 
| 68615 | 1584 | by (auto simp: filtermap_filtermap) | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1585 | |
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1586 | lemma filterlim_at_top_mirror: "(LIM x at_top. f x :> F) \<longleftrightarrow> (LIM x at_bot. f (-x::real) :> F)" | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1587 | unfolding filterlim_def at_top_mirror filtermap_filtermap .. | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1588 | |
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1589 | lemma filterlim_at_bot_mirror: "(LIM x at_bot. f x :> F) \<longleftrightarrow> (LIM x at_top. f (-x::real) :> F)" | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1590 | unfolding filterlim_def at_bot_mirror filtermap_filtermap .. | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1591 | |
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1592 | lemma filterlim_uminus_at_top: "(LIM x F. f x :> at_top) \<longleftrightarrow> (LIM x F. - (f x) :: real :> at_bot)" | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1593 | using filterlim_compose[OF filterlim_uminus_at_bot_at_top, of f F] | 
| 63546 | 1594 | and filterlim_compose[OF filterlim_uminus_at_top_at_bot, of "\<lambda>x. - f x" F] | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1595 | by auto | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1596 | |
| 68721 | 1597 | lemma tendsto_at_botI_sequentially: | 
| 1598 | fixes f :: "real \<Rightarrow> 'b::first_countable_topology" | |
| 1599 | assumes *: "\<And>X. filterlim X at_bot sequentially \<Longrightarrow> (\<lambda>n. f (X n)) \<longlonglongrightarrow> y" | |
| 1600 | shows "(f \<longlongrightarrow> y) at_bot" | |
| 1601 | unfolding filterlim_at_bot_mirror | |
| 1602 | proof (rule tendsto_at_topI_sequentially) | |
| 1603 | fix X :: "nat \<Rightarrow> real" assume "filterlim X at_top sequentially" | |
| 1604 | thus "(\<lambda>n. f (-X n)) \<longlonglongrightarrow> y" by (intro *) (auto simp: filterlim_uminus_at_top) | |
| 1605 | qed | |
| 1606 | ||
| 67950 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1607 | lemma filterlim_at_infinity_imp_filterlim_at_top: | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1608 | assumes "filterlim (f :: 'a \<Rightarrow> real) at_infinity F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1609 | assumes "eventually (\<lambda>x. f x > 0) F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1610 | shows "filterlim f at_top F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1611 | proof - | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1612 | from assms(2) have *: "eventually (\<lambda>x. norm (f x) = f x) F" by eventually_elim simp | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1613 | from assms(1) show ?thesis unfolding filterlim_at_infinity_conv_norm_at_top | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1614 | by (subst (asm) filterlim_cong[OF refl refl *]) | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1615 | qed | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1616 | |
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1617 | lemma filterlim_at_infinity_imp_filterlim_at_bot: | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1618 | assumes "filterlim (f :: 'a \<Rightarrow> real) at_infinity F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1619 | assumes "eventually (\<lambda>x. f x < 0) F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1620 | shows "filterlim f at_bot F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1621 | proof - | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1622 | from assms(2) have *: "eventually (\<lambda>x. norm (f x) = -f x) F" by eventually_elim simp | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1623 | from assms(1) have "filterlim (\<lambda>x. - f x) at_top F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1624 | unfolding filterlim_at_infinity_conv_norm_at_top | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1625 | by (subst (asm) filterlim_cong[OF refl refl *]) | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1626 | thus ?thesis by (simp add: filterlim_uminus_at_top) | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1627 | qed | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1628 | |
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1629 | lemma filterlim_uminus_at_bot: "(LIM x F. f x :> at_bot) \<longleftrightarrow> (LIM x F. - (f x) :: real :> at_top)" | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1630 | unfolding filterlim_uminus_at_top by simp | 
| 50323 | 1631 | |
| 50347 | 1632 | lemma filterlim_inverse_at_top_right: "LIM x at_right (0::real). inverse x :> at_top" | 
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1633 | unfolding filterlim_at_top_gt[where c=0] eventually_at_filter | 
| 50347 | 1634 | proof safe | 
| 63546 | 1635 | fix Z :: real | 
| 1636 | assume [arith]: "0 < Z" | |
| 50347 | 1637 | then have "eventually (\<lambda>x. x < inverse Z) (nhds 0)" | 
| 68615 | 1638 | by (auto simp: eventually_nhds_metric dist_real_def intro!: exI[of _ "\<bar>inverse Z\<bar>"]) | 
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1639 |   then show "eventually (\<lambda>x. x \<noteq> 0 \<longrightarrow> x \<in> {0<..} \<longrightarrow> Z \<le> inverse x) (nhds 0)"
 | 
| 61810 | 1640 | by (auto elim!: eventually_mono simp: inverse_eq_divide field_simps) | 
| 50347 | 1641 | qed | 
| 1642 | ||
| 50325 | 1643 | lemma tendsto_inverse_0: | 
| 61076 | 1644 | fixes x :: "_ \<Rightarrow> 'a::real_normed_div_algebra" | 
| 61973 | 1645 | shows "(inverse \<longlongrightarrow> (0::'a)) at_infinity" | 
| 50325 | 1646 | unfolding tendsto_Zfun_iff diff_0_right Zfun_def eventually_at_infinity | 
| 1647 | proof safe | |
| 63546 | 1648 | fix r :: real | 
| 1649 | assume "0 < r" | |
| 50325 | 1650 | show "\<exists>b. \<forall>x. b \<le> norm x \<longrightarrow> norm (inverse x :: 'a) < r" | 
| 1651 | proof (intro exI[of _ "inverse (r / 2)"] allI impI) | |
| 1652 | fix x :: 'a | |
| 60758 | 1653 | from \<open>0 < r\<close> have "0 < inverse (r / 2)" by simp | 
| 50325 | 1654 | also assume *: "inverse (r / 2) \<le> norm x" | 
| 1655 | finally show "norm (inverse x) < r" | |
| 63546 | 1656 | using * \<open>0 < r\<close> | 
| 1657 | by (subst nonzero_norm_inverse) (simp_all add: inverse_eq_divide field_simps) | |
| 50325 | 1658 | qed | 
| 1659 | qed | |
| 1660 | ||
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1661 | lemma tendsto_add_filterlim_at_infinity: | 
| 63546 | 1662 | fixes c :: "'b::real_normed_vector" | 
| 1663 | and F :: "'a filter" | |
| 1664 | assumes "(f \<longlongrightarrow> c) F" | |
| 1665 | and "filterlim g at_infinity F" | |
| 1666 | shows "filterlim (\<lambda>x. f x + g x) at_infinity F" | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1667 | proof (subst filterlim_at_infinity[OF order_refl], safe) | 
| 63546 | 1668 | fix r :: real | 
| 1669 | assume r: "r > 0" | |
| 1670 | from assms(1) have "((\<lambda>x. norm (f x)) \<longlongrightarrow> norm c) F" | |
| 1671 | by (rule tendsto_norm) | |
| 1672 | then have "eventually (\<lambda>x. norm (f x) < norm c + 1) F" | |
| 1673 | by (rule order_tendstoD) simp_all | |
| 1674 | moreover from r have "r + norm c + 1 > 0" | |
| 1675 | by (intro add_pos_nonneg) simp_all | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1676 | with assms(2) have "eventually (\<lambda>x. norm (g x) \<ge> r + norm c + 1) F" | 
| 63546 | 1677 | unfolding filterlim_at_infinity[OF order_refl] | 
| 1678 | by (elim allE[of _ "r + norm c + 1"]) simp_all | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1679 | ultimately show "eventually (\<lambda>x. norm (f x + g x) \<ge> r) F" | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1680 | proof eventually_elim | 
| 63546 | 1681 | fix x :: 'a | 
| 1682 | assume A: "norm (f x) < norm c + 1" and B: "r + norm c + 1 \<le> norm (g x)" | |
| 1683 | from A B have "r \<le> norm (g x) - norm (f x)" | |
| 1684 | by simp | |
| 1685 | also have "norm (g x) - norm (f x) \<le> norm (g x + f x)" | |
| 1686 | by (rule norm_diff_ineq) | |
| 1687 | finally show "r \<le> norm (f x + g x)" | |
| 1688 | by (simp add: add_ac) | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1689 | qed | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1690 | qed | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1691 | |
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1692 | lemma tendsto_add_filterlim_at_infinity': | 
| 63546 | 1693 | fixes c :: "'b::real_normed_vector" | 
| 1694 | and F :: "'a filter" | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1695 | assumes "filterlim f at_infinity F" | 
| 63546 | 1696 | and "(g \<longlongrightarrow> c) F" | 
| 1697 | shows "filterlim (\<lambda>x. f x + g x) at_infinity F" | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1698 | by (subst add.commute) (rule tendsto_add_filterlim_at_infinity assms)+ | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1699 | |
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1700 | lemma filterlim_inverse_at_right_top: "LIM x at_top. inverse x :> at_right (0::real)" | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1701 | unfolding filterlim_at | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1702 | by (auto simp: eventually_at_top_dense) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1703 | (metis tendsto_inverse_0 filterlim_mono at_top_le_at_infinity order_refl) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1704 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1705 | lemma filterlim_inverse_at_top: | 
| 61973 | 1706 | "(f \<longlongrightarrow> (0 :: real)) F \<Longrightarrow> eventually (\<lambda>x. 0 < f x) F \<Longrightarrow> LIM x F. inverse (f x) :> at_top" | 
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1707 | by (intro filterlim_compose[OF filterlim_inverse_at_top_right]) | 
| 61810 | 1708 | (simp add: filterlim_def eventually_filtermap eventually_mono at_within_def le_principal) | 
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1709 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1710 | lemma filterlim_inverse_at_bot_neg: | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1711 | "LIM x (at_left (0::real)). inverse x :> at_bot" | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1712 | by (simp add: filterlim_inverse_at_top_right filterlim_uminus_at_bot filterlim_at_left_to_right) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1713 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1714 | lemma filterlim_inverse_at_bot: | 
| 61973 | 1715 | "(f \<longlongrightarrow> (0 :: real)) F \<Longrightarrow> eventually (\<lambda>x. f x < 0) F \<Longrightarrow> LIM x F. inverse (f x) :> at_bot" | 
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1716 | unfolding filterlim_uminus_at_bot inverse_minus_eq[symmetric] | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1717 | by (rule filterlim_inverse_at_top) (simp_all add: tendsto_minus_cancel_left[symmetric]) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1718 | |
| 50347 | 1719 | lemma at_right_to_top: "(at_right (0::real)) = filtermap inverse at_top" | 
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1720 | by (intro filtermap_fun_inverse[symmetric, where g=inverse]) | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1721 | (auto intro: filterlim_inverse_at_top_right filterlim_inverse_at_right_top) | 
| 50347 | 1722 | |
| 1723 | lemma eventually_at_right_to_top: | |
| 1724 | "eventually P (at_right (0::real)) \<longleftrightarrow> eventually (\<lambda>x. P (inverse x)) at_top" | |
| 1725 | unfolding at_right_to_top eventually_filtermap .. | |
| 1726 | ||
| 1727 | lemma filterlim_at_right_to_top: | |
| 1728 | "filterlim f F (at_right (0::real)) \<longleftrightarrow> (LIM x at_top. f (inverse x) :> F)" | |
| 1729 | unfolding filterlim_def at_right_to_top filtermap_filtermap .. | |
| 1730 | ||
| 1731 | lemma at_top_to_right: "at_top = filtermap inverse (at_right (0::real))" | |
| 1732 | unfolding at_right_to_top filtermap_filtermap inverse_inverse_eq filtermap_ident .. | |
| 1733 | ||
| 1734 | lemma eventually_at_top_to_right: | |
| 1735 | "eventually P at_top \<longleftrightarrow> eventually (\<lambda>x. P (inverse x)) (at_right (0::real))" | |
| 1736 | unfolding at_top_to_right eventually_filtermap .. | |
| 1737 | ||
| 1738 | lemma filterlim_at_top_to_right: | |
| 1739 | "filterlim f F at_top \<longleftrightarrow> (LIM x (at_right (0::real)). f (inverse x) :> F)" | |
| 1740 | unfolding filterlim_def at_top_to_right filtermap_filtermap .. | |
| 1741 | ||
| 50325 | 1742 | lemma filterlim_inverse_at_infinity: | 
| 61076 | 1743 |   fixes x :: "_ \<Rightarrow> 'a::{real_normed_div_algebra, division_ring}"
 | 
| 50325 | 1744 | shows "filterlim inverse at_infinity (at (0::'a))" | 
| 1745 | unfolding filterlim_at_infinity[OF order_refl] | |
| 1746 | proof safe | |
| 63546 | 1747 | fix r :: real | 
| 1748 | assume "0 < r" | |
| 50325 | 1749 | then show "eventually (\<lambda>x::'a. r \<le> norm (inverse x)) (at 0)" | 
| 1750 | unfolding eventually_at norm_inverse | |
| 1751 | by (intro exI[of _ "inverse r"]) | |
| 1752 | (auto simp: norm_conv_dist[symmetric] field_simps inverse_eq_divide) | |
| 1753 | qed | |
| 1754 | ||
| 1755 | lemma filterlim_inverse_at_iff: | |
| 61076 | 1756 |   fixes g :: "'a \<Rightarrow> 'b::{real_normed_div_algebra, division_ring}"
 | 
| 50325 | 1757 | shows "(LIM x F. inverse (g x) :> at 0) \<longleftrightarrow> (LIM x F. g x :> at_infinity)" | 
| 1758 | unfolding filterlim_def filtermap_filtermap[symmetric] | |
| 1759 | proof | |
| 1760 | assume "filtermap g F \<le> at_infinity" | |
| 1761 | then have "filtermap inverse (filtermap g F) \<le> filtermap inverse at_infinity" | |
| 1762 | by (rule filtermap_mono) | |
| 1763 | also have "\<dots> \<le> at 0" | |
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1764 | using tendsto_inverse_0[where 'a='b] | 
| 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 1765 | by (auto intro!: exI[of _ 1] | 
| 63546 | 1766 | simp: le_principal eventually_filtermap filterlim_def at_within_def eventually_at_infinity) | 
| 50325 | 1767 | finally show "filtermap inverse (filtermap g F) \<le> at 0" . | 
| 1768 | next | |
| 1769 | assume "filtermap inverse (filtermap g F) \<le> at 0" | |
| 1770 | then have "filtermap inverse (filtermap inverse (filtermap g F)) \<le> filtermap inverse (at 0)" | |
| 1771 | by (rule filtermap_mono) | |
| 1772 | with filterlim_inverse_at_infinity show "filtermap g F \<le> at_infinity" | |
| 1773 | by (auto intro: order_trans simp: filterlim_def filtermap_filtermap) | |
| 1774 | qed | |
| 1775 | ||
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1776 | lemma tendsto_mult_filterlim_at_infinity: | 
| 63546 | 1777 | fixes c :: "'a::real_normed_field" | 
| 64394 | 1778 | assumes "(f \<longlongrightarrow> c) F" "c \<noteq> 0" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1779 | assumes "filterlim g at_infinity F" | 
| 63546 | 1780 | shows "filterlim (\<lambda>x. f x * g x) at_infinity F" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1781 | proof - | 
| 61973 | 1782 | have "((\<lambda>x. inverse (f x) * inverse (g x)) \<longlongrightarrow> inverse c * 0) F" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1783 | by (intro tendsto_mult tendsto_inverse assms filterlim_compose[OF tendsto_inverse_0]) | 
| 63546 | 1784 | then have "filterlim (\<lambda>x. inverse (f x) * inverse (g x)) (at (inverse c * 0)) F" | 
| 1785 | unfolding filterlim_at | |
| 1786 | using assms | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1787 | by (auto intro: filterlim_at_infinity_imp_eventually_ne tendsto_imp_eventually_ne eventually_conj) | 
| 63546 | 1788 | then show ?thesis | 
| 1789 | by (subst filterlim_inverse_at_iff[symmetric]) simp_all | |
| 68611 | 1790 | qed | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1791 | |
| 77221 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1792 | lemma filterlim_power_int_neg_at_infinity: | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1793 |   fixes f :: "_ \<Rightarrow> 'a::{real_normed_div_algebra, division_ring}"
 | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1794 | assumes "n < 0" and lim: "(f \<longlongrightarrow> 0) F" and ev: "eventually (\<lambda>x. f x \<noteq> 0) F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1795 | shows "filterlim (\<lambda>x. f x powi n) at_infinity F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1796 | proof - | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1797 | have lim': "((\<lambda>x. f x ^ nat (- n)) \<longlongrightarrow> 0) F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1798 | by (rule tendsto_eq_intros lim)+ (use \<open>n < 0\<close> in auto) | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1799 | have ev': "eventually (\<lambda>x. f x ^ nat (-n) \<noteq> 0) F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1800 | using ev by eventually_elim (use \<open>n < 0\<close> in auto) | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1801 | have "filterlim (\<lambda>x. inverse (f x ^ nat (-n))) at_infinity F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1802 | by (intro filterlim_compose[OF filterlim_inverse_at_infinity]) | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1803 | (use lim' ev' in \<open>auto simp: filterlim_at\<close>) | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1804 | thus ?thesis | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1805 | using \<open>n < 0\<close> by (simp add: power_int_def power_inverse) | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1806 | qed | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1807 | |
| 61973 | 1808 | lemma tendsto_inverse_0_at_top: "LIM x F. f x :> at_top \<Longrightarrow> ((\<lambda>x. inverse (f x) :: real) \<longlongrightarrow> 0) F" | 
| 73885 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1809 | by (metis filterlim_at filterlim_mono[OF _ at_top_le_at_infinity order_refl] filterlim_inverse_at_iff) | 
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1810 | |
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1811 | lemma filterlim_inverse_at_top_iff: | 
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1812 | "eventually (\<lambda>x. 0 < f x) F \<Longrightarrow> (LIM x F. inverse (f x) :> at_top) \<longleftrightarrow> (f \<longlongrightarrow> (0 :: real)) F" | 
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1813 | by (auto dest: tendsto_inverse_0_at_top filterlim_inverse_at_top) | 
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1814 | |
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1815 | lemma filterlim_at_top_iff_inverse_0: | 
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1816 | "eventually (\<lambda>x. 0 < f x) F \<Longrightarrow> (LIM x F. f x :> at_top) \<longleftrightarrow> ((inverse \<circ> f) \<longlongrightarrow> (0 :: real)) F" | 
| 
26171a89466a
A few useful lemmas about derivatives, colinearity and other topics
 paulson <lp15@cam.ac.uk> parents: 
73795diff
changeset | 1817 | using filterlim_inverse_at_top_iff [of "inverse \<circ> f"] by auto | 
| 50419 | 1818 | |
| 63556 | 1819 | lemma real_tendsto_divide_at_top: | 
| 1820 | fixes c::"real" | |
| 1821 | assumes "(f \<longlongrightarrow> c) F" | |
| 1822 | assumes "filterlim g at_top F" | |
| 1823 | shows "((\<lambda>x. f x / g x) \<longlongrightarrow> 0) F" | |
| 1824 | by (auto simp: divide_inverse_commute | |
| 1825 | intro!: tendsto_mult[THEN tendsto_eq_rhs] tendsto_inverse_0_at_top assms) | |
| 1826 | ||
| 63546 | 1827 | lemma mult_nat_left_at_top: "c > 0 \<Longrightarrow> filterlim (\<lambda>x. c * x) at_top sequentially" | 
| 1828 | for c :: nat | |
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 1829 | by (rule filterlim_subseq) (auto simp: strict_mono_def) | 
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1830 | |
| 63546 | 1831 | lemma mult_nat_right_at_top: "c > 0 \<Longrightarrow> filterlim (\<lambda>x. x * c) at_top sequentially" | 
| 1832 | for c :: nat | |
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 1833 | by (rule filterlim_subseq) (auto simp: strict_mono_def) | 
| 63546 | 1834 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1835 | lemma filterlim_times_pos: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1836 | "LIM x F1. c * f x :> at_right l" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1837 | if "filterlim f (at_right p) F1" "0 < c" "l = c * p" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1838 |   for c::"'a::{linordered_field, linorder_topology}"
 | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1839 | unfolding filterlim_iff | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1840 | proof safe | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1841 | fix P | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1842 | assume "\<forall>\<^sub>F x in at_right l. P x" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1843 | then obtain d where "c * p < d" "\<And>y. y > c * p \<Longrightarrow> y < d \<Longrightarrow> P y" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1844 | unfolding \<open>l = _ \<close> eventually_at_right_field | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1845 | by auto | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1846 | then have "\<forall>\<^sub>F a in at_right p. P (c * a)" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1847 | by (auto simp: eventually_at_right_field \<open>0 < c\<close> field_simps intro!: exI[where x="d/c"]) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1848 | from that(1)[unfolded filterlim_iff, rule_format, OF this] | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1849 | show "\<forall>\<^sub>F x in F1. P (c * f x)" . | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1850 | qed | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1851 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1852 | lemma filtermap_nhds_times: "c \<noteq> 0 \<Longrightarrow> filtermap (times c) (nhds a) = nhds (c * a)" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1853 | for a c :: "'a::real_normed_field" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1854 | by (rule filtermap_fun_inverse[where g="\<lambda>x. inverse c * x"]) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1855 | (auto intro!: tendsto_eq_intros filterlim_ident) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1856 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1857 | lemma filtermap_times_pos_at_right: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1858 |   fixes c::"'a::{linordered_field, linorder_topology}"
 | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1859 | assumes "c > 0" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1860 | shows "filtermap (times c) (at_right p) = at_right (c * p)" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1861 | using assms | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1862 | by (intro filtermap_fun_inverse[where g="\<lambda>x. inverse c * x"]) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1863 | (auto intro!: filterlim_ident filterlim_times_pos) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1864 | |
| 63546 | 1865 | lemma at_to_infinity: "(at (0::'a::{real_normed_field,field})) = filtermap inverse at_infinity"
 | 
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1866 | proof (rule antisym) | 
| 61973 | 1867 | have "(inverse \<longlongrightarrow> (0::'a)) at_infinity" | 
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1868 | by (fact tendsto_inverse_0) | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1869 | then show "filtermap inverse at_infinity \<le> at (0::'a)" | 
| 68615 | 1870 | using filterlim_def filterlim_ident filterlim_inverse_at_iff by fastforce | 
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1871 | next | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1872 | have "filtermap inverse (filtermap inverse (at (0::'a))) \<le> filtermap inverse at_infinity" | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1873 | using filterlim_inverse_at_infinity unfolding filterlim_def | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1874 | by (rule filtermap_mono) | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1875 | then show "at (0::'a) \<le> filtermap inverse at_infinity" | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1876 | by (simp add: filtermap_ident filtermap_filtermap) | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1877 | qed | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1878 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1879 | lemma lim_at_infinity_0: | 
| 63546 | 1880 |   fixes l :: "'a::{real_normed_field,field}"
 | 
| 1881 | shows "(f \<longlongrightarrow> l) at_infinity \<longleftrightarrow> ((f \<circ> inverse) \<longlongrightarrow> l) (at (0::'a))" | |
| 1882 | by (simp add: tendsto_compose_filtermap at_to_infinity filtermap_filtermap) | |
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1883 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1884 | lemma lim_zero_infinity: | 
| 63546 | 1885 |   fixes l :: "'a::{real_normed_field,field}"
 | 
| 61973 | 1886 | shows "((\<lambda>x. f(1 / x)) \<longlongrightarrow> l) (at (0::'a)) \<Longrightarrow> (f \<longlongrightarrow> l) at_infinity" | 
| 63546 | 1887 | by (simp add: inverse_eq_divide lim_at_infinity_0 comp_def) | 
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1888 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1889 | |
| 60758 | 1890 | text \<open> | 
| 63546 | 1891 | We only show rules for multiplication and addition when the functions are either against a real | 
| 1892 |   value or against infinity. Further rules are easy to derive by using @{thm
 | |
| 1893 | filterlim_uminus_at_top}. | |
| 60758 | 1894 | \<close> | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1895 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1896 | lemma filterlim_tendsto_pos_mult_at_top: | 
| 63546 | 1897 | assumes f: "(f \<longlongrightarrow> c) F" | 
| 1898 | and c: "0 < c" | |
| 1899 | and g: "LIM x F. g x :> at_top" | |
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1900 | shows "LIM x F. (f x * g x :: real) :> at_top" | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1901 | unfolding filterlim_at_top_gt[where c=0] | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1902 | proof safe | 
| 63546 | 1903 | fix Z :: real | 
| 1904 | assume "0 < Z" | |
| 60758 | 1905 | from f \<open>0 < c\<close> have "eventually (\<lambda>x. c / 2 < f x) F" | 
| 61810 | 1906 | by (auto dest!: tendstoD[where e="c / 2"] elim!: eventually_mono | 
| 63546 | 1907 | simp: dist_real_def abs_real_def split: if_split_asm) | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1908 | moreover from g have "eventually (\<lambda>x. (Z / c * 2) \<le> g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1909 | unfolding filterlim_at_top by auto | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1910 | ultimately show "eventually (\<lambda>x. Z \<le> f x * g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1911 | proof eventually_elim | 
| 63546 | 1912 | case (elim x) | 
| 60758 | 1913 | with \<open>0 < Z\<close> \<open>0 < c\<close> have "c / 2 * (Z / c * 2) \<le> f x * g x" | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1914 | by (intro mult_mono) (auto simp: zero_le_divide_iff) | 
| 60758 | 1915 | with \<open>0 < c\<close> show "Z \<le> f x * g x" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1916 | by simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1917 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1918 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1919 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1920 | lemma filterlim_at_top_mult_at_top: | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1921 | assumes f: "LIM x F. f x :> at_top" | 
| 63546 | 1922 | and g: "LIM x F. g x :> at_top" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1923 | shows "LIM x F. (f x * g x :: real) :> at_top" | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1924 | unfolding filterlim_at_top_gt[where c=0] | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1925 | proof safe | 
| 63546 | 1926 | fix Z :: real | 
| 1927 | assume "0 < Z" | |
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1928 | from f have "eventually (\<lambda>x. 1 \<le> f x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1929 | unfolding filterlim_at_top by auto | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1930 | moreover from g have "eventually (\<lambda>x. Z \<le> g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1931 | unfolding filterlim_at_top by auto | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1932 | ultimately show "eventually (\<lambda>x. Z \<le> f x * g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1933 | proof eventually_elim | 
| 63546 | 1934 | case (elim x) | 
| 60758 | 1935 | with \<open>0 < Z\<close> have "1 * Z \<le> f x * g x" | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1936 | by (intro mult_mono) (auto simp: zero_le_divide_iff) | 
| 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 1937 | then show "Z \<le> f x * g x" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1938 | by simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1939 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1940 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1941 | |
| 63556 | 1942 | lemma filterlim_at_top_mult_tendsto_pos: | 
| 1943 | assumes f: "(f \<longlongrightarrow> c) F" | |
| 1944 | and c: "0 < c" | |
| 1945 | and g: "LIM x F. g x :> at_top" | |
| 1946 | shows "LIM x F. (g x * f x:: real) :> at_top" | |
| 1947 | by (auto simp: mult.commute intro!: filterlim_tendsto_pos_mult_at_top f c g) | |
| 1948 | ||
| 50419 | 1949 | lemma filterlim_tendsto_pos_mult_at_bot: | 
| 63546 | 1950 | fixes c :: real | 
| 1951 | assumes "(f \<longlongrightarrow> c) F" "0 < c" "filterlim g at_bot F" | |
| 50419 | 1952 | shows "LIM x F. f x * g x :> at_bot" | 
| 1953 | using filterlim_tendsto_pos_mult_at_top[OF assms(1,2), of "\<lambda>x. - g x"] assms(3) | |
| 1954 | unfolding filterlim_uminus_at_bot by simp | |
| 1955 | ||
| 60182 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1956 | lemma filterlim_tendsto_neg_mult_at_bot: | 
| 63546 | 1957 | fixes c :: real | 
| 1958 | assumes c: "(f \<longlongrightarrow> c) F" "c < 0" and g: "filterlim g at_top F" | |
| 60182 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1959 | shows "LIM x F. f x * g x :> at_bot" | 
| 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1960 | using c filterlim_tendsto_pos_mult_at_top[of "\<lambda>x. - f x" "- c" F, OF _ _ g] | 
| 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1961 | unfolding filterlim_uminus_at_bot tendsto_minus_cancel_left by simp | 
| 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1962 | |
| 77221 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1963 | |
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1964 | lemma filterlim_cmult_at_bot_at_top: | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1965 | assumes "filterlim (h :: _ \<Rightarrow> real) at_top F" "c \<noteq> 0" "G = (if c > 0 then at_top else at_bot)" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1966 | shows "filterlim (\<lambda>x. c * h x) G F" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1967 | using assms filterlim_tendsto_pos_mult_at_top[OF tendsto_const[of c], of h F] | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1968 | filterlim_tendsto_neg_mult_at_bot[OF tendsto_const[of c], of h F] by simp | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 1969 | |
| 56330 | 1970 | lemma filterlim_pow_at_top: | 
| 63721 | 1971 | fixes f :: "'a \<Rightarrow> real" | 
| 63546 | 1972 | assumes "0 < n" | 
| 1973 | and f: "LIM x F. f x :> at_top" | |
| 56330 | 1974 | shows "LIM x F. (f x)^n :: real :> at_top" | 
| 63546 | 1975 | using \<open>0 < n\<close> | 
| 1976 | proof (induct n) | |
| 1977 | case 0 | |
| 1978 | then show ?case by simp | |
| 1979 | next | |
| 56330 | 1980 | case (Suc n) with f show ?case | 
| 1981 | by (cases "n = 0") (auto intro!: filterlim_at_top_mult_at_top) | |
| 63546 | 1982 | qed | 
| 56330 | 1983 | |
| 1984 | lemma filterlim_pow_at_bot_even: | |
| 1985 | fixes f :: "real \<Rightarrow> real" | |
| 1986 | shows "0 < n \<Longrightarrow> LIM x F. f x :> at_bot \<Longrightarrow> even n \<Longrightarrow> LIM x F. (f x)^n :> at_top" | |
| 1987 | using filterlim_pow_at_top[of n "\<lambda>x. - f x" F] by (simp add: filterlim_uminus_at_top) | |
| 1988 | ||
| 1989 | lemma filterlim_pow_at_bot_odd: | |
| 1990 | fixes f :: "real \<Rightarrow> real" | |
| 1991 | shows "0 < n \<Longrightarrow> LIM x F. f x :> at_bot \<Longrightarrow> odd n \<Longrightarrow> LIM x F. (f x)^n :> at_bot" | |
| 1992 | using filterlim_pow_at_top[of n "\<lambda>x. - f x" F] by (simp add: filterlim_uminus_at_bot) | |
| 1993 | ||
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1994 | lemma filterlim_power_at_infinity [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1995 | fixes F and f :: "'a \<Rightarrow> 'b :: real_normed_div_algebra" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1996 | assumes "filterlim f at_infinity F" "n > 0" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1997 | shows "filterlim (\<lambda>x. f x ^ n) at_infinity F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1998 | by (rule filterlim_norm_at_top_imp_at_infinity) | 
| 68611 | 1999 | (auto simp: norm_power intro!: filterlim_pow_at_top assms | 
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 2000 | intro: filterlim_at_infinity_imp_norm_at_top) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 2001 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2002 | lemma filterlim_tendsto_add_at_top: | 
| 61973 | 2003 | assumes f: "(f \<longlongrightarrow> c) F" | 
| 63546 | 2004 | and g: "LIM x F. g x :> at_top" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2005 | shows "LIM x F. (f x + g x :: real) :> at_top" | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2006 | unfolding filterlim_at_top_gt[where c=0] | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2007 | proof safe | 
| 63546 | 2008 | fix Z :: real | 
| 2009 | assume "0 < Z" | |
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2010 | from f have "eventually (\<lambda>x. c - 1 < f x) F" | 
| 61810 | 2011 | by (auto dest!: tendstoD[where e=1] elim!: eventually_mono simp: dist_real_def) | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 2012 | moreover from g have "eventually (\<lambda>x. Z - (c - 1) \<le> g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2013 | unfolding filterlim_at_top by auto | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 2014 | ultimately show "eventually (\<lambda>x. Z \<le> f x + g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2015 | by eventually_elim simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2016 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2017 | |
| 50347 | 2018 | lemma LIM_at_top_divide: | 
| 2019 | fixes f g :: "'a \<Rightarrow> real" | |
| 61973 | 2020 | assumes f: "(f \<longlongrightarrow> a) F" "0 < a" | 
| 63546 | 2021 | and g: "(g \<longlongrightarrow> 0) F" "eventually (\<lambda>x. 0 < g x) F" | 
| 50347 | 2022 | shows "LIM x F. f x / g x :> at_top" | 
| 2023 | unfolding divide_inverse | |
| 2024 | by (rule filterlim_tendsto_pos_mult_at_top[OF f]) (rule filterlim_inverse_at_top[OF g]) | |
| 2025 | ||
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2026 | lemma filterlim_at_top_add_at_top: | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2027 | assumes f: "LIM x F. f x :> at_top" | 
| 63546 | 2028 | and g: "LIM x F. g x :> at_top" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2029 | shows "LIM x F. (f x + g x :: real) :> at_top" | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2030 | unfolding filterlim_at_top_gt[where c=0] | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2031 | proof safe | 
| 63546 | 2032 | fix Z :: real | 
| 2033 | assume "0 < Z" | |
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 2034 | from f have "eventually (\<lambda>x. 0 \<le> f x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2035 | unfolding filterlim_at_top by auto | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 2036 | moreover from g have "eventually (\<lambda>x. Z \<le> g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2037 | unfolding filterlim_at_top by auto | 
| 50346 
a75c6429c3c3
add filterlim rules for eventually monotone bijective functions; mirror rules for at_top, at_bot; apply them to prove convergence of arctan at infinity and tan at pi/2
 hoelzl parents: 
50331diff
changeset | 2038 | ultimately show "eventually (\<lambda>x. Z \<le> f x + g x) F" | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2039 | by eventually_elim simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2040 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 2041 | |
| 50331 | 2042 | lemma tendsto_divide_0: | 
| 61076 | 2043 |   fixes f :: "_ \<Rightarrow> 'a::{real_normed_div_algebra, division_ring}"
 | 
| 61973 | 2044 | assumes f: "(f \<longlongrightarrow> c) F" | 
| 63546 | 2045 | and g: "LIM x F. g x :> at_infinity" | 
| 61973 | 2046 | shows "((\<lambda>x. f x / g x) \<longlongrightarrow> 0) F" | 
| 63546 | 2047 | using tendsto_mult[OF f filterlim_compose[OF tendsto_inverse_0 g]] | 
| 2048 | by (simp add: divide_inverse) | |
| 50331 | 2049 | |
| 2050 | lemma linear_plus_1_le_power: | |
| 2051 | fixes x :: real | |
| 2052 | assumes x: "0 \<le> x" | |
| 2053 | shows "real n * x + 1 \<le> (x + 1) ^ n" | |
| 2054 | proof (induct n) | |
| 63546 | 2055 | case 0 | 
| 2056 | then show ?case by simp | |
| 2057 | next | |
| 50331 | 2058 | case (Suc n) | 
| 63546 | 2059 | from x have "real (Suc n) * x + 1 \<le> (x + 1) * (real n * x + 1)" | 
| 2060 | by (simp add: field_simps) | |
| 50331 | 2061 | also have "\<dots> \<le> (x + 1)^Suc n" | 
| 2062 | using Suc x by (simp add: mult_left_mono) | |
| 2063 | finally show ?case . | |
| 63546 | 2064 | qed | 
| 50331 | 2065 | |
| 2066 | lemma filterlim_realpow_sequentially_gt1: | |
| 2067 | fixes x :: "'a :: real_normed_div_algebra" | |
| 2068 | assumes x[arith]: "1 < norm x" | |
| 2069 | shows "LIM n sequentially. x ^ n :> at_infinity" | |
| 2070 | proof (intro filterlim_at_infinity[THEN iffD2] allI impI) | |
| 63546 | 2071 | fix y :: real | 
| 2072 | assume "0 < y" | |
| 72219 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 2073 | obtain N :: nat where "y < real N * (norm x - 1)" | 
| 
0f38c96a0a74
tidying up some theorem statements
 paulson <lp15@cam.ac.uk> parents: 
71837diff
changeset | 2074 | by (meson diff_gt_0_iff_gt reals_Archimedean3 x) | 
| 63546 | 2075 | also have "\<dots> \<le> real N * (norm x - 1) + 1" | 
| 2076 | by simp | |
| 2077 | also have "\<dots> \<le> (norm x - 1 + 1) ^ N" | |
| 2078 | by (rule linear_plus_1_le_power) simp | |
| 2079 | also have "\<dots> = norm x ^ N" | |
| 2080 | by simp | |
| 50331 | 2081 | finally have "\<forall>n\<ge>N. y \<le> norm x ^ n" | 
| 2082 | by (metis order_less_le_trans power_increasing order_less_imp_le x) | |
| 2083 | then show "eventually (\<lambda>n. y \<le> norm (x ^ n)) sequentially" | |
| 2084 | unfolding eventually_sequentially | |
| 2085 | by (auto simp: norm_power) | |
| 2086 | qed simp | |
| 2087 | ||
| 51471 | 2088 | |
| 66456 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2089 | lemma filterlim_divide_at_infinity: | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2090 | fixes f g :: "'a \<Rightarrow> 'a :: real_normed_field" | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2091 | assumes "filterlim f (nhds c) F" "filterlim g (at 0) F" "c \<noteq> 0" | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2092 | shows "filterlim (\<lambda>x. f x / g x) at_infinity F" | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2093 | proof - | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2094 | have "filterlim (\<lambda>x. f x * inverse (g x)) at_infinity F" | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2095 | by (intro tendsto_mult_filterlim_at_infinity[OF assms(1,3)] | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2096 | filterlim_compose [OF filterlim_inverse_at_infinity assms(2)]) | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2097 | thus ?thesis by (simp add: field_simps) | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2098 | qed | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 2099 | |
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2100 | subsection \<open>Floor and Ceiling\<close> | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2101 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2102 | lemma eventually_floor_less: | 
| 63546 | 2103 |   fixes f :: "'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2104 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 2105 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2106 | shows "\<forall>\<^sub>F x in F. of_int (floor l) < f x" | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2107 | by (intro order_tendstoD[OF f]) (metis Ints_of_int antisym_conv2 floor_correct l) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2108 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2109 | lemma eventually_less_ceiling: | 
| 63546 | 2110 |   fixes f :: "'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2111 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 2112 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2113 | shows "\<forall>\<^sub>F x in F. f x < of_int (ceiling l)" | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2114 | by (intro order_tendstoD[OF f]) (metis Ints_of_int l le_of_int_ceiling less_le) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2115 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2116 | lemma eventually_floor_eq: | 
| 63546 | 2117 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2118 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 2119 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2120 | shows "\<forall>\<^sub>F x in F. floor (f x) = floor l" | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2121 | using eventually_floor_less[OF assms] eventually_less_ceiling[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2122 | by eventually_elim (meson floor_less_iff less_ceiling_iff not_less_iff_gr_or_eq) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2123 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2124 | lemma eventually_ceiling_eq: | 
| 63546 | 2125 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2126 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 2127 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2128 | shows "\<forall>\<^sub>F x in F. ceiling (f x) = ceiling l" | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2129 | using eventually_floor_less[OF assms] eventually_less_ceiling[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2130 | by eventually_elim (meson floor_less_iff less_ceiling_iff not_less_iff_gr_or_eq) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2131 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2132 | lemma tendsto_of_int_floor: | 
| 63546 | 2133 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2134 | assumes "(f \<longlongrightarrow> l) F" | 
| 63546 | 2135 | and "l \<notin> \<int>" | 
| 2136 |   shows "((\<lambda>x. of_int (floor (f x)) :: 'c::{ring_1,topological_space}) \<longlongrightarrow> of_int (floor l)) F"
 | |
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2137 | using eventually_floor_eq[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2138 | by (simp add: eventually_mono topological_tendstoI) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2139 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2140 | lemma tendsto_of_int_ceiling: | 
| 63546 | 2141 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2142 | assumes "(f \<longlongrightarrow> l) F" | 
| 63546 | 2143 | and "l \<notin> \<int>" | 
| 2144 |   shows "((\<lambda>x. of_int (ceiling (f x)):: 'c::{ring_1,topological_space}) \<longlongrightarrow> of_int (ceiling l)) F"
 | |
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2145 | using eventually_ceiling_eq[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2146 | by (simp add: eventually_mono topological_tendstoI) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2147 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2148 | lemma continuous_on_of_int_floor: | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2149 |   "continuous_on (UNIV - \<int>::'a::{order_topology, floor_ceiling} set)
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2150 |     (\<lambda>x. of_int (floor x)::'b::{ring_1, topological_space})"
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2151 | unfolding continuous_on_def | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2152 | by (auto intro!: tendsto_of_int_floor) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2153 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2154 | lemma continuous_on_of_int_ceiling: | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2155 |   "continuous_on (UNIV - \<int>::'a::{order_topology, floor_ceiling} set)
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2156 |     (\<lambda>x. of_int (ceiling x)::'b::{ring_1, topological_space})"
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2157 | unfolding continuous_on_def | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2158 | by (auto intro!: tendsto_of_int_ceiling) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2159 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 2160 | |
| 60758 | 2161 | subsection \<open>Limits of Sequences\<close> | 
| 51526 | 2162 | |
| 62368 | 2163 | lemma [trans]: "X = Y \<Longrightarrow> Y \<longlonglongrightarrow> z \<Longrightarrow> X \<longlonglongrightarrow> z" | 
| 51526 | 2164 | by simp | 
| 2165 | ||
| 2166 | lemma LIMSEQ_iff: | |
| 2167 | fixes L :: "'a::real_normed_vector" | |
| 61969 | 2168 | shows "(X \<longlonglongrightarrow> L) = (\<forall>r>0. \<exists>no. \<forall>n \<ge> no. norm (X n - L) < r)" | 
| 60017 
b785d6d06430
Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
 paulson <lp15@cam.ac.uk> parents: 
59867diff
changeset | 2169 | unfolding lim_sequentially dist_norm .. | 
| 51526 | 2170 | |
| 63546 | 2171 | lemma LIMSEQ_I: "(\<And>r. 0 < r \<Longrightarrow> \<exists>no. \<forall>n\<ge>no. norm (X n - L) < r) \<Longrightarrow> X \<longlonglongrightarrow> L" | 
| 2172 | for L :: "'a::real_normed_vector" | |
| 2173 | by (simp add: LIMSEQ_iff) | |
| 2174 | ||
| 2175 | lemma LIMSEQ_D: "X \<longlonglongrightarrow> L \<Longrightarrow> 0 < r \<Longrightarrow> \<exists>no. \<forall>n\<ge>no. norm (X n - L) < r" | |
| 2176 | for L :: "'a::real_normed_vector" | |
| 2177 | by (simp add: LIMSEQ_iff) | |
| 2178 | ||
| 2179 | lemma LIMSEQ_linear: "X \<longlonglongrightarrow> x \<Longrightarrow> l > 0 \<Longrightarrow> (\<lambda> n. X (n * l)) \<longlonglongrightarrow> x" | |
| 51526 | 2180 | unfolding tendsto_def eventually_sequentially | 
| 57512 
cc97b347b301
reduced name variants for assoc and commute on plus and mult
 haftmann parents: 
57447diff
changeset | 2181 | by (metis div_le_dividend div_mult_self1_is_m le_trans mult.commute) | 
| 51526 | 2182 | |
| 63546 | 2183 | |
| 2184 | text \<open>Transformation of limit.\<close> | |
| 2185 | ||
| 2186 | lemma Lim_transform: "(g \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f x - g x) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> a) F" | |
| 2187 | for a b :: "'a::real_normed_vector" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2188 | using tendsto_add [of g a F "\<lambda>x. f x - g x" 0] by simp | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2189 | |
| 63546 | 2190 | lemma Lim_transform2: "(f \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f x - g x) \<longlongrightarrow> 0) F \<Longrightarrow> (g \<longlongrightarrow> a) F" | 
| 2191 | for a b :: "'a::real_normed_vector" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2192 | by (erule Lim_transform) (simp add: tendsto_minus_cancel) | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2193 | |
| 63546 | 2194 | proposition Lim_transform_eq: "((\<lambda>x. f x - g x) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> a) F \<longleftrightarrow> (g \<longlongrightarrow> a) F" | 
| 2195 | for a :: "'a::real_normed_vector" | |
| 2196 | using Lim_transform Lim_transform2 by blast | |
| 62379 
340738057c8c
An assortment of useful lemmas about sums, norm, etc. Also: norm_conv_dist [symmetric] is now a simprule!
 paulson <lp15@cam.ac.uk> parents: 
62369diff
changeset | 2197 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2198 | lemma Lim_transform_eventually: | 
| 70532 
fcf3b891ccb1
new material; rotated premises of Lim_transform_eventually
 paulson <lp15@cam.ac.uk> parents: 
70365diff
changeset | 2199 | "\<lbrakk>(f \<longlongrightarrow> l) F; eventually (\<lambda>x. f x = g x) F\<rbrakk> \<Longrightarrow> (g \<longlongrightarrow> l) F" | 
| 68615 | 2200 | using eventually_elim2 by (fastforce simp add: tendsto_def) | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2201 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2202 | lemma Lim_transform_within: | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2203 | assumes "(f \<longlongrightarrow> l) (at x within S)" | 
| 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2204 | and "0 < d" | 
| 63546 | 2205 | and "\<And>x'. x'\<in>S \<Longrightarrow> 0 < dist x' x \<Longrightarrow> dist x' x < d \<Longrightarrow> f x' = g x'" | 
| 61973 | 2206 | shows "(g \<longlongrightarrow> l) (at x within S)" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2207 | proof (rule Lim_transform_eventually) | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2208 | show "eventually (\<lambda>x. f x = g x) (at x within S)" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2209 | using assms by (auto simp: eventually_at) | 
| 63546 | 2210 | show "(f \<longlongrightarrow> l) (at x within S)" | 
| 2211 | by fact | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2212 | qed | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2213 | |
| 67706 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2214 | lemma filterlim_transform_within: | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2215 | assumes "filterlim g G (at x within S)" | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2216 | assumes "G \<le> F" "0<d" "(\<And>x'. x' \<in> S \<Longrightarrow> 0 < dist x' x \<Longrightarrow> dist x' x < d \<Longrightarrow> f x' = g x') " | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2217 | shows "filterlim f F (at x within S)" | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2218 | using assms | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2219 | apply (elim filterlim_mono_eventually) | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2220 | unfolding eventually_at by auto | 
| 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 2221 | |
| 63546 | 2222 | text \<open>Common case assuming being away from some crucial point like 0.\<close> | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2223 | lemma Lim_transform_away_within: | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2224 | fixes a b :: "'a::t1_space" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2225 | assumes "a \<noteq> b" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2226 | and "\<forall>x\<in>S. x \<noteq> a \<and> x \<noteq> b \<longrightarrow> f x = g x" | 
| 61973 | 2227 | and "(f \<longlongrightarrow> l) (at a within S)" | 
| 2228 | shows "(g \<longlongrightarrow> l) (at a within S)" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2229 | proof (rule Lim_transform_eventually) | 
| 63546 | 2230 | show "(f \<longlongrightarrow> l) (at a within S)" | 
| 2231 | by fact | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2232 | show "eventually (\<lambda>x. f x = g x) (at a within S)" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2233 | unfolding eventually_at_topological | 
| 63546 | 2234 |     by (rule exI [where x="- {b}"]) (simp add: open_Compl assms)
 | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2235 | qed | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2236 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2237 | lemma Lim_transform_away_at: | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2238 | fixes a b :: "'a::t1_space" | 
| 63546 | 2239 | assumes ab: "a \<noteq> b" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2240 | and fg: "\<forall>x. x \<noteq> a \<and> x \<noteq> b \<longrightarrow> f x = g x" | 
| 61973 | 2241 | and fl: "(f \<longlongrightarrow> l) (at a)" | 
| 2242 | shows "(g \<longlongrightarrow> l) (at a)" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2243 | using Lim_transform_away_within[OF ab, of UNIV f g l] fg fl by simp | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2244 | |
| 63546 | 2245 | text \<open>Alternatively, within an open set.\<close> | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2246 | lemma Lim_transform_within_open: | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2247 | assumes "(f \<longlongrightarrow> l) (at a within T)" | 
| 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2248 | and "open s" and "a \<in> s" | 
| 63546 | 2249 | and "\<And>x. x\<in>s \<Longrightarrow> x \<noteq> a \<Longrightarrow> f x = g x" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2250 | shows "(g \<longlongrightarrow> l) (at a within T)" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2251 | proof (rule Lim_transform_eventually) | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2252 | show "eventually (\<lambda>x. f x = g x) (at a within T)" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2253 | unfolding eventually_at_topological | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2254 | using assms by auto | 
| 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2255 | show "(f \<longlongrightarrow> l) (at a within T)" by fact | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2256 | qed | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2257 | |
| 63546 | 2258 | |
| 2259 | text \<open>A congruence rule allowing us to transform limits assuming not at point.\<close> | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2260 | |
| 72220 | 2261 | lemma Lim_cong_within: | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2262 | assumes "a = b" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2263 | and "x = y" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2264 | and "S = T" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2265 | and "\<And>x. x \<noteq> b \<Longrightarrow> x \<in> T \<Longrightarrow> f x = g x" | 
| 61973 | 2266 | shows "(f \<longlongrightarrow> x) (at a within S) \<longleftrightarrow> (g \<longlongrightarrow> y) (at b within T)" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2267 | unfolding tendsto_def eventually_at_topological | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2268 | using assms by simp | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2269 | |
| 63546 | 2270 | text \<open>An unbounded sequence's inverse tends to 0.\<close> | 
| 65578 
e4997c181cce
New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
 paulson <lp15@cam.ac.uk> parents: 
65204diff
changeset | 2271 | lemma LIMSEQ_inverse_zero: | 
| 
e4997c181cce
New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
 paulson <lp15@cam.ac.uk> parents: 
65204diff
changeset | 2272 | assumes "\<And>r::real. \<exists>N. \<forall>n\<ge>N. r < X n" | 
| 
e4997c181cce
New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
 paulson <lp15@cam.ac.uk> parents: 
65204diff
changeset | 2273 | shows "(\<lambda>n. inverse (X n)) \<longlonglongrightarrow> 0" | 
| 51526 | 2274 | apply (rule filterlim_compose[OF tendsto_inverse_0]) | 
| 68615 | 2275 | by (metis assms eventually_at_top_linorderI filterlim_at_top_dense filterlim_at_top_imp_at_infinity) | 
| 51526 | 2276 | |
| 69593 | 2277 | text \<open>The sequence \<^term>\<open>1/n\<close> tends to 0 as \<^term>\<open>n\<close> tends to infinity.\<close> | 
| 63546 | 2278 | lemma LIMSEQ_inverse_real_of_nat: "(\<lambda>n. inverse (real (Suc n))) \<longlonglongrightarrow> 0" | 
| 51526 | 2279 | by (metis filterlim_compose tendsto_inverse_0 filterlim_mono order_refl filterlim_Suc | 
| 63546 | 2280 | filterlim_compose[OF filterlim_real_sequentially] at_top_le_at_infinity) | 
| 2281 | ||
| 2282 | text \<open> | |
| 69593 | 2283 | The sequence \<^term>\<open>r + 1/n\<close> tends to \<^term>\<open>r\<close> as \<^term>\<open>n\<close> tends to | 
| 63546 | 2284 | infinity is now easily proved. | 
| 2285 | \<close> | |
| 2286 | ||
| 2287 | lemma LIMSEQ_inverse_real_of_nat_add: "(\<lambda>n. r + inverse (real (Suc n))) \<longlonglongrightarrow> r" | |
| 51526 | 2288 | using tendsto_add [OF tendsto_const LIMSEQ_inverse_real_of_nat] by auto | 
| 2289 | ||
| 63546 | 2290 | lemma LIMSEQ_inverse_real_of_nat_add_minus: "(\<lambda>n. r + -inverse (real (Suc n))) \<longlonglongrightarrow> r" | 
| 51526 | 2291 | using tendsto_add [OF tendsto_const tendsto_minus [OF LIMSEQ_inverse_real_of_nat]] | 
| 2292 | by auto | |
| 2293 | ||
| 63546 | 2294 | lemma LIMSEQ_inverse_real_of_nat_add_minus_mult: "(\<lambda>n. r * (1 + - inverse (real (Suc n)))) \<longlonglongrightarrow> r" | 
| 51526 | 2295 | using tendsto_mult [OF tendsto_const LIMSEQ_inverse_real_of_nat_add_minus [of 1]] | 
| 2296 | by auto | |
| 2297 | ||
| 61973 | 2298 | lemma lim_inverse_n: "((\<lambda>n. inverse(of_nat n)) \<longlongrightarrow> (0::'a::real_normed_field)) sequentially" | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2299 | using lim_1_over_n by (simp add: inverse_eq_divide) | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2300 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2301 | lemma lim_inverse_n': "((\<lambda>n. 1 / n) \<longlongrightarrow> 0) sequentially" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2302 | using lim_inverse_n | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2303 | by (simp add: inverse_eq_divide) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2304 | |
| 61969 | 2305 | lemma LIMSEQ_Suc_n_over_n: "(\<lambda>n. of_nat (Suc n) / of_nat n :: 'a :: real_normed_field) \<longlonglongrightarrow> 1" | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2306 | proof (rule Lim_transform_eventually) | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2307 | show "eventually (\<lambda>n. 1 + inverse (of_nat n :: 'a) = of_nat (Suc n) / of_nat n) sequentially" | 
| 63546 | 2308 | using eventually_gt_at_top[of "0::nat"] | 
| 2309 | by eventually_elim (simp add: field_simps) | |
| 61969 | 2310 | have "(\<lambda>n. 1 + inverse (of_nat n) :: 'a) \<longlonglongrightarrow> 1 + 0" | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2311 | by (intro tendsto_add tendsto_const lim_inverse_n) | 
| 63546 | 2312 | then show "(\<lambda>n. 1 + inverse (of_nat n) :: 'a) \<longlonglongrightarrow> 1" | 
| 2313 | by simp | |
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2314 | qed | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2315 | |
| 61969 | 2316 | lemma LIMSEQ_n_over_Suc_n: "(\<lambda>n. of_nat n / of_nat (Suc n) :: 'a :: real_normed_field) \<longlonglongrightarrow> 1" | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2317 | proof (rule Lim_transform_eventually) | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2318 | show "eventually (\<lambda>n. inverse (of_nat (Suc n) / of_nat n :: 'a) = | 
| 63546 | 2319 | of_nat n / of_nat (Suc n)) sequentially" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2320 | using eventually_gt_at_top[of "0::nat"] | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2321 | by eventually_elim (simp add: field_simps del: of_nat_Suc) | 
| 61969 | 2322 | have "(\<lambda>n. inverse (of_nat (Suc n) / of_nat n :: 'a)) \<longlonglongrightarrow> inverse 1" | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2323 | by (intro tendsto_inverse LIMSEQ_Suc_n_over_n) simp_all | 
| 63546 | 2324 | then show "(\<lambda>n. inverse (of_nat (Suc n) / of_nat n :: 'a)) \<longlonglongrightarrow> 1" | 
| 2325 | by simp | |
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2326 | qed | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2327 | |
| 63546 | 2328 | |
| 60758 | 2329 | subsection \<open>Convergence on sequences\<close> | 
| 51526 | 2330 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2331 | lemma convergent_cong: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2332 | assumes "eventually (\<lambda>x. f x = g x) sequentially" | 
| 63546 | 2333 | shows "convergent f \<longleftrightarrow> convergent g" | 
| 2334 | unfolding convergent_def | |
| 2335 | by (subst filterlim_cong[OF refl refl assms]) (rule refl) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2336 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2337 | lemma convergent_Suc_iff: "convergent (\<lambda>n. f (Suc n)) \<longleftrightarrow> convergent f" | 
| 71827 | 2338 | by (auto simp: convergent_def filterlim_sequentially_Suc) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2339 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2340 | lemma convergent_ignore_initial_segment: "convergent (\<lambda>n. f (n + m)) = convergent f" | 
| 63546 | 2341 | proof (induct m arbitrary: f) | 
| 2342 | case 0 | |
| 2343 | then show ?case by simp | |
| 2344 | next | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2345 | case (Suc m) | 
| 63546 | 2346 | have "convergent (\<lambda>n. f (n + Suc m)) \<longleftrightarrow> convergent (\<lambda>n. f (Suc n + m))" | 
| 2347 | by simp | |
| 2348 | also have "\<dots> \<longleftrightarrow> convergent (\<lambda>n. f (n + m))" | |
| 2349 | by (rule convergent_Suc_iff) | |
| 2350 | also have "\<dots> \<longleftrightarrow> convergent f" | |
| 2351 | by (rule Suc) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2352 | finally show ?case . | 
| 63546 | 2353 | qed | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2354 | |
| 51526 | 2355 | lemma convergent_add: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2356 | fixes X Y :: "nat \<Rightarrow> 'a::topological_monoid_add" | 
| 51526 | 2357 | assumes "convergent (\<lambda>n. X n)" | 
| 63546 | 2358 | and "convergent (\<lambda>n. Y n)" | 
| 51526 | 2359 | shows "convergent (\<lambda>n. X n + Y n)" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 2360 | using assms unfolding convergent_def by (blast intro: tendsto_add) | 
| 51526 | 2361 | |
| 64267 | 2362 | lemma convergent_sum: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2363 | fixes X :: "'a \<Rightarrow> nat \<Rightarrow> 'b::topological_comm_monoid_add" | 
| 63915 | 2364 | shows "(\<And>i. i \<in> A \<Longrightarrow> convergent (\<lambda>n. X i n)) \<Longrightarrow> convergent (\<lambda>n. \<Sum>i\<in>A. X i n)" | 
| 2365 | by (induct A rule: infinite_finite_induct) (simp_all add: convergent_const convergent_add) | |
| 51526 | 2366 | |
| 2367 | lemma (in bounded_linear) convergent: | |
| 2368 | assumes "convergent (\<lambda>n. X n)" | |
| 2369 | shows "convergent (\<lambda>n. f (X n))" | |
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 2370 | using assms unfolding convergent_def by (blast intro: tendsto) | 
| 51526 | 2371 | |
| 2372 | lemma (in bounded_bilinear) convergent: | |
| 63546 | 2373 | assumes "convergent (\<lambda>n. X n)" | 
| 2374 | and "convergent (\<lambda>n. Y n)" | |
| 51526 | 2375 | shows "convergent (\<lambda>n. X n ** Y n)" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 2376 | using assms unfolding convergent_def by (blast intro: tendsto) | 
| 51526 | 2377 | |
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2378 | lemma convergent_minus_iff: | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2379 | fixes X :: "nat \<Rightarrow> 'a::topological_group_add" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2380 | shows "convergent X \<longleftrightarrow> convergent (\<lambda>n. - X n)" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2381 | unfolding convergent_def by (force dest: tendsto_minus) | 
| 51526 | 2382 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2383 | lemma convergent_diff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2384 | fixes X Y :: "nat \<Rightarrow> 'a::topological_group_add" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2385 | assumes "convergent (\<lambda>n. X n)" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2386 | assumes "convergent (\<lambda>n. Y n)" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2387 | shows "convergent (\<lambda>n. X n - Y n)" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 2388 | using assms unfolding convergent_def by (blast intro: tendsto_diff) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2389 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2390 | lemma convergent_norm: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2391 | assumes "convergent f" | 
| 63546 | 2392 | shows "convergent (\<lambda>n. norm (f n))" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2393 | proof - | 
| 63546 | 2394 | from assms have "f \<longlonglongrightarrow> lim f" | 
| 2395 | by (simp add: convergent_LIMSEQ_iff) | |
| 2396 | then have "(\<lambda>n. norm (f n)) \<longlonglongrightarrow> norm (lim f)" | |
| 2397 | by (rule tendsto_norm) | |
| 2398 | then show ?thesis | |
| 2399 | by (auto simp: convergent_def) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2400 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2401 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2402 | lemma convergent_of_real: | 
| 63546 | 2403 | "convergent f \<Longrightarrow> convergent (\<lambda>n. of_real (f n) :: 'a::real_normed_algebra_1)" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2404 | unfolding convergent_def by (blast intro!: tendsto_of_real) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2405 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2406 | lemma convergent_add_const_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2407 | "convergent (\<lambda>n. c + f n :: 'a::topological_ab_group_add) \<longleftrightarrow> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2408 | proof | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2409 | assume "convergent (\<lambda>n. c + f n)" | 
| 63546 | 2410 | from convergent_diff[OF this convergent_const[of c]] show "convergent f" | 
| 2411 | by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2412 | next | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2413 | assume "convergent f" | 
| 63546 | 2414 | from convergent_add[OF convergent_const[of c] this] show "convergent (\<lambda>n. c + f n)" | 
| 2415 | by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2416 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2417 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2418 | lemma convergent_add_const_right_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2419 | "convergent (\<lambda>n. f n + c :: 'a::topological_ab_group_add) \<longleftrightarrow> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2420 | using convergent_add_const_iff[of c f] by (simp add: add_ac) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2421 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2422 | lemma convergent_diff_const_right_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2423 | "convergent (\<lambda>n. f n - c :: 'a::topological_ab_group_add) \<longleftrightarrow> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2424 | using convergent_add_const_right_iff[of f "-c"] by (simp add: add_ac) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2425 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2426 | lemma convergent_mult: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2427 | fixes X Y :: "nat \<Rightarrow> 'a::topological_semigroup_mult" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2428 | assumes "convergent (\<lambda>n. X n)" | 
| 63546 | 2429 | and "convergent (\<lambda>n. Y n)" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2430 | shows "convergent (\<lambda>n. X n * Y n)" | 
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 2431 | using assms unfolding convergent_def by (blast intro: tendsto_mult) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2432 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2433 | lemma convergent_mult_const_iff: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2434 | assumes "c \<noteq> 0" | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2435 |   shows "convergent (\<lambda>n. c * f n :: 'a::{field,topological_semigroup_mult}) \<longleftrightarrow> convergent f"
 | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2436 | proof | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2437 | assume "convergent (\<lambda>n. c * f n)" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2438 | from assms convergent_mult[OF this convergent_const[of "inverse c"]] | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2439 | show "convergent f" by (simp add: field_simps) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2440 | next | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2441 | assume "convergent f" | 
| 63546 | 2442 | from convergent_mult[OF convergent_const[of c] this] show "convergent (\<lambda>n. c * f n)" | 
| 2443 | by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2444 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2445 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2446 | lemma convergent_mult_const_right_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2447 |   fixes c :: "'a::{field,topological_semigroup_mult}"
 | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2448 | assumes "c \<noteq> 0" | 
| 63546 | 2449 | shows "convergent (\<lambda>n. f n * c) \<longleftrightarrow> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2450 | using convergent_mult_const_iff[OF assms, of f] by (simp add: mult_ac) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2451 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2452 | lemma convergent_imp_Bseq: "convergent f \<Longrightarrow> Bseq f" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2453 | by (simp add: Cauchy_Bseq convergent_Cauchy) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2454 | |
| 51526 | 2455 | |
| 60758 | 2456 | text \<open>A monotone sequence converges to its least upper bound.\<close> | 
| 51526 | 2457 | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2458 | lemma LIMSEQ_incseq_SUP: | 
| 63546 | 2459 |   fixes X :: "nat \<Rightarrow> 'a::{conditionally_complete_linorder,linorder_topology}"
 | 
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2460 | assumes u: "bdd_above (range X)" | 
| 63546 | 2461 | and X: "incseq X" | 
| 61969 | 2462 | shows "X \<longlonglongrightarrow> (SUP i. X i)" | 
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2463 | by (rule order_tendstoI) | 
| 63546 | 2464 | (auto simp: eventually_sequentially u less_cSUP_iff | 
| 2465 | intro: X[THEN incseqD] less_le_trans cSUP_lessD[OF u]) | |
| 51526 | 2466 | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2467 | lemma LIMSEQ_decseq_INF: | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2468 |   fixes X :: "nat \<Rightarrow> 'a::{conditionally_complete_linorder, linorder_topology}"
 | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2469 | assumes u: "bdd_below (range X)" | 
| 63546 | 2470 | and X: "decseq X" | 
| 61969 | 2471 | shows "X \<longlonglongrightarrow> (INF i. X i)" | 
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2472 | by (rule order_tendstoI) | 
| 63546 | 2473 | (auto simp: eventually_sequentially u cINF_less_iff | 
| 2474 | intro: X[THEN decseqD] le_less_trans less_cINF_D[OF u]) | |
| 2475 | ||
| 2476 | text \<open>Main monotonicity theorem.\<close> | |
| 2477 | ||
| 2478 | lemma Bseq_monoseq_convergent: "Bseq X \<Longrightarrow> monoseq X \<Longrightarrow> convergent X" | |
| 2479 | for X :: "nat \<Rightarrow> real" | |
| 2480 | by (auto simp: monoseq_iff convergent_def intro: LIMSEQ_decseq_INF LIMSEQ_incseq_SUP | |
| 2481 | dest: Bseq_bdd_above Bseq_bdd_below) | |
| 2482 | ||
| 2483 | lemma Bseq_mono_convergent: "Bseq X \<Longrightarrow> (\<forall>m n. m \<le> n \<longrightarrow> X m \<le> X n) \<Longrightarrow> convergent X" | |
| 2484 | for X :: "nat \<Rightarrow> real" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2485 | by (auto intro!: Bseq_monoseq_convergent incseq_imp_monoseq simp: incseq_def) | 
| 51526 | 2486 | |
| 63546 | 2487 | lemma monoseq_imp_convergent_iff_Bseq: "monoseq f \<Longrightarrow> convergent f \<longleftrightarrow> Bseq f" | 
| 2488 | for f :: "nat \<Rightarrow> real" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2489 | using Bseq_monoseq_convergent[of f] convergent_imp_Bseq[of f] by blast | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2490 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2491 | lemma Bseq_monoseq_convergent'_inc: | 
| 63546 | 2492 | fixes f :: "nat \<Rightarrow> real" | 
| 2493 | shows "Bseq (\<lambda>n. f (n + M)) \<Longrightarrow> (\<And>m n. M \<le> m \<Longrightarrow> m \<le> n \<Longrightarrow> f m \<le> f n) \<Longrightarrow> convergent f" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2494 | by (subst convergent_ignore_initial_segment [symmetric, of _ M]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2495 | (auto intro!: Bseq_monoseq_convergent simp: monoseq_def) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2496 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2497 | lemma Bseq_monoseq_convergent'_dec: | 
| 63546 | 2498 | fixes f :: "nat \<Rightarrow> real" | 
| 2499 | shows "Bseq (\<lambda>n. f (n + M)) \<Longrightarrow> (\<And>m n. M \<le> m \<Longrightarrow> m \<le> n \<Longrightarrow> f m \<ge> f n) \<Longrightarrow> convergent f" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2500 | by (subst convergent_ignore_initial_segment [symmetric, of _ M]) | 
| 63546 | 2501 | (auto intro!: Bseq_monoseq_convergent simp: monoseq_def) | 
| 2502 | ||
| 2503 | lemma Cauchy_iff: "Cauchy X \<longleftrightarrow> (\<forall>e>0. \<exists>M. \<forall>m\<ge>M. \<forall>n\<ge>M. norm (X m - X n) < e)" | |
| 2504 | for X :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 51526 | 2505 | unfolding Cauchy_def dist_norm .. | 
| 2506 | ||
| 63546 | 2507 | lemma CauchyI: "(\<And>e. 0 < e \<Longrightarrow> \<exists>M. \<forall>m\<ge>M. \<forall>n\<ge>M. norm (X m - X n) < e) \<Longrightarrow> Cauchy X" | 
| 2508 | for X :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 2509 | by (simp add: Cauchy_iff) | |
| 2510 | ||
| 2511 | lemma CauchyD: "Cauchy X \<Longrightarrow> 0 < e \<Longrightarrow> \<exists>M. \<forall>m\<ge>M. \<forall>n\<ge>M. norm (X m - X n) < e" | |
| 2512 | for X :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 2513 | by (simp add: Cauchy_iff) | |
| 51526 | 2514 | |
| 2515 | lemma incseq_convergent: | |
| 2516 | fixes X :: "nat \<Rightarrow> real" | |
| 63546 | 2517 | assumes "incseq X" | 
| 2518 | and "\<forall>i. X i \<le> B" | |
| 61969 | 2519 | obtains L where "X \<longlonglongrightarrow> L" "\<forall>i. X i \<le> L" | 
| 51526 | 2520 | proof atomize_elim | 
| 60758 | 2521 | from incseq_bounded[OF assms] \<open>incseq X\<close> Bseq_monoseq_convergent[of X] | 
| 61969 | 2522 | obtain L where "X \<longlonglongrightarrow> L" | 
| 51526 | 2523 | by (auto simp: convergent_def monoseq_def incseq_def) | 
| 61969 | 2524 | with \<open>incseq X\<close> show "\<exists>L. X \<longlonglongrightarrow> L \<and> (\<forall>i. X i \<le> L)" | 
| 51526 | 2525 | by (auto intro!: exI[of _ L] incseq_le) | 
| 2526 | qed | |
| 2527 | ||
| 2528 | lemma decseq_convergent: | |
| 2529 | fixes X :: "nat \<Rightarrow> real" | |
| 63546 | 2530 | assumes "decseq X" | 
| 2531 | and "\<forall>i. B \<le> X i" | |
| 61969 | 2532 | obtains L where "X \<longlonglongrightarrow> L" "\<forall>i. L \<le> X i" | 
| 51526 | 2533 | proof atomize_elim | 
| 60758 | 2534 | from decseq_bounded[OF assms] \<open>decseq X\<close> Bseq_monoseq_convergent[of X] | 
| 61969 | 2535 | obtain L where "X \<longlonglongrightarrow> L" | 
| 51526 | 2536 | by (auto simp: convergent_def monoseq_def decseq_def) | 
| 61969 | 2537 | with \<open>decseq X\<close> show "\<exists>L. X \<longlonglongrightarrow> L \<and> (\<forall>i. L \<le> X i)" | 
| 68532 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 2538 | by (auto intro!: exI[of _ L] decseq_ge) | 
| 51526 | 2539 | qed | 
| 2540 | ||
| 70694 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2541 | lemma monoseq_convergent: | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2542 | fixes X :: "nat \<Rightarrow> real" | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2543 | assumes X: "monoseq X" and B: "\<And>i. \<bar>X i\<bar> \<le> B" | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2544 | obtains L where "X \<longlonglongrightarrow> L" | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2545 | using X unfolding monoseq_iff | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2546 | proof | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2547 | assume "incseq X" | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2548 | show thesis | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2549 | using abs_le_D1 [OF B] incseq_convergent [OF \<open>incseq X\<close>] that by meson | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2550 | next | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2551 | assume "decseq X" | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2552 | show thesis | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2553 | using decseq_convergent [OF \<open>decseq X\<close>] that | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2554 | by (metis B abs_le_iff add.inverse_inverse neg_le_iff_le) | 
| 
ae37b8fbf023
New theory Equivalence_Measurable_On_Borel, with the HOL Light notion of measurable_on and its equivalence to ours
 paulson <lp15@cam.ac.uk> parents: 
70688diff
changeset | 2555 | qed | 
| 63546 | 2556 | |
| 77102 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2557 | subsection \<open>More about @{term filterlim} (thanks to Wenda Li)\<close>
 | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2558 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2559 | lemma filterlim_at_infinity_times: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2560 | fixes f :: "'a \<Rightarrow> 'b::real_normed_field" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2561 | assumes "filterlim f at_infinity F" "filterlim g at_infinity F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2562 | shows "filterlim (\<lambda>x. f x * g x) at_infinity F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2563 | proof - | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2564 | have "((\<lambda>x. inverse (f x) * inverse (g x)) \<longlongrightarrow> 0 * 0) F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2565 | by (intro tendsto_mult tendsto_inverse assms filterlim_compose[OF tendsto_inverse_0]) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2566 | then have "filterlim (\<lambda>x. inverse (f x) * inverse (g x)) (at 0) F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2567 | unfolding filterlim_at using assms | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2568 | by (auto intro: filterlim_at_infinity_imp_eventually_ne tendsto_imp_eventually_ne eventually_conj) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2569 | then show ?thesis | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2570 | by (subst filterlim_inverse_at_iff[symmetric]) simp_all | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2571 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2572 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2573 | lemma filterlim_at_top_at_bot[elim]: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2574 | fixes f::"'a \<Rightarrow> 'b::unbounded_dense_linorder" and F::"'a filter" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2575 | assumes top:"filterlim f at_top F" and bot: "filterlim f at_bot F" and "F\<noteq>bot" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2576 | shows False | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2577 | proof - | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2578 | obtain c::'b where True by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2579 | have "\<forall>\<^sub>F x in F. c < f x" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2580 | using top unfolding filterlim_at_top_dense by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2581 | moreover have "\<forall>\<^sub>F x in F. f x < c" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2582 | using bot unfolding filterlim_at_bot_dense by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2583 | ultimately have "\<forall>\<^sub>F x in F. c < f x \<and> f x < c" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2584 | using eventually_conj by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2585 | then have "\<forall>\<^sub>F x in F. False" by (auto elim:eventually_mono) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2586 | then show False using \<open>F\<noteq>bot\<close> by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2587 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2588 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2589 | lemma filterlim_at_top_nhds[elim]: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2590 |   fixes f::"'a \<Rightarrow> 'b::{unbounded_dense_linorder,order_topology}" and F::"'a filter"
 | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2591 | assumes top:"filterlim f at_top F" and tendsto: "(f \<longlongrightarrow> c) F" and "F\<noteq>bot" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2592 | shows False | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2593 | proof - | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2594 | obtain c'::'b where "c'>c" using gt_ex by blast | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2595 | have "\<forall>\<^sub>F x in F. c' < f x" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2596 | using top unfolding filterlim_at_top_dense by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2597 | moreover have "\<forall>\<^sub>F x in F. f x < c'" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2598 | using order_tendstoD[OF tendsto,of c'] \<open>c'>c\<close> by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2599 | ultimately have "\<forall>\<^sub>F x in F. c' < f x \<and> f x < c'" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2600 | using eventually_conj by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2601 | then have "\<forall>\<^sub>F x in F. False" by (auto elim:eventually_mono) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2602 | then show False using \<open>F\<noteq>bot\<close> by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2603 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2604 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2605 | lemma filterlim_at_bot_nhds[elim]: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2606 |   fixes f::"'a \<Rightarrow> 'b::{unbounded_dense_linorder,order_topology}" and F::"'a filter"
 | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2607 | assumes top:"filterlim f at_bot F" and tendsto: "(f \<longlongrightarrow> c) F" and "F\<noteq>bot" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2608 | shows False | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2609 | proof - | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2610 | obtain c'::'b where "c'<c" using lt_ex by blast | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2611 | have "\<forall>\<^sub>F x in F. c' > f x" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2612 | using top unfolding filterlim_at_bot_dense by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2613 | moreover have "\<forall>\<^sub>F x in F. f x > c'" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2614 | using order_tendstoD[OF tendsto,of c'] \<open>c'<c\<close> by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2615 | ultimately have "\<forall>\<^sub>F x in F. c' < f x \<and> f x < c'" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2616 | using eventually_conj by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2617 | then have "\<forall>\<^sub>F x in F. False" by (auto elim:eventually_mono) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2618 | then show False using \<open>F\<noteq>bot\<close> by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2619 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2620 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2621 | lemma eventually_times_inverse_1: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2622 |   fixes f::"'a \<Rightarrow> 'b::{field,t2_space}"
 | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2623 | assumes "(f \<longlongrightarrow> c) F" "c\<noteq>0" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2624 | shows "\<forall>\<^sub>F x in F. inverse (f x) * f x = 1" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2625 | by (smt (verit) assms eventually_mono mult.commute right_inverse tendsto_imp_eventually_ne) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2626 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2627 | lemma filterlim_at_infinity_divide_iff: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2628 | fixes f::"'a \<Rightarrow> 'b::real_normed_field" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2629 | assumes "(f \<longlongrightarrow> c) F" "c\<noteq>0" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2630 | shows "(LIM x F. f x / g x :> at_infinity) \<longleftrightarrow> (LIM x F. g x :> at 0)" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2631 | proof | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2632 | assume "LIM x F. f x / g x :> at_infinity" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2633 | then have "LIM x F. inverse (f x) * (f x / g x) :> at_infinity" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2634 | using assms tendsto_inverse tendsto_mult_filterlim_at_infinity by fastforce | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2635 | then have "LIM x F. inverse (g x) :> at_infinity" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2636 | apply (elim filterlim_mono_eventually) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2637 | using eventually_times_inverse_1[OF assms] | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2638 | by (auto elim:eventually_mono simp add:field_simps) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2639 | then show "filterlim g (at 0) F" using filterlim_inverse_at_iff[symmetric] by force | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2640 | next | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2641 | assume "filterlim g (at 0) F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2642 | then have "filterlim (\<lambda>x. inverse (g x)) at_infinity F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2643 | using filterlim_compose filterlim_inverse_at_infinity by blast | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2644 | then have "LIM x F. f x * inverse (g x) :> at_infinity" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2645 | using tendsto_mult_filterlim_at_infinity[OF assms, of "\<lambda>x. inverse(g x)"] | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2646 | by simp | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2647 | then show "LIM x F. f x / g x :> at_infinity" by (simp add: divide_inverse) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2648 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2649 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2650 | lemma filterlim_tendsto_pos_mult_at_top_iff: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2651 | fixes f::"'a \<Rightarrow> real" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2652 | assumes "(f \<longlongrightarrow> c) F" and "0 < c" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2653 | shows "(LIM x F. (f x * g x) :> at_top) \<longleftrightarrow> (LIM x F. g x :> at_top)" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2654 | proof | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2655 | assume "filterlim g at_top F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2656 | then show "LIM x F. f x * g x :> at_top" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2657 | using filterlim_tendsto_pos_mult_at_top[OF assms] by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2658 | next | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2659 | assume asm:"LIM x F. f x * g x :> at_top" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2660 | have "((\<lambda>x. inverse (f x)) \<longlongrightarrow> inverse c) F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2661 | using tendsto_inverse[OF assms(1)] \<open>0<c\<close> by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2662 | moreover have "inverse c >0" using assms(2) by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2663 | ultimately have "LIM x F. inverse (f x) * (f x * g x) :> at_top" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2664 | using filterlim_tendsto_pos_mult_at_top[OF _ _ asm,of "\<lambda>x. inverse (f x)" "inverse c"] by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2665 | then show "LIM x F. g x :> at_top" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2666 | apply (elim filterlim_mono_eventually) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2667 | apply simp_all[2] | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2668 | using eventually_times_inverse_1[OF assms(1)] \<open>c>0\<close> eventually_mono by fastforce | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2669 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2670 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2671 | lemma filterlim_tendsto_pos_mult_at_bot_iff: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2672 | fixes c :: real | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2673 | assumes "(f \<longlongrightarrow> c) F" "0 < c" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2674 | shows "(LIM x F. f x * g x :> at_bot) \<longleftrightarrow> filterlim g at_bot F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2675 | using filterlim_tendsto_pos_mult_at_top_iff[OF assms(1,2), of "\<lambda>x. - g x"] | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2676 | unfolding filterlim_uminus_at_bot by simp | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2677 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2678 | lemma filterlim_tendsto_neg_mult_at_top_iff: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2679 | fixes f::"'a \<Rightarrow> real" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2680 | assumes "(f \<longlongrightarrow> c) F" and "c < 0" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2681 | shows "(LIM x F. (f x * g x) :> at_top) \<longleftrightarrow> (LIM x F. g x :> at_bot)" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2682 | proof - | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2683 | have "(LIM x F. f x * g x :> at_top) = (LIM x F. - g x :> at_top)" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2684 | apply (rule filterlim_tendsto_pos_mult_at_top_iff[of "\<lambda>x. - f x" "-c" F "\<lambda>x. - g x", simplified]) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2685 | using assms by (auto intro: tendsto_intros ) | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2686 | also have "... = (LIM x F. g x :> at_bot)" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2687 | using filterlim_uminus_at_bot[symmetric] by auto | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2688 | finally show ?thesis . | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2689 | qed | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2690 | |
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2691 | lemma filterlim_tendsto_neg_mult_at_bot_iff: | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2692 | fixes c :: real | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2693 | assumes "(f \<longlongrightarrow> c) F" "0 > c" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2694 | shows "(LIM x F. f x * g x :> at_bot) \<longleftrightarrow> filterlim g at_top F" | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2695 | using filterlim_tendsto_neg_mult_at_top_iff[OF assms(1,2), of "\<lambda>x. - g x"] | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2696 | unfolding filterlim_uminus_at_top by simp | 
| 
780161d4b55c
Moved in some material from the AFP entry Winding_number_eval
 paulson <lp15@cam.ac.uk> parents: 
76724diff
changeset | 2697 | |
| 60758 | 2698 | subsection \<open>Power Sequences\<close> | 
| 51526 | 2699 | |
| 63546 | 2700 | lemma Bseq_realpow: "0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> Bseq (\<lambda>n. x ^ n)" | 
| 2701 | for x :: real | |
| 68615 | 2702 | by (metis decseq_bounded decseq_def power_decreasing zero_le_power) | 
| 63546 | 2703 | |
| 2704 | lemma monoseq_realpow: "0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> monoseq (\<lambda>n. x ^ n)" | |
| 2705 | for x :: real | |
| 68615 | 2706 | using monoseq_def power_decreasing by blast | 
| 63546 | 2707 | |
| 2708 | lemma convergent_realpow: "0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> convergent (\<lambda>n. x ^ n)" | |
| 2709 | for x :: real | |
| 2710 | by (blast intro!: Bseq_monoseq_convergent Bseq_realpow monoseq_realpow) | |
| 2711 | ||
| 2712 | lemma LIMSEQ_inverse_realpow_zero: "1 < x \<Longrightarrow> (\<lambda>n. inverse (x ^ n)) \<longlonglongrightarrow> 0" | |
| 2713 | for x :: real | |
| 51526 | 2714 | by (rule filterlim_compose[OF tendsto_inverse_0 filterlim_realpow_sequentially_gt1]) simp | 
| 2715 | ||
| 2716 | lemma LIMSEQ_realpow_zero: | |
| 63546 | 2717 | fixes x :: real | 
| 2718 | assumes "0 \<le> x" "x < 1" | |
| 2719 | shows "(\<lambda>n. x ^ n) \<longlonglongrightarrow> 0" | |
| 2720 | proof (cases "x = 0") | |
| 77221 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 2721 | case False | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 2722 | with \<open>0 \<le> x\<close> have "1 < inverse x" | 
| 
0cdb384bf56a
More new theorems from the number theory development
 paulson <lp15@cam.ac.uk> parents: 
77102diff
changeset | 2723 | using \<open>x < 1\<close> by (simp add: one_less_inverse) | 
| 63546 | 2724 | then have "(\<lambda>n. inverse (inverse x ^ n)) \<longlonglongrightarrow> 0" | 
| 51526 | 2725 | by (rule LIMSEQ_inverse_realpow_zero) | 
| 63546 | 2726 | then show ?thesis by (simp add: power_inverse) | 
| 2727 | next | |
| 2728 | case True | |
| 2729 | show ?thesis | |
| 2730 | by (rule LIMSEQ_imp_Suc) (simp add: True) | |
| 2731 | qed | |
| 2732 | ||
| 70723 
4e39d87c9737
imported new material mostly due to Sébastien Gouëzel
 paulson <lp15@cam.ac.uk> parents: 
70694diff
changeset | 2733 | lemma LIMSEQ_power_zero [tendsto_intros]: "norm x < 1 \<Longrightarrow> (\<lambda>n. x ^ n) \<longlonglongrightarrow> 0" | 
| 63546 | 2734 | for x :: "'a::real_normed_algebra_1" | 
| 2735 | apply (drule LIMSEQ_realpow_zero [OF norm_ge_zero]) | |
| 68615 | 2736 | by (simp add: Zfun_le norm_power_ineq tendsto_Zfun_iff) | 
| 51526 | 2737 | |
| 61969 | 2738 | lemma LIMSEQ_divide_realpow_zero: "1 < x \<Longrightarrow> (\<lambda>n. a / (x ^ n) :: real) \<longlonglongrightarrow> 0" | 
| 51526 | 2739 | by (rule tendsto_divide_0 [OF tendsto_const filterlim_realpow_sequentially_gt1]) simp | 
| 2740 | ||
| 63556 | 2741 | lemma | 
| 2742 | tendsto_power_zero: | |
| 2743 | fixes x::"'a::real_normed_algebra_1" | |
| 2744 | assumes "filterlim f at_top F" | |
| 2745 | assumes "norm x < 1" | |
| 2746 | shows "((\<lambda>y. x ^ (f y)) \<longlongrightarrow> 0) F" | |
| 2747 | proof (rule tendstoI) | |
| 2748 | fix e::real assume "0 < e" | |
| 2749 | from tendstoD[OF LIMSEQ_power_zero[OF \<open>norm x < 1\<close>] \<open>0 < e\<close>] | |
| 2750 | have "\<forall>\<^sub>F xa in sequentially. norm (x ^ xa) < e" | |
| 2751 | by simp | |
| 2752 | then obtain N where N: "norm (x ^ n) < e" if "n \<ge> N" for n | |
| 2753 | by (auto simp: eventually_sequentially) | |
| 2754 | have "\<forall>\<^sub>F i in F. f i \<ge> N" | |
| 2755 | using \<open>filterlim f sequentially F\<close> | |
| 2756 | by (simp add: filterlim_at_top) | |
| 2757 | then show "\<forall>\<^sub>F i in F. dist (x ^ f i) 0 < e" | |
| 68615 | 2758 | by eventually_elim (auto simp: N) | 
| 63556 | 2759 | qed | 
| 2760 | ||
| 69593 | 2761 | text \<open>Limit of \<^term>\<open>c^n\<close> for \<^term>\<open>\<bar>c\<bar> < 1\<close>.\<close> | 
| 51526 | 2762 | |
| 68614 | 2763 | lemma LIMSEQ_abs_realpow_zero: "\<bar>c\<bar> < 1 \<Longrightarrow> (\<lambda>n. \<bar>c\<bar> ^ n :: real) \<longlonglongrightarrow> 0" | 
| 51526 | 2764 | by (rule LIMSEQ_realpow_zero [OF abs_ge_zero]) | 
| 2765 | ||
| 68614 | 2766 | lemma LIMSEQ_abs_realpow_zero2: "\<bar>c\<bar> < 1 \<Longrightarrow> (\<lambda>n. c ^ n :: real) \<longlonglongrightarrow> 0" | 
| 51526 | 2767 | by (rule LIMSEQ_power_zero) simp | 
| 2768 | ||
| 2769 | ||
| 60758 | 2770 | subsection \<open>Limits of Functions\<close> | 
| 51526 | 2771 | |
| 63546 | 2772 | lemma LIM_eq: "f \<midarrow>a\<rightarrow> L = (\<forall>r>0. \<exists>s>0. \<forall>x. x \<noteq> a \<and> norm (x - a) < s \<longrightarrow> norm (f x - L) < r)" | 
| 2773 | for a :: "'a::real_normed_vector" and L :: "'b::real_normed_vector" | |
| 2774 | by (simp add: LIM_def dist_norm) | |
| 51526 | 2775 | |
| 2776 | lemma LIM_I: | |
| 63546 | 2777 | "(\<And>r. 0 < r \<Longrightarrow> \<exists>s>0. \<forall>x. x \<noteq> a \<and> norm (x - a) < s \<longrightarrow> norm (f x - L) < r) \<Longrightarrow> f \<midarrow>a\<rightarrow> L" | 
| 2778 | for a :: "'a::real_normed_vector" and L :: "'b::real_normed_vector" | |
| 2779 | by (simp add: LIM_eq) | |
| 2780 | ||
| 2781 | lemma LIM_D: "f \<midarrow>a\<rightarrow> L \<Longrightarrow> 0 < r \<Longrightarrow> \<exists>s>0.\<forall>x. x \<noteq> a \<and> norm (x - a) < s \<longrightarrow> norm (f x - L) < r" | |
| 2782 | for a :: "'a::real_normed_vector" and L :: "'b::real_normed_vector" | |
| 2783 | by (simp add: LIM_eq) | |
| 2784 | ||
| 2785 | lemma LIM_offset: "f \<midarrow>a\<rightarrow> L \<Longrightarrow> (\<lambda>x. f (x + k)) \<midarrow>(a - k)\<rightarrow> L" | |
| 2786 | for a :: "'a::real_normed_vector" | |
| 2787 | by (simp add: filtermap_at_shift[symmetric, of a k] filterlim_def filtermap_filtermap) | |
| 2788 | ||
| 2789 | lemma LIM_offset_zero: "f \<midarrow>a\<rightarrow> L \<Longrightarrow> (\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> L" | |
| 2790 | for a :: "'a::real_normed_vector" | |
| 2791 | by (drule LIM_offset [where k = a]) (simp add: add.commute) | |
| 2792 | ||
| 2793 | lemma LIM_offset_zero_cancel: "(\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> L \<Longrightarrow> f \<midarrow>a\<rightarrow> L" | |
| 2794 | for a :: "'a::real_normed_vector" | |
| 2795 | by (drule LIM_offset [where k = "- a"]) simp | |
| 2796 | ||
| 72245 | 2797 | lemma LIM_offset_zero_iff: "NO_MATCH 0 a \<Longrightarrow> f \<midarrow>a\<rightarrow> L \<longleftrightarrow> (\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> L" | 
| 63546 | 2798 | for f :: "'a :: real_normed_vector \<Rightarrow> _" | 
| 51642 
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
 hoelzl parents: 
51641diff
changeset | 2799 | using LIM_offset_zero_cancel[of f a L] LIM_offset_zero[of f L a] by auto | 
| 
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
 hoelzl parents: 
51641diff
changeset | 2800 | |
| 70999 
5b753486c075
Inverse function theorem + lemmas
 paulson <lp15@cam.ac.uk> parents: 
70817diff
changeset | 2801 | lemma tendsto_offset_zero_iff: | 
| 
5b753486c075
Inverse function theorem + lemmas
 paulson <lp15@cam.ac.uk> parents: 
70817diff
changeset | 2802 | fixes f :: "'a :: real_normed_vector \<Rightarrow> _" | 
| 72245 | 2803 | assumes " NO_MATCH 0 a" "a \<in> S" "open S" | 
| 70999 
5b753486c075
Inverse function theorem + lemmas
 paulson <lp15@cam.ac.uk> parents: 
70817diff
changeset | 2804 | shows "(f \<longlongrightarrow> L) (at a within S) \<longleftrightarrow> ((\<lambda>h. f (a + h)) \<longlongrightarrow> L) (at 0)" | 
| 72245 | 2805 | using assms by (simp add: tendsto_within_open_NO_MATCH LIM_offset_zero_iff) | 
| 70999 
5b753486c075
Inverse function theorem + lemmas
 paulson <lp15@cam.ac.uk> parents: 
70817diff
changeset | 2806 | |
| 63546 | 2807 | lemma LIM_zero: "(f \<longlongrightarrow> l) F \<Longrightarrow> ((\<lambda>x. f x - l) \<longlongrightarrow> 0) F" | 
| 65578 
e4997c181cce
New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
 paulson <lp15@cam.ac.uk> parents: 
65204diff
changeset | 2808 | for f :: "'a \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 2809 | unfolding tendsto_iff dist_norm by simp | 
| 51526 | 2810 | |
| 2811 | lemma LIM_zero_cancel: | |
| 65578 
e4997c181cce
New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
 paulson <lp15@cam.ac.uk> parents: 
65204diff
changeset | 2812 | fixes f :: "'a \<Rightarrow> 'b::real_normed_vector" | 
| 61973 | 2813 | shows "((\<lambda>x. f x - l) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> l) F" | 
| 51526 | 2814 | unfolding tendsto_iff dist_norm by simp | 
| 2815 | ||
| 63546 | 2816 | lemma LIM_zero_iff: "((\<lambda>x. f x - l) \<longlongrightarrow> 0) F = (f \<longlongrightarrow> l) F" | 
| 65578 
e4997c181cce
New material from PNT proof, as well as more default [simp] declarations. Also removed duplicate theorems about geometric series
 paulson <lp15@cam.ac.uk> parents: 
65204diff
changeset | 2817 | for f :: "'a \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 2818 | unfolding tendsto_iff dist_norm by simp | 
| 51526 | 2819 | |
| 2820 | lemma LIM_imp_LIM: | |
| 2821 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_vector" | |
| 2822 | fixes g :: "'a::topological_space \<Rightarrow> 'c::real_normed_vector" | |
| 61976 | 2823 | assumes f: "f \<midarrow>a\<rightarrow> l" | 
| 63546 | 2824 | and le: "\<And>x. x \<noteq> a \<Longrightarrow> norm (g x - m) \<le> norm (f x - l)" | 
| 61976 | 2825 | shows "g \<midarrow>a\<rightarrow> m" | 
| 63546 | 2826 | by (rule metric_LIM_imp_LIM [OF f]) (simp add: dist_norm le) | 
| 51526 | 2827 | |
| 2828 | lemma LIM_equal2: | |
| 2829 | fixes f g :: "'a::real_normed_vector \<Rightarrow> 'b::topological_space" | |
| 63546 | 2830 | assumes "0 < R" | 
| 2831 | and "\<And>x. x \<noteq> a \<Longrightarrow> norm (x - a) < R \<Longrightarrow> f x = g x" | |
| 61976 | 2832 | shows "g \<midarrow>a\<rightarrow> l \<Longrightarrow> f \<midarrow>a\<rightarrow> l" | 
| 68594 | 2833 | by (rule metric_LIM_equal2 [OF _ assms]) (simp_all add: dist_norm) | 
| 51526 | 2834 | |
| 2835 | lemma LIM_compose2: | |
| 2836 | fixes a :: "'a::real_normed_vector" | |
| 61976 | 2837 | assumes f: "f \<midarrow>a\<rightarrow> b" | 
| 63546 | 2838 | and g: "g \<midarrow>b\<rightarrow> c" | 
| 2839 | and inj: "\<exists>d>0. \<forall>x. x \<noteq> a \<and> norm (x - a) < d \<longrightarrow> f x \<noteq> b" | |
| 61976 | 2840 | shows "(\<lambda>x. g (f x)) \<midarrow>a\<rightarrow> c" | 
| 63546 | 2841 | by (rule metric_LIM_compose2 [OF f g inj [folded dist_norm]]) | 
| 51526 | 2842 | |
| 2843 | lemma real_LIM_sandwich_zero: | |
| 2844 | fixes f g :: "'a::topological_space \<Rightarrow> real" | |
| 61976 | 2845 | assumes f: "f \<midarrow>a\<rightarrow> 0" | 
| 63546 | 2846 | and 1: "\<And>x. x \<noteq> a \<Longrightarrow> 0 \<le> g x" | 
| 2847 | and 2: "\<And>x. x \<noteq> a \<Longrightarrow> g x \<le> f x" | |
| 61976 | 2848 | shows "g \<midarrow>a\<rightarrow> 0" | 
| 51526 | 2849 | proof (rule LIM_imp_LIM [OF f]) (* FIXME: use tendsto_sandwich *) | 
| 63546 | 2850 | fix x | 
| 2851 | assume x: "x \<noteq> a" | |
| 2852 | with 1 have "norm (g x - 0) = g x" by simp | |
| 51526 | 2853 | also have "g x \<le> f x" by (rule 2 [OF x]) | 
| 2854 | also have "f x \<le> \<bar>f x\<bar>" by (rule abs_ge_self) | |
| 2855 | also have "\<bar>f x\<bar> = norm (f x - 0)" by simp | |
| 2856 | finally show "norm (g x - 0) \<le> norm (f x - 0)" . | |
| 2857 | qed | |
| 2858 | ||
| 2859 | ||
| 60758 | 2860 | subsection \<open>Continuity\<close> | 
| 51526 | 2861 | |
| 63546 | 2862 | lemma LIM_isCont_iff: "(f \<midarrow>a\<rightarrow> f a) = ((\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> f a)" | 
| 2863 | for f :: "'a::real_normed_vector \<Rightarrow> 'b::topological_space" | |
| 2864 | by (rule iffI [OF LIM_offset_zero LIM_offset_zero_cancel]) | |
| 2865 | ||
| 2866 | lemma isCont_iff: "isCont f x = (\<lambda>h. f (x + h)) \<midarrow>0\<rightarrow> f x" | |
| 2867 | for f :: "'a::real_normed_vector \<Rightarrow> 'b::topological_space" | |
| 2868 | by (simp add: isCont_def LIM_isCont_iff) | |
| 51526 | 2869 | |
| 2870 | lemma isCont_LIM_compose2: | |
| 2871 | fixes a :: "'a::real_normed_vector" | |
| 2872 | assumes f [unfolded isCont_def]: "isCont f a" | |
| 63546 | 2873 | and g: "g \<midarrow>f a\<rightarrow> l" | 
| 2874 | and inj: "\<exists>d>0. \<forall>x. x \<noteq> a \<and> norm (x - a) < d \<longrightarrow> f x \<noteq> f a" | |
| 61976 | 2875 | shows "(\<lambda>x. g (f x)) \<midarrow>a\<rightarrow> l" | 
| 63546 | 2876 | by (rule LIM_compose2 [OF f g inj]) | 
| 2877 | ||
| 2878 | lemma isCont_norm [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. norm (f x)) a" | |
| 2879 | for f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | |
| 51526 | 2880 | by (fact continuous_norm) | 
| 2881 | ||
| 63546 | 2882 | lemma isCont_rabs [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. \<bar>f x\<bar>) a" | 
| 2883 | for f :: "'a::t2_space \<Rightarrow> real" | |
| 51526 | 2884 | by (fact continuous_rabs) | 
| 2885 | ||
| 63546 | 2886 | lemma isCont_add [simp]: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x + g x) a" | 
| 2887 | for f :: "'a::t2_space \<Rightarrow> 'b::topological_monoid_add" | |
| 51526 | 2888 | by (fact continuous_add) | 
| 2889 | ||
| 63546 | 2890 | lemma isCont_minus [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. - f x) a" | 
| 2891 | for f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | |
| 51526 | 2892 | by (fact continuous_minus) | 
| 2893 | ||
| 63546 | 2894 | lemma isCont_diff [simp]: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x - g x) a" | 
| 2895 | for f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | |
| 51526 | 2896 | by (fact continuous_diff) | 
| 2897 | ||
| 63546 | 2898 | lemma isCont_mult [simp]: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x * g x) a" | 
| 2899 | for f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_algebra" | |
| 51526 | 2900 | by (fact continuous_mult) | 
| 2901 | ||
| 63546 | 2902 | lemma (in bounded_linear) isCont: "isCont g a \<Longrightarrow> isCont (\<lambda>x. f (g x)) a" | 
| 51526 | 2903 | by (fact continuous) | 
| 2904 | ||
| 63546 | 2905 | lemma (in bounded_bilinear) isCont: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x ** g x) a" | 
| 51526 | 2906 | by (fact continuous) | 
| 2907 | ||
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2908 | lemmas isCont_scaleR [simp] = | 
| 51526 | 2909 | bounded_bilinear.isCont [OF bounded_bilinear_scaleR] | 
| 2910 | ||
| 2911 | lemmas isCont_of_real [simp] = | |
| 2912 | bounded_linear.isCont [OF bounded_linear_of_real] | |
| 2913 | ||
| 63546 | 2914 | lemma isCont_power [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. f x ^ n) a" | 
| 2915 |   for f :: "'a::t2_space \<Rightarrow> 'b::{power,real_normed_algebra}"
 | |
| 51526 | 2916 | by (fact continuous_power) | 
| 2917 | ||
| 64267 | 2918 | lemma isCont_sum [simp]: "\<forall>i\<in>A. isCont (f i) a \<Longrightarrow> isCont (\<lambda>x. \<Sum>i\<in>A. f i x) a" | 
| 63546 | 2919 | for f :: "'a \<Rightarrow> 'b::t2_space \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 64267 | 2920 | by (auto intro: continuous_sum) | 
| 51526 | 2921 | |
| 63546 | 2922 | |
| 60758 | 2923 | subsection \<open>Uniform Continuity\<close> | 
| 51526 | 2924 | |
| 63104 | 2925 | lemma uniformly_continuous_on_def: | 
| 2926 | fixes f :: "'a::metric_space \<Rightarrow> 'b::metric_space" | |
| 2927 | shows "uniformly_continuous_on s f \<longleftrightarrow> | |
| 2928 | (\<forall>e>0. \<exists>d>0. \<forall>x\<in>s. \<forall>x'\<in>s. dist x' x < d \<longrightarrow> dist (f x') (f x) < e)" | |
| 2929 | unfolding uniformly_continuous_on_uniformity | |
| 2930 | uniformity_dist filterlim_INF filterlim_principal eventually_inf_principal | |
| 2931 | by (force simp: Ball_def uniformity_dist[symmetric] eventually_uniformity_metric) | |
| 2932 | ||
| 63546 | 2933 | abbreviation isUCont :: "['a::metric_space \<Rightarrow> 'b::metric_space] \<Rightarrow> bool" | 
| 2934 | where "isUCont f \<equiv> uniformly_continuous_on UNIV f" | |
| 2935 | ||
| 2936 | lemma isUCont_def: "isUCont f \<longleftrightarrow> (\<forall>r>0. \<exists>s>0. \<forall>x y. dist x y < s \<longrightarrow> dist (f x) (f y) < r)" | |
| 63104 | 2937 | by (auto simp: uniformly_continuous_on_def dist_commute) | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 2938 | |
| 63546 | 2939 | lemma isUCont_isCont: "isUCont f \<Longrightarrow> isCont f x" | 
| 63104 | 2940 | by (drule uniformly_continuous_imp_continuous) (simp add: continuous_on_eq_continuous_at) | 
| 2941 | ||
| 2942 | lemma uniformly_continuous_on_Cauchy: | |
| 63546 | 2943 | fixes f :: "'a::metric_space \<Rightarrow> 'b::metric_space" | 
| 63104 | 2944 | assumes "uniformly_continuous_on S f" "Cauchy X" "\<And>n. X n \<in> S" | 
| 2945 | shows "Cauchy (\<lambda>n. f (X n))" | |
| 2946 | using assms | |
| 68594 | 2947 | unfolding uniformly_continuous_on_def by (meson Cauchy_def) | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 2948 | |
| 63546 | 2949 | lemma isUCont_Cauchy: "isUCont f \<Longrightarrow> Cauchy X \<Longrightarrow> Cauchy (\<lambda>n. f (X n))" | 
| 63104 | 2950 | by (rule uniformly_continuous_on_Cauchy[where S=UNIV and f=f]) simp_all | 
| 68611 | 2951 | |
| 51526 | 2952 | lemma (in bounded_linear) isUCont: "isUCont f" | 
| 63546 | 2953 | unfolding isUCont_def dist_norm | 
| 51526 | 2954 | proof (intro allI impI) | 
| 63546 | 2955 | fix r :: real | 
| 2956 | assume r: "0 < r" | |
| 2957 | obtain K where K: "0 < K" and norm_le: "norm (f x) \<le> norm x * K" for x | |
| 61649 
268d88ec9087
Tweaks for "real": Removal of [iff] status for some lemmas, adding [simp] for others. Plus fixes.
 paulson <lp15@cam.ac.uk> parents: 
61609diff
changeset | 2958 | using pos_bounded by blast | 
| 51526 | 2959 | show "\<exists>s>0. \<forall>x y. norm (x - y) < s \<longrightarrow> norm (f x - f y) < r" | 
| 2960 | proof (rule exI, safe) | |
| 56541 | 2961 | from r K show "0 < r / K" by simp | 
| 51526 | 2962 | next | 
| 2963 | fix x y :: 'a | |
| 2964 | assume xy: "norm (x - y) < r / K" | |
| 2965 | have "norm (f x - f y) = norm (f (x - y))" by (simp only: diff) | |
| 2966 | also have "\<dots> \<le> norm (x - y) * K" by (rule norm_le) | |
| 2967 | also from K xy have "\<dots> < r" by (simp only: pos_less_divide_eq) | |
| 2968 | finally show "norm (f x - f y) < r" . | |
| 2969 | qed | |
| 2970 | qed | |
| 2971 | ||
| 2972 | lemma (in bounded_linear) Cauchy: "Cauchy X \<Longrightarrow> Cauchy (\<lambda>n. f (X n))" | |
| 63546 | 2973 | by (rule isUCont [THEN isUCont_Cauchy]) | 
| 51526 | 2974 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2975 | lemma LIM_less_bound: | 
| 51526 | 2976 | fixes f :: "real \<Rightarrow> real" | 
| 2977 |   assumes ev: "b < x" "\<forall> x' \<in> { b <..< x}. 0 \<le> f x'" and "isCont f x"
 | |
| 2978 | shows "0 \<le> f x" | |
| 63952 
354808e9f44b
new material connected with HOL Light measure theory, plus more rationalisation
 paulson <lp15@cam.ac.uk> parents: 
63915diff
changeset | 2979 | proof (rule tendsto_lowerbound) | 
| 61973 | 2980 | show "(f \<longlongrightarrow> f x) (at_left x)" | 
| 60758 | 2981 | using \<open>isCont f x\<close> by (simp add: filterlim_at_split isCont_def) | 
| 51526 | 2982 | show "eventually (\<lambda>x. 0 \<le> f x) (at_left x)" | 
| 51641 
cd05e9fcc63d
remove the within-filter, replace "at" by "at _ within UNIV" (This allows to remove a couple of redundant lemmas)
 hoelzl parents: 
51531diff
changeset | 2983 | using ev by (auto simp: eventually_at dist_real_def intro!: exI[of _ "x - b"]) | 
| 51526 | 2984 | qed simp | 
| 51471 | 2985 | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 2986 | |
| 60758 | 2987 | subsection \<open>Nested Intervals and Bisection -- Needed for Compactness\<close> | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 2988 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 2989 | lemma nested_sequence_unique: | 
| 61969 | 2990 | assumes "\<forall>n. f n \<le> f (Suc n)" "\<forall>n. g (Suc n) \<le> g n" "\<forall>n. f n \<le> g n" "(\<lambda>n. f n - g n) \<longlonglongrightarrow> 0" | 
| 2991 | shows "\<exists>l::real. ((\<forall>n. f n \<le> l) \<and> f \<longlonglongrightarrow> l) \<and> ((\<forall>n. l \<le> g n) \<and> g \<longlonglongrightarrow> l)" | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 2992 | proof - | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 2993 | have "incseq f" unfolding incseq_Suc_iff by fact | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 2994 | have "decseq g" unfolding decseq_Suc_iff by fact | 
| 63546 | 2995 | have "f n \<le> g 0" for n | 
| 2996 | proof - | |
| 2997 | from \<open>decseq g\<close> have "g n \<le> g 0" | |
| 2998 | by (rule decseqD) simp | |
| 2999 | with \<open>\<forall>n. f n \<le> g n\<close>[THEN spec, of n] show ?thesis | |
| 3000 | by auto | |
| 3001 | qed | |
| 61969 | 3002 | then obtain u where "f \<longlonglongrightarrow> u" "\<forall>i. f i \<le> u" | 
| 60758 | 3003 | using incseq_convergent[OF \<open>incseq f\<close>] by auto | 
| 63546 | 3004 | moreover have "f 0 \<le> g n" for n | 
| 3005 | proof - | |
| 60758 | 3006 | from \<open>incseq f\<close> have "f 0 \<le> f n" by (rule incseqD) simp | 
| 63546 | 3007 | with \<open>\<forall>n. f n \<le> g n\<close>[THEN spec, of n] show ?thesis | 
| 3008 | by simp | |
| 3009 | qed | |
| 61969 | 3010 | then obtain l where "g \<longlonglongrightarrow> l" "\<forall>i. l \<le> g i" | 
| 60758 | 3011 | using decseq_convergent[OF \<open>decseq g\<close>] by auto | 
| 61969 | 3012 | moreover note LIMSEQ_unique[OF assms(4) tendsto_diff[OF \<open>f \<longlonglongrightarrow> u\<close> \<open>g \<longlonglongrightarrow> l\<close>]] | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3013 | ultimately show ?thesis by auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3014 | qed | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3015 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3016 | lemma Bolzano[consumes 1, case_names trans local]: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3017 | fixes P :: "real \<Rightarrow> real \<Rightarrow> bool" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3018 | assumes [arith]: "a \<le> b" | 
| 63546 | 3019 | and trans: "\<And>a b c. P a b \<Longrightarrow> P b c \<Longrightarrow> a \<le> b \<Longrightarrow> b \<le> c \<Longrightarrow> P a c" | 
| 3020 | and local: "\<And>x. a \<le> x \<Longrightarrow> x \<le> b \<Longrightarrow> \<exists>d>0. \<forall>a b. a \<le> x \<and> x \<le> b \<and> b - a < d \<longrightarrow> P a b" | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3021 | shows "P a b" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3022 | proof - | 
| 74513 
67d87d224e00
A few new lemmas plus some refinements
 paulson <lp15@cam.ac.uk> parents: 
74475diff
changeset | 3023 | define bisect where "bisect \<equiv> \<lambda>(x,y). if P x ((x+y) / 2) then ((x+y)/2, y) else (x, (x+y)/2)" | 
| 
67d87d224e00
A few new lemmas plus some refinements
 paulson <lp15@cam.ac.uk> parents: 
74475diff
changeset | 3024 | define l u where "l n \<equiv> fst ((bisect^^n)(a,b))" and "u n \<equiv> snd ((bisect^^n)(a,b))" for n | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3025 | have l[simp]: "l 0 = a" "\<And>n. l (Suc n) = (if P (l n) ((l n + u n) / 2) then (l n + u n) / 2 else l n)" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3026 | and u[simp]: "u 0 = b" "\<And>n. u (Suc n) = (if P (l n) ((l n + u n) / 2) then u n else (l n + u n) / 2)" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3027 | by (simp_all add: l_def u_def bisect_def split: prod.split) | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3028 | |
| 63546 | 3029 | have [simp]: "l n \<le> u n" for n by (induct n) auto | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3030 | |
| 61969 | 3031 | have "\<exists>x. ((\<forall>n. l n \<le> x) \<and> l \<longlonglongrightarrow> x) \<and> ((\<forall>n. x \<le> u n) \<and> u \<longlonglongrightarrow> x)" | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3032 | proof (safe intro!: nested_sequence_unique) | 
| 63546 | 3033 | show "l n \<le> l (Suc n)" "u (Suc n) \<le> u n" for n | 
| 3034 | by (induct n) auto | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3035 | next | 
| 63546 | 3036 | have "l n - u n = (a - b) / 2^n" for n | 
| 3037 | by (induct n) (auto simp: field_simps) | |
| 3038 | then show "(\<lambda>n. l n - u n) \<longlonglongrightarrow> 0" | |
| 3039 | by (simp add: LIMSEQ_divide_realpow_zero) | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3040 | qed fact | 
| 63546 | 3041 | then obtain x where x: "\<And>n. l n \<le> x" "\<And>n. x \<le> u n" and "l \<longlonglongrightarrow> x" "u \<longlonglongrightarrow> x" | 
| 3042 | by auto | |
| 3043 | obtain d where "0 < d" and d: "a \<le> x \<Longrightarrow> x \<le> b \<Longrightarrow> b - a < d \<Longrightarrow> P a b" for a b | |
| 60758 | 3044 | using \<open>l 0 \<le> x\<close> \<open>x \<le> u 0\<close> local[of x] by auto | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3045 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3046 | show "P a b" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3047 | proof (rule ccontr) | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 3048 | assume "\<not> P a b" | 
| 63546 | 3049 | have "\<not> P (l n) (u n)" for n | 
| 3050 | proof (induct n) | |
| 3051 | case 0 | |
| 3052 | then show ?case | |
| 3053 | by (simp add: \<open>\<not> P a b\<close>) | |
| 3054 | next | |
| 3055 | case (Suc n) | |
| 3056 | with trans[of "l n" "(l n + u n) / 2" "u n"] show ?case | |
| 3057 | by auto | |
| 3058 | qed | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3059 | moreover | 
| 63546 | 3060 |     {
 | 
| 3061 | have "eventually (\<lambda>n. x - d / 2 < l n) sequentially" | |
| 61969 | 3062 | using \<open>0 < d\<close> \<open>l \<longlonglongrightarrow> x\<close> by (intro order_tendstoD[of _ x]) auto | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3063 | moreover have "eventually (\<lambda>n. u n < x + d / 2) sequentially" | 
| 61969 | 3064 | using \<open>0 < d\<close> \<open>u \<longlonglongrightarrow> x\<close> by (intro order_tendstoD[of _ x]) auto | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3065 | ultimately have "eventually (\<lambda>n. P (l n) (u n)) sequentially" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3066 | proof eventually_elim | 
| 63546 | 3067 | case (elim n) | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3068 | from add_strict_mono[OF this] have "u n - l n < d" by simp | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3069 | with x show "P (l n) (u n)" by (rule d) | 
| 63546 | 3070 | qed | 
| 3071 | } | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3072 | ultimately show False by simp | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3073 | qed | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3074 | qed | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3075 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3076 | lemma compact_Icc[simp, intro]: "compact {a .. b::real}"
 | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3077 | proof (cases "a \<le> b", rule compactI) | 
| 63546 | 3078 | fix C | 
| 3079 |   assume C: "a \<le> b" "\<forall>t\<in>C. open t" "{a..b} \<subseteq> \<Union>C"
 | |
| 63040 | 3080 |   define T where "T = {a .. b}"
 | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3081 |   from C(1,3) show "\<exists>C'\<subseteq>C. finite C' \<and> {a..b} \<subseteq> \<Union>C'"
 | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3082 | proof (induct rule: Bolzano) | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3083 | case (trans a b c) | 
| 63546 | 3084 |     then have *: "{a..c} = {a..b} \<union> {b..c}"
 | 
| 3085 | by auto | |
| 3086 | with trans obtain C1 C2 | |
| 3087 |       where "C1\<subseteq>C" "finite C1" "{a..b} \<subseteq> \<Union>C1" "C2\<subseteq>C" "finite C2" "{b..c} \<subseteq> \<Union>C2"
 | |
| 3088 | by auto | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3089 | with trans show ?case | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3090 | unfolding * by (intro exI[of _ "C1 \<union> C2"]) auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3091 | next | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3092 | case (local x) | 
| 63546 | 3093 | with C have "x \<in> \<Union>C" by auto | 
| 3094 | with C(2) obtain c where "x \<in> c" "open c" "c \<in> C" | |
| 3095 | by auto | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3096 |     then obtain e where "0 < e" "{x - e <..< x + e} \<subseteq> c"
 | 
| 62101 | 3097 | by (auto simp: open_dist dist_real_def subset_eq Ball_def abs_less_iff) | 
| 60758 | 3098 | with \<open>c \<in> C\<close> show ?case | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3099 |       by (safe intro!: exI[of _ "e/2"] exI[of _ "{c}"]) auto
 | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3100 | qed | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3101 | qed simp | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3102 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3103 | |
| 57447 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3104 | lemma continuous_image_closed_interval: | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3105 | fixes a b and f :: "real \<Rightarrow> real" | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3106 |   defines "S \<equiv> {a..b}"
 | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3107 | assumes "a \<le> b" and f: "continuous_on S f" | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3108 |   shows "\<exists>c d. f`S = {c..d} \<and> c \<le> d"
 | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3109 | proof - | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3110 |   have S: "compact S" "S \<noteq> {}"
 | 
| 60758 | 3111 | using \<open>a \<le> b\<close> by (auto simp: S_def) | 
| 57447 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3112 | obtain c where "c \<in> S" "\<forall>d\<in>S. f d \<le> f c" | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3113 | using continuous_attains_sup[OF S f] by auto | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3114 | moreover obtain d where "d \<in> S" "\<forall>c\<in>S. f d \<le> f c" | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3115 | using continuous_attains_inf[OF S f] by auto | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3116 | moreover have "connected (f`S)" | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3117 | using connected_continuous_image[OF f] connected_Icc by (auto simp: S_def) | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3118 |   ultimately have "f ` S = {f d .. f c} \<and> f d \<le> f c"
 | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3119 | by (auto simp: connected_iff_interval) | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3120 | then show ?thesis | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3121 | by auto | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3122 | qed | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 3123 | |
| 60974 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 3124 | lemma open_Collect_positive: | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 3125 | fixes f :: "'a::topological_space \<Rightarrow> real" | 
| 63546 | 3126 | assumes f: "continuous_on s f" | 
| 3127 |   shows "\<exists>A. open A \<and> A \<inter> s = {x\<in>s. 0 < f x}"
 | |
| 3128 |   using continuous_on_open_invariant[THEN iffD1, OF f, rule_format, of "{0 <..}"]
 | |
| 3129 | by (auto simp: Int_def field_simps) | |
| 60974 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 3130 | |
| 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 3131 | lemma open_Collect_less_Int: | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 3132 | fixes f g :: "'a::topological_space \<Rightarrow> real" | 
| 63546 | 3133 | assumes f: "continuous_on s f" | 
| 3134 | and g: "continuous_on s g" | |
| 3135 |   shows "\<exists>A. open A \<and> A \<inter> s = {x\<in>s. f x < g x}"
 | |
| 3136 | using open_Collect_positive[OF continuous_on_diff[OF g f]] by (simp add: field_simps) | |
| 60974 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 3137 | |
| 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 3138 | |
| 60758 | 3139 | subsection \<open>Boundedness of continuous functions\<close> | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3140 | |
| 60758 | 3141 | text\<open>By bisection, function continuous on closed interval is bounded above\<close> | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3142 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3143 | lemma isCont_eq_Ub: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3144 | fixes f :: "real \<Rightarrow> 'a::linorder_topology" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3145 | shows "a \<le> b \<Longrightarrow> \<forall>x::real. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x \<Longrightarrow> | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3146 | \<exists>M. (\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> f x \<le> M) \<and> (\<exists>x. a \<le> x \<and> x \<le> b \<and> f x = M)" | 
| 63546 | 3147 |   using continuous_attains_sup[of "{a..b}" f]
 | 
| 68615 | 3148 | by (auto simp: continuous_at_imp_continuous_on Ball_def Bex_def) | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3149 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3150 | lemma isCont_eq_Lb: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3151 | fixes f :: "real \<Rightarrow> 'a::linorder_topology" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3152 | shows "a \<le> b \<Longrightarrow> \<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x \<Longrightarrow> | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3153 | \<exists>M. (\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> M \<le> f x) \<and> (\<exists>x. a \<le> x \<and> x \<le> b \<and> f x = M)" | 
| 63546 | 3154 |   using continuous_attains_inf[of "{a..b}" f]
 | 
| 68615 | 3155 | by (auto simp: continuous_at_imp_continuous_on Ball_def Bex_def) | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3156 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3157 | lemma isCont_bounded: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3158 | fixes f :: "real \<Rightarrow> 'a::linorder_topology" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3159 | shows "a \<le> b \<Longrightarrow> \<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x \<Longrightarrow> \<exists>M. \<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> f x \<le> M" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3160 | using isCont_eq_Ub[of a b f] by auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3161 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3162 | lemma isCont_has_Ub: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3163 | fixes f :: "real \<Rightarrow> 'a::linorder_topology" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3164 | shows "a \<le> b \<Longrightarrow> \<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x \<Longrightarrow> | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3165 | \<exists>M. (\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> f x \<le> M) \<and> (\<forall>N. N < M \<longrightarrow> (\<exists>x. a \<le> x \<and> x \<le> b \<and> N < f x))" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3166 | using isCont_eq_Ub[of a b f] by auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3167 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3168 | lemma isCont_Lb_Ub: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3169 | fixes f :: "real \<Rightarrow> real" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3170 | assumes "a \<le> b" "\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 3171 | shows "\<exists>L M. (\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> L \<le> f x \<and> f x \<le> M) \<and> | 
| 63546 | 3172 | (\<forall>y. L \<le> y \<and> y \<le> M \<longrightarrow> (\<exists>x. a \<le> x \<and> x \<le> b \<and> (f x = y)))" | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3173 | proof - | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3174 | obtain M where M: "a \<le> M" "M \<le> b" "\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> f x \<le> f M" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3175 | using isCont_eq_Ub[OF assms] by auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3176 | obtain L where L: "a \<le> L" "L \<le> b" "\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> f L \<le> f x" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3177 | using isCont_eq_Lb[OF assms] by auto | 
| 68615 | 3178 | have "(\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> f L \<le> f x \<and> f x \<le> f M)" | 
| 3179 | using M L by simp | |
| 3180 | moreover | |
| 3181 | have "(\<forall>y. f L \<le> y \<and> y \<le> f M \<longrightarrow> (\<exists>x\<ge>a. x \<le> b \<and> f x = y))" | |
| 3182 | proof (cases "L \<le> M") | |
| 3183 | case True then show ?thesis | |
| 3184 | using IVT[of f L _ M] M L assms by (metis order.trans) | |
| 3185 | next | |
| 3186 | case False then show ?thesis | |
| 3187 | using IVT2[of f L _ M] | |
| 3188 | by (metis L(2) M(1) assms(2) le_cases order.trans) | |
| 3189 | qed | |
| 3190 | ultimately show ?thesis | |
| 3191 | by blast | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3192 | qed | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3193 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3194 | |
| 63546 | 3195 | text \<open>Continuity of inverse function.\<close> | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3196 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3197 | lemma isCont_inverse_function: | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3198 | fixes f g :: "real \<Rightarrow> real" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3199 | assumes d: "0 < d" | 
| 68611 | 3200 | and inj: "\<And>z. \<bar>z-x\<bar> \<le> d \<Longrightarrow> g (f z) = z" | 
| 3201 | and cont: "\<And>z. \<bar>z-x\<bar> \<le> d \<Longrightarrow> isCont f z" | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3202 | shows "isCont g (f x)" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3203 | proof - | 
| 63546 | 3204 | let ?A = "f (x - d)" | 
| 3205 | let ?B = "f (x + d)" | |
| 3206 |   let ?D = "{x - d..x + d}"
 | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3207 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3208 | have f: "continuous_on ?D f" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3209 | using cont by (intro continuous_at_imp_continuous_on ballI) auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3210 | then have g: "continuous_on (f`?D) g" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3211 | using inj by (intro continuous_on_inv) auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3212 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3213 |   from d f have "{min ?A ?B <..< max ?A ?B} \<subseteq> f ` ?D"
 | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3214 | by (intro connected_contains_Ioo connected_continuous_image) (auto split: split_min split_max) | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3215 |   with g have "continuous_on {min ?A ?B <..< max ?A ?B} g"
 | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3216 | by (rule continuous_on_subset) | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3217 | moreover | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3218 | have "(?A < f x \<and> f x < ?B) \<or> (?B < f x \<and> f x < ?A)" | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3219 | using d inj by (intro continuous_inj_imp_mono[OF _ _ f] inj_on_imageI2[of g, OF inj_onI]) auto | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3220 |   then have "f x \<in> {min ?A ?B <..< max ?A ?B}"
 | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3221 | by auto | 
| 68615 | 3222 | ultimately show ?thesis | 
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3223 | by (simp add: continuous_on_eq_continuous_at) | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3224 | qed | 
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3225 | |
| 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3226 | lemma isCont_inverse_function2: | 
| 63546 | 3227 | fixes f g :: "real \<Rightarrow> real" | 
| 3228 | shows | |
| 68611 | 3229 | "\<lbrakk>a < x; x < b; | 
| 3230 | \<And>z. \<lbrakk>a \<le> z; z \<le> b\<rbrakk> \<Longrightarrow> g (f z) = z; | |
| 3231 | \<And>z. \<lbrakk>a \<le> z; z \<le> b\<rbrakk> \<Longrightarrow> isCont f z\<rbrakk> \<Longrightarrow> isCont g (f x)" | |
| 63546 | 3232 | apply (rule isCont_inverse_function [where f=f and d="min (x - a) (b - x)"]) | 
| 3233 | apply (simp_all add: abs_le_iff) | |
| 3234 | done | |
| 51529 
2d2f59e6055a
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
 hoelzl parents: 
51526diff
changeset | 3235 | |
| 63546 | 3236 | text \<open>Bartle/Sherbert: Introduction to Real Analysis, Theorem 4.2.9, p. 110.\<close> | 
| 3237 | lemma LIM_fun_gt_zero: "f \<midarrow>c\<rightarrow> l \<Longrightarrow> 0 < l \<Longrightarrow> \<exists>r. 0 < r \<and> (\<forall>x. x \<noteq> c \<and> \<bar>c - x\<bar> < r \<longrightarrow> 0 < f x)" | |
| 3238 | for f :: "real \<Rightarrow> real" | |
| 68615 | 3239 | by (force simp: dest: LIM_D) | 
| 63546 | 3240 | |
| 3241 | lemma LIM_fun_less_zero: "f \<midarrow>c\<rightarrow> l \<Longrightarrow> l < 0 \<Longrightarrow> \<exists>r. 0 < r \<and> (\<forall>x. x \<noteq> c \<and> \<bar>c - x\<bar> < r \<longrightarrow> f x < 0)" | |
| 3242 | for f :: "real \<Rightarrow> real" | |
| 68615 | 3243 | by (drule LIM_D [where r="-l"]) force+ | 
| 63546 | 3244 | |
| 3245 | lemma LIM_fun_not_zero: "f \<midarrow>c\<rightarrow> l \<Longrightarrow> l \<noteq> 0 \<Longrightarrow> \<exists>r. 0 < r \<and> (\<forall>x. x \<noteq> c \<and> \<bar>c - x\<bar> < r \<longrightarrow> f x \<noteq> 0)" | |
| 3246 | for f :: "real \<Rightarrow> real" | |
| 68615 | 3247 | using LIM_fun_gt_zero[of f l c] LIM_fun_less_zero[of f l c] by (auto simp: neq_iff) | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 3248 | |
| 77943 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3249 | lemma Lim_topological: | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3250 | "(f \<longlongrightarrow> l) net \<longleftrightarrow> | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3251 | trivial_limit net \<or> (\<forall>S. open S \<longrightarrow> l \<in> S \<longrightarrow> eventually (\<lambda>x. f x \<in> S) net)" | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3252 | unfolding tendsto_def trivial_limit_eq by auto | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3253 | |
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3254 | lemma eventually_within_Un: | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3255 | "eventually P (at x within (s \<union> t)) \<longleftrightarrow> | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3256 | eventually P (at x within s) \<and> eventually P (at x within t)" | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3257 | unfolding eventually_at_filter | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3258 | by (auto elim!: eventually_rev_mp) | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3259 | |
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3260 | lemma Lim_within_Un: | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3261 | "(f \<longlongrightarrow> l) (at x within (s \<union> t)) \<longleftrightarrow> | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3262 | (f \<longlongrightarrow> l) (at x within s) \<and> (f \<longlongrightarrow> l) (at x within t)" | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3263 | unfolding tendsto_def | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3264 | by (auto simp: eventually_within_Un) | 
| 
ffdad62bc235
Importation of additional lemmas from metric.ml
 paulson <lp15@cam.ac.uk> parents: 
77221diff
changeset | 3265 | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 3266 | end |