| author | paulson <lp15@cam.ac.uk> | 
| Wed, 04 Jul 2018 11:00:06 +0100 | |
| changeset 68586 | 006da53a8ac1 | 
| parent 68532 | f8b98d31ad45 | 
| child 68594 | 5b05ede597b8 | 
| 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 | |
| 60758 | 14 | subsection \<open>Filter going to infinity norm\<close> | 
| 51526 | 15 | |
| 63546 | 16 | definition at_infinity :: "'a::real_normed_vector filter" | 
| 17 |   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 | 18 | |
| 57276 | 19 | lemma eventually_at_infinity: "eventually P at_infinity \<longleftrightarrow> (\<exists>b. \<forall>x. b \<le> norm x \<longrightarrow> P x)" | 
| 20 | unfolding at_infinity_def | |
| 21 | by (subst eventually_INF_base) | |
| 22 | (auto simp: subset_eq eventually_principal intro!: exI[of _ "max a b" for a b]) | |
| 31392 | 23 | |
| 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 | 24 | corollary eventually_at_infinity_pos: | 
| 63546 | 25 | "eventually p at_infinity \<longleftrightarrow> (\<exists>b. 0 < b \<and> (\<forall>x. norm x \<ge> b \<longrightarrow> p x))" | 
| 26 | apply (simp add: eventually_at_infinity) | |
| 27 | apply auto | |
| 28 | apply (case_tac "b \<le> 0") | |
| 29 | using norm_ge_zero order_trans zero_less_one apply blast | |
| 30 | apply force | |
| 31 | done | |
| 32 | ||
| 33 | lemma at_infinity_eq_at_top_bot: "(at_infinity :: real filter) = sup at_top at_bot" | |
| 57276 | 34 | apply (simp add: filter_eq_iff eventually_sup eventually_at_infinity | 
| 63546 | 35 | eventually_at_top_linorder eventually_at_bot_linorder) | 
| 57276 | 36 | apply safe | 
| 63546 | 37 | apply (rule_tac x="b" in exI) | 
| 38 | apply simp | |
| 39 | apply (rule_tac x="- b" in exI) | |
| 40 | apply simp | |
| 41 | apply (rule_tac x="max (- Na) N" in exI) | |
| 42 | apply (auto simp: abs_real_def) | |
| 57276 | 43 | done | 
| 50325 | 44 | |
| 57276 | 45 | lemma at_top_le_at_infinity: "at_top \<le> (at_infinity :: real filter)" | 
| 50325 | 46 | unfolding at_infinity_eq_at_top_bot by simp | 
| 47 | ||
| 57276 | 48 | lemma at_bot_le_at_infinity: "at_bot \<le> (at_infinity :: real filter)" | 
| 50325 | 49 | unfolding at_infinity_eq_at_top_bot by simp | 
| 50 | ||
| 63546 | 51 | lemma filterlim_at_top_imp_at_infinity: "filterlim f at_top F \<Longrightarrow> filterlim f at_infinity F" | 
| 52 | 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 | 53 | 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 | 54 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 55 | 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 | 56 | 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 | 57 | |
| 63546 | 58 | lemma lim_infinity_imp_sequentially: "(f \<longlongrightarrow> l) at_infinity \<Longrightarrow> ((\<lambda>n. f(n)) \<longlongrightarrow> l) sequentially" | 
| 59 | 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 | 60 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 61 | |
| 60758 | 62 | subsubsection \<open>Boundedness\<close> | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 63 | |
| 63546 | 64 | definition Bfun :: "('a \<Rightarrow> 'b::metric_space) \<Rightarrow> 'a filter \<Rightarrow> bool"
 | 
| 65 | where Bfun_metric_def: "Bfun f F = (\<exists>y. \<exists>K>0. eventually (\<lambda>x. dist (f x) y \<le> K) F)" | |
| 66 | ||
| 67 | abbreviation Bseq :: "(nat \<Rightarrow> 'a::metric_space) \<Rightarrow> bool" | |
| 68 | 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 | 69 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 70 | 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 | 71 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 72 | 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 | 73 | 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 | 74 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 75 | 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 | 76 | unfolding Bfun_metric_def by (subst (asm) eventually_sequentially_seg) | 
| 31355 | 77 | |
| 63546 | 78 | 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 | 79 | 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 | 80 | proof safe | 
| 63546 | 81 | fix y K | 
| 82 | 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 | 83 | 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 | 84 | 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 | 85 | 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 | 86 | by eventually_elim auto | 
| 60758 | 87 | 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 | 88 | 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 | 89 | qed (force simp del: norm_conv_dist [symmetric]) | 
| 31355 | 90 | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 91 | lemma BfunI: | 
| 63546 | 92 | assumes K: "eventually (\<lambda>x. norm (f x) \<le> K) F" | 
| 93 | shows "Bfun f F" | |
| 94 | unfolding Bfun_def | |
| 31355 | 95 | proof (intro exI conjI allI) | 
| 96 | show "0 < max K 1" by simp | |
| 44195 | 97 | show "eventually (\<lambda>x. norm (f x) \<le> max K 1) F" | 
| 63546 | 98 | using K by (rule eventually_mono) simp | 
| 31355 | 99 | qed | 
| 100 | ||
| 101 | lemma BfunE: | |
| 44195 | 102 | assumes "Bfun f F" | 
| 103 | obtains B where "0 < B" and "eventually (\<lambda>x. norm (f x) \<le> B) F" | |
| 63546 | 104 | using assms unfolding Bfun_def by blast | 
| 31355 | 105 | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 106 | lemma Cauchy_Bseq: "Cauchy X \<Longrightarrow> Bseq X" | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 107 | unfolding Cauchy_def Bfun_metric_def eventually_sequentially | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 108 | apply (erule_tac x=1 in allE) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 109 | apply simp | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 110 | apply safe | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 111 | apply (rule_tac x="X M" in exI) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 112 | apply (rule_tac x=1 in exI) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 113 | apply (erule_tac x=M in allE) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 114 | apply simp | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 115 | apply (rule_tac x=M in exI) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 116 | apply (auto simp: dist_commute) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 117 | done | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 118 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 119 | |
| 60758 | 120 | subsubsection \<open>Bounded Sequences\<close> | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 121 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 122 | 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 | 123 | 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 | 124 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 125 | lemma BseqI2': "\<forall>n\<ge>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 | 126 | 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 | 127 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 128 | 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 | 129 | unfolding Bfun_def eventually_sequentially | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 130 | proof safe | 
| 63546 | 131 | fix N K | 
| 132 | 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 | 133 | 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 | 134 |     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 | 135 | (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 | 136 | qed auto | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 137 | |
| 63546 | 138 | lemma BseqE: "Bseq X \<Longrightarrow> (\<And>K. 0 < K \<Longrightarrow> \<forall>n. norm (X n) \<le> K \<Longrightarrow> Q) \<Longrightarrow> Q" | 
| 139 | unfolding Bseq_def by auto | |
| 140 | ||
| 141 | lemma BseqD: "Bseq X \<Longrightarrow> \<exists>K. 0 < K \<and> (\<forall>n. norm (X n) \<le> K)" | |
| 142 | by (simp add: Bseq_def) | |
| 143 | ||
| 144 | lemma BseqI: "0 < K \<Longrightarrow> \<forall>n. norm (X n) \<le> K \<Longrightarrow> Bseq X" | |
| 145 | by (auto simp add: Bseq_def) | |
| 146 | ||
| 147 | lemma Bseq_bdd_above: "Bseq X \<Longrightarrow> bdd_above (range X)" | |
| 148 | for X :: "nat \<Rightarrow> real" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 149 | proof (elim BseqE, intro bdd_aboveI2) | 
| 63546 | 150 | fix K n | 
| 151 | assume "0 < K" "\<forall>n. norm (X n) \<le> K" | |
| 152 | then show "X n \<le> K" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 153 | by (auto elim!: allE[of _ n]) | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 154 | qed | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 155 | |
| 63546 | 156 | lemma Bseq_bdd_above': "Bseq X \<Longrightarrow> bdd_above (range (\<lambda>n. norm (X n)))" | 
| 157 | for X :: "nat \<Rightarrow> 'a :: real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 158 | proof (elim BseqE, intro bdd_aboveI2) | 
| 63546 | 159 | fix K n | 
| 160 | assume "0 < K" "\<forall>n. norm (X n) \<le> K" | |
| 161 | then show "norm (X n) \<le> K" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 162 | by (auto elim!: allE[of _ n]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 163 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 164 | |
| 63546 | 165 | lemma Bseq_bdd_below: "Bseq X \<Longrightarrow> bdd_below (range X)" | 
| 166 | for X :: "nat \<Rightarrow> real" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 167 | proof (elim BseqE, intro bdd_belowI2) | 
| 63546 | 168 | fix K n | 
| 169 | assume "0 < K" "\<forall>n. norm (X n) \<le> K" | |
| 170 | then show "- K \<le> X n" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 171 | by (auto elim!: allE[of _ n]) | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 172 | qed | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 173 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 174 | lemma Bseq_eventually_mono: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 175 | assumes "eventually (\<lambda>n. norm (f n) \<le> norm (g n)) sequentially" "Bseq g" | 
| 63546 | 176 | shows "Bseq f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 177 | proof - | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 178 | 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 | 179 | unfolding Bfun_def by fast | 
| 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 180 | 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 | 181 | by (fast elim: eventually_elim2 order_trans) | 
| 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 182 | with `0 < K` show "Bseq f" | 
| 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 183 | unfolding Bfun_def by fast | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 184 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 185 | |
| 63546 | 186 | 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 | 187 | proof safe | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 188 | fix K :: real | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 189 | 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 | 190 | 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 | 191 | 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 | 192 | 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 | 193 | by (blast intro: order_trans) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 194 | 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 | 195 | 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 | 196 | 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 | 197 | 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 | 198 | qed | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 199 | |
| 63546 | 200 | text \<open>Alternative definition for \<open>Bseq\<close>.\<close> | 
| 201 | lemma Bseq_iff: "Bseq X \<longleftrightarrow> (\<exists>N. \<forall>n. norm (X n) \<le> real(Suc N))" | |
| 202 | by (simp add: Bseq_def) (simp add: lemma_NBseq_def) | |
| 203 | ||
| 204 | lemma lemma_NBseq_def2: "(\<exists>K > 0. \<forall>n. norm (X n) \<le> K) = (\<exists>N. \<forall>n. norm (X n) < real(Suc N))" | |
| 205 | apply (subst lemma_NBseq_def) | |
| 206 | apply auto | |
| 207 | apply (rule_tac x = "Suc N" in exI) | |
| 208 | apply (rule_tac [2] x = N in exI) | |
| 209 | apply auto | |
| 210 | prefer 2 apply (blast intro: order_less_imp_le) | |
| 211 | apply (drule_tac x = n in spec) | |
| 212 | apply simp | |
| 213 | done | |
| 214 | ||
| 215 | text \<open>Yet another definition for Bseq.\<close> | |
| 216 | lemma Bseq_iff1a: "Bseq X \<longleftrightarrow> (\<exists>N. \<forall>n. norm (X n) < real (Suc N))" | |
| 217 | by (simp add: Bseq_def lemma_NBseq_def2) | |
| 218 | ||
| 219 | subsubsection \<open>A Few More Equivalence Theorems for Boundedness\<close> | |
| 220 | ||
| 221 | text \<open>Alternative formulation for boundedness.\<close> | |
| 222 | lemma Bseq_iff2: "Bseq X \<longleftrightarrow> (\<exists>k > 0. \<exists>x. \<forall>n. norm (X n + - x) \<le> k)" | |
| 223 | apply (unfold Bseq_def) | |
| 224 | apply safe | |
| 225 | apply (rule_tac [2] x = "k + norm x" in exI) | |
| 226 | apply (rule_tac x = K in exI) | |
| 227 | apply simp | |
| 228 | apply (rule exI [where x = 0]) | |
| 229 | apply auto | |
| 230 | apply (erule order_less_le_trans) | |
| 231 | apply simp | |
| 232 | apply (drule_tac x=n in spec) | |
| 233 | apply (drule order_trans [OF norm_triangle_ineq2]) | |
| 234 | apply simp | |
| 235 | done | |
| 236 | ||
| 237 | text \<open>Alternative formulation for boundedness.\<close> | |
| 238 | lemma Bseq_iff3: "Bseq X \<longleftrightarrow> (\<exists>k>0. \<exists>N. \<forall>n. norm (X n + - X N) \<le> k)" | |
| 239 | (is "?P \<longleftrightarrow> ?Q") | |
| 53602 | 240 | proof | 
| 241 | assume ?P | |
| 63546 | 242 | then obtain K where *: "0 < K" and **: "\<And>n. norm (X n) \<le> K" | 
| 243 | by (auto simp add: Bseq_def) | |
| 53602 | 244 | 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 | 245 | 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 | 246 | by (auto intro: order_trans norm_triangle_ineq4) | 
| 
b1d955791529
more simplification rules on unary and binary minus
 haftmann parents: 
53602diff
changeset | 247 | 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 | 248 | by simp | 
| 60758 | 249 | with \<open>0 < K + norm (X 0)\<close> show ?Q by blast | 
| 53602 | 250 | next | 
| 63546 | 251 | assume ?Q | 
| 252 | then show ?P by (auto simp add: Bseq_iff2) | |
| 53602 | 253 | qed | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 254 | |
| 63546 | 255 | lemma BseqI2: "\<forall>n. k \<le> f n \<and> f n \<le> K \<Longrightarrow> Bseq f" | 
| 256 | for k K :: real | |
| 257 | apply (simp add: Bseq_def) | |
| 258 | apply (rule_tac x = "(\<bar>k\<bar> + \<bar>K\<bar>) + 1" in exI) | |
| 259 | apply auto | |
| 260 | apply (drule_tac x = n in spec) | |
| 261 | apply arith | |
| 262 | done | |
| 263 | ||
| 264 | ||
| 265 | subsubsection \<open>Upper Bounds and Lubs of Bounded Sequences\<close> | |
| 266 | ||
| 267 | 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 | 268 | by (simp add: Bseq_def) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 269 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 270 | lemma Bseq_add: | 
| 63546 | 271 | fixes f :: "nat \<Rightarrow> 'a::real_normed_vector" | 
| 272 | assumes "Bseq f" | |
| 273 | shows "Bseq (\<lambda>x. f x + c)" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 274 | proof - | 
| 63546 | 275 | from assms obtain K where K: "\<And>x. norm (f x) \<le> K" | 
| 276 | unfolding Bseq_def by blast | |
| 61531 
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 | fix x :: nat | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 279 | 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 | 280 | also have "norm (f x) \<le> K" by (rule K) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 281 | finally have "norm (f x + c) \<le> K + norm c" by simp | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 282 | } | 
| 63546 | 283 | then show ?thesis by (rule BseqI') | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 284 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 285 | |
| 63546 | 286 | lemma Bseq_add_iff: "Bseq (\<lambda>x. f x + c) \<longleftrightarrow> Bseq f" | 
| 287 | for f :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 288 | 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 | 289 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 290 | lemma Bseq_mult: | 
| 63546 | 291 | fixes f g :: "nat \<Rightarrow> 'a::real_normed_field" | 
| 292 | assumes "Bseq f" and "Bseq g" | |
| 293 | shows "Bseq (\<lambda>x. f x * g x)" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 294 | proof - | 
| 63546 | 295 | from assms obtain K1 K2 where K: "norm (f x) \<le> K1" "K1 > 0" "norm (g x) \<le> K2" "K2 > 0" | 
| 296 | for x | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 297 | unfolding Bseq_def by blast | 
| 63546 | 298 | then have "norm (f x * g x) \<le> K1 * K2" for x | 
| 299 | by (auto simp: norm_mult intro!: mult_mono) | |
| 300 | then show ?thesis by (rule BseqI') | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 301 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 302 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 303 | lemma Bfun_const [simp]: "Bfun (\<lambda>_. c) F" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 304 | 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 | 305 | |
| 63546 | 306 | lemma Bseq_cmult_iff: | 
| 307 | fixes c :: "'a::real_normed_field" | |
| 308 | assumes "c \<noteq> 0" | |
| 309 | shows "Bseq (\<lambda>x. c * f x) \<longleftrightarrow> Bseq f" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 310 | proof | 
| 63546 | 311 | assume "Bseq (\<lambda>x. c * f x)" | 
| 312 | with Bfun_const have "Bseq (\<lambda>x. inverse c * (c * f x))" | |
| 313 | by (rule Bseq_mult) | |
| 314 | with \<open>c \<noteq> 0\<close> show "Bseq f" | |
| 315 | by (simp add: divide_simps) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 316 | qed (intro Bseq_mult Bfun_const) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 317 | |
| 63546 | 318 | lemma Bseq_subseq: "Bseq f \<Longrightarrow> Bseq (\<lambda>x. f (g x))" | 
| 319 | for f :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 320 | unfolding Bseq_def by auto | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 321 | |
| 63546 | 322 | lemma Bseq_Suc_iff: "Bseq (\<lambda>n. f (Suc n)) \<longleftrightarrow> Bseq f" | 
| 323 | for f :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 324 | using Bseq_offset[of f 1] by (auto intro: Bseq_subseq) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 325 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 326 | lemma increasing_Bseq_subseq_iff: | 
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 327 | assumes "\<And>x y. x \<le> y \<Longrightarrow> norm (f x :: 'a::real_normed_vector) \<le> norm (f y)" "strict_mono g" | 
| 63546 | 328 | shows "Bseq (\<lambda>x. f (g x)) \<longleftrightarrow> Bseq f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 329 | proof | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 330 | assume "Bseq (\<lambda>x. f (g x))" | 
| 63546 | 331 | then obtain K where K: "\<And>x. norm (f (g x)) \<le> K" | 
| 332 | unfolding Bseq_def by auto | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 333 |   {
 | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 334 | fix x :: nat | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 335 | 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 | 336 | by (auto simp: filterlim_at_top eventually_at_top_linorder) | 
| 63546 | 337 | then have "norm (f x) \<le> norm (f (g y))" | 
| 338 | using assms(1) by blast | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 339 | also have "norm (f (g y)) \<le> K" by (rule K) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 340 | finally have "norm (f x) \<le> K" . | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 341 | } | 
| 63546 | 342 | then show "Bseq f" by (rule BseqI') | 
| 343 | qed (use Bseq_subseq[of f g] in simp_all) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 344 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 345 | lemma nonneg_incseq_Bseq_subseq_iff: | 
| 63546 | 346 | fixes f :: "nat \<Rightarrow> real" | 
| 347 | and g :: "nat \<Rightarrow> nat" | |
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 348 | assumes "\<And>x. f x \<ge> 0" "incseq f" "strict_mono g" | 
| 63546 | 349 | shows "Bseq (\<lambda>x. f (g x)) \<longleftrightarrow> Bseq f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 350 | using assms by (intro increasing_Bseq_subseq_iff) (auto simp: incseq_def) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 351 | |
| 63546 | 352 | lemma Bseq_eq_bounded: "range f \<subseteq> {a..b} \<Longrightarrow> Bseq f"
 | 
| 353 | for a b :: real | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 354 | apply (simp add: subset_eq) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 355 | apply (rule BseqI'[where K="max (norm a) (norm b)"]) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 356 | apply (erule_tac x=n in allE) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 357 | apply auto | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 358 | done | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 359 | |
| 63546 | 360 | lemma incseq_bounded: "incseq X \<Longrightarrow> \<forall>i. X i \<le> B \<Longrightarrow> Bseq X" | 
| 361 | for B :: real | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 362 | 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 | 363 | |
| 63546 | 364 | lemma decseq_bounded: "decseq X \<Longrightarrow> \<forall>i. B \<le> X i \<Longrightarrow> Bseq X" | 
| 365 | for B :: real | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 366 | 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 | 367 | |
| 63546 | 368 | |
| 60758 | 369 | subsection \<open>Bounded Monotonic Sequences\<close> | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 370 | |
| 63546 | 371 | subsubsection \<open>A Bounded and Monotonic Sequence Converges\<close> | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 372 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 373 | (* TODO: delete *) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 374 | (* FIXME: one use in NSA/HSEQ.thy *) | 
| 63546 | 375 | lemma Bmonoseq_LIMSEQ: "\<forall>n. m \<le> n \<longrightarrow> X n = X m \<Longrightarrow> \<exists>L. X \<longlonglongrightarrow> L" | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 376 | apply (rule_tac x="X m" in exI) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 377 | apply (rule filterlim_cong[THEN iffD2, OF refl refl _ tendsto_const]) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 378 | unfolding eventually_sequentially | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 379 | apply blast | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 380 | done | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 381 | |
| 63546 | 382 | |
| 60758 | 383 | 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 | 384 | |
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 385 | definition Zfun :: "('a \<Rightarrow> 'b::real_normed_vector) \<Rightarrow> 'a filter \<Rightarrow> bool"
 | 
| 44195 | 386 | 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 | 387 | |
| 63546 | 388 | lemma ZfunI: "(\<And>r. 0 < r \<Longrightarrow> eventually (\<lambda>x. norm (f x) < r) F) \<Longrightarrow> Zfun f F" | 
| 389 | by (simp add: Zfun_def) | |
| 390 | ||
| 391 | lemma ZfunD: "Zfun f F \<Longrightarrow> 0 < r \<Longrightarrow> eventually (\<lambda>x. norm (f x) < r) F" | |
| 392 | by (simp add: Zfun_def) | |
| 393 | ||
| 394 | 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 | 395 | unfolding Zfun_def by (auto elim!: eventually_rev_mp) | 
| 31355 | 396 | |
| 44195 | 397 | 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 | 398 | unfolding Zfun_def by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 399 | |
| 44195 | 400 | 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 | 401 | unfolding Zfun_def by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 402 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 403 | lemma Zfun_imp_Zfun: | 
| 44195 | 404 | assumes f: "Zfun f F" | 
| 63546 | 405 | and g: "eventually (\<lambda>x. norm (g x) \<le> norm (f x) * K) F" | 
| 44195 | 406 | shows "Zfun (\<lambda>x. g x) F" | 
| 63546 | 407 | proof (cases "0 < K") | 
| 408 | case K: True | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 409 | show ?thesis | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 410 | proof (rule ZfunI) | 
| 63546 | 411 | fix r :: real | 
| 412 | assume "0 < r" | |
| 413 | then have "0 < r / K" using K by simp | |
| 44195 | 414 | 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 | 415 | using ZfunD [OF f] by blast | 
| 44195 | 416 | with g show "eventually (\<lambda>x. norm (g x) < r) F" | 
| 46887 | 417 | proof eventually_elim | 
| 418 | case (elim x) | |
| 63546 | 419 | 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 | 420 | by (simp add: pos_less_divide_eq K) | 
| 63546 | 421 | then show ?case | 
| 46887 | 422 | 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 | 423 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 424 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 425 | next | 
| 63546 | 426 | case False | 
| 427 | then have K: "K \<le> 0" by (simp only: not_less) | |
| 31355 | 428 | show ?thesis | 
| 429 | proof (rule ZfunI) | |
| 430 | fix r :: real | |
| 431 | assume "0 < r" | |
| 44195 | 432 | from g show "eventually (\<lambda>x. norm (g x) < r) F" | 
| 46887 | 433 | proof eventually_elim | 
| 434 | case (elim x) | |
| 435 | also have "norm (f x) * K \<le> norm (f x) * 0" | |
| 31355 | 436 | using K norm_ge_zero by (rule mult_left_mono) | 
| 46887 | 437 | finally show ?case | 
| 60758 | 438 | using \<open>0 < r\<close> by simp | 
| 31355 | 439 | qed | 
| 440 | qed | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 441 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 442 | |
| 63546 | 443 | lemma Zfun_le: "Zfun g F \<Longrightarrow> \<forall>x. norm (f x) \<le> norm (g x) \<Longrightarrow> Zfun f F" | 
| 444 | 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 | 445 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 446 | lemma Zfun_add: | 
| 63546 | 447 | assumes f: "Zfun f F" | 
| 448 | and g: "Zfun g F" | |
| 44195 | 449 | 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 | 450 | proof (rule ZfunI) | 
| 63546 | 451 | fix r :: real | 
| 452 | assume "0 < r" | |
| 453 | then have r: "0 < r / 2" by simp | |
| 44195 | 454 | 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 | 455 | 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 | 456 | moreover | 
| 44195 | 457 | 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 | 458 | 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 | 459 | ultimately | 
| 44195 | 460 | show "eventually (\<lambda>x. norm (f x + g x) < r) F" | 
| 46887 | 461 | proof eventually_elim | 
| 462 | case (elim x) | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 463 | 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 | 464 | by (rule norm_triangle_ineq) | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 465 | also have "\<dots> < r/2 + r/2" | 
| 46887 | 466 | using elim by (rule add_strict_mono) | 
| 467 | finally show ?case | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 468 | by simp | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 469 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 470 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 471 | |
| 44195 | 472 | 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 | 473 | unfolding Zfun_def by simp | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 474 | |
| 63546 | 475 | 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 | 476 | 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 | 477 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 478 | lemma (in bounded_linear) Zfun: | 
| 44195 | 479 | assumes g: "Zfun g F" | 
| 480 | 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 | 481 | proof - | 
| 63546 | 482 | 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 | 483 | using bounded by blast | 
| 44195 | 484 | then have "eventually (\<lambda>x. norm (f (g x)) \<le> norm (g x) * K) F" | 
| 31355 | 485 | by simp | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 486 | with g show ?thesis | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 487 | by (rule Zfun_imp_Zfun) | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 488 | qed | 
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 489 | |
| 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 490 | lemma (in bounded_bilinear) Zfun: | 
| 44195 | 491 | assumes f: "Zfun f F" | 
| 63546 | 492 | and g: "Zfun g F" | 
| 44195 | 493 | 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 | 494 | proof (rule ZfunI) | 
| 63546 | 495 | fix r :: real | 
| 496 | assume r: "0 < r" | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 497 | obtain K where K: "0 < K" | 
| 63546 | 498 | 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 | 499 | using pos_bounded by blast | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 500 | 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 | 501 | by (rule positive_imp_inverse_positive) | 
| 44195 | 502 | have "eventually (\<lambda>x. norm (f x) < r) F" | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 503 | 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 | 504 | moreover | 
| 44195 | 505 | 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 | 506 | 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 | 507 | ultimately | 
| 44195 | 508 | show "eventually (\<lambda>x. norm (f x ** g x) < r) F" | 
| 46887 | 509 | proof eventually_elim | 
| 510 | case (elim x) | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 511 | 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 | 512 | by (rule norm_le) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 513 | also have "norm (f x) * norm (g x) * K < r * inverse K * K" | 
| 46887 | 514 | 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 | 515 | 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 | 516 | by simp | 
| 46887 | 517 | finally show ?case . | 
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 518 | qed | 
| 
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 | |
| 63546 | 521 | 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 | 522 | 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 | 523 | |
| 63546 | 524 | 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 | 525 | 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 | 526 | |
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 527 | 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 | 528 | 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 | 529 | 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 | 530 | |
| 61973 | 531 | 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 | 532 | 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 | 533 | |
| 63546 | 534 | lemma tendsto_0_le: | 
| 535 | "(f \<longlongrightarrow> 0) F \<Longrightarrow> eventually (\<lambda>x. norm (g x) \<le> norm (f x) * K) F \<Longrightarrow> (g \<longlongrightarrow> 0) F" | |
| 56366 | 536 | by (simp add: Zfun_imp_Zfun tendsto_Zfun_iff) | 
| 537 | ||
| 63546 | 538 | |
| 60758 | 539 | subsubsection \<open>Distance and norms\<close> | 
| 36662 
621122eeb138
generalize types of LIMSEQ and LIM; generalize many lemmas
 huffman parents: 
36656diff
changeset | 540 | |
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 541 | lemma tendsto_dist [tendsto_intros]: | 
| 63546 | 542 | fixes l m :: "'a::metric_space" | 
| 543 | assumes f: "(f \<longlongrightarrow> l) F" | |
| 544 | and g: "(g \<longlongrightarrow> m) F" | |
| 61973 | 545 | 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 | 546 | proof (rule tendstoI) | 
| 63546 | 547 | fix e :: real | 
| 548 | assume "0 < e" | |
| 549 | 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 | 550 | 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 | 551 | 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 | 552 | proof (eventually_elim) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 553 | case (elim x) | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 554 | 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 | 555 | unfolding dist_real_def | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 556 | using dist_triangle2 [of "f x" "g x" "l"] | 
| 63546 | 557 | and dist_triangle2 [of "g x" "l" "m"] | 
| 558 | and dist_triangle3 [of "l" "m" "f x"] | |
| 559 | 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 | 560 | by arith | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 561 | qed | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 562 | qed | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 563 | |
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 564 | lemma continuous_dist[continuous_intros]: | 
| 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 565 | 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 | 566 | 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 | 567 | 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 | 568 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 569 | 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 | 570 | 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 | 571 | 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 | 572 | 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 | 573 | |
| 63546 | 574 | 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 | 575 | unfolding norm_conv_dist by (intro tendsto_intros) | 
| 36662 
621122eeb138
generalize types of LIMSEQ and LIM; generalize many lemmas
 huffman parents: 
36656diff
changeset | 576 | |
| 63546 | 577 | 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 | 578 | 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 | 579 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 580 | 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 | 581 | "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 | 582 | 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 | 583 | |
| 63546 | 584 | lemma tendsto_norm_zero: "(f \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. norm (f x)) \<longlongrightarrow> 0) F" | 
| 585 | by (drule tendsto_norm) simp | |
| 586 | ||
| 587 | 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 | 588 | unfolding tendsto_iff dist_norm by simp | 
| 36662 
621122eeb138
generalize types of LIMSEQ and LIM; generalize many lemmas
 huffman parents: 
36656diff
changeset | 589 | |
| 63546 | 590 | 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 | 591 | 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 | 592 | |
| 63546 | 593 | lemma tendsto_rabs [tendsto_intros]: "(f \<longlongrightarrow> l) F \<Longrightarrow> ((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> \<bar>l\<bar>) F" | 
| 594 | for l :: real | |
| 595 | by (fold real_norm_def) (rule tendsto_norm) | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 596 | |
| 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 | 597 | 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 | 598 | "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 | 599 | 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 | 600 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 601 | 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 | 602 | "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 | 603 | 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 | 604 | |
| 63546 | 605 | lemma tendsto_rabs_zero: "(f \<longlongrightarrow> (0::real)) F \<Longrightarrow> ((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> 0) F" | 
| 606 | by (fold real_norm_def) (rule tendsto_norm_zero) | |
| 607 | ||
| 608 | lemma tendsto_rabs_zero_cancel: "((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> (0::real)) F \<Longrightarrow> (f \<longlongrightarrow> 0) F" | |
| 609 | by (fold real_norm_def) (rule tendsto_norm_zero_cancel) | |
| 610 | ||
| 611 | lemma tendsto_rabs_zero_iff: "((\<lambda>x. \<bar>f x\<bar>) \<longlongrightarrow> (0::real)) F \<longleftrightarrow> (f \<longlongrightarrow> 0) F" | |
| 612 | by (fold real_norm_def) (rule tendsto_norm_zero_iff) | |
| 613 | ||
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 614 | |
| 62368 | 615 | subsection \<open>Topological Monoid\<close> | 
| 616 | ||
| 617 | class topological_monoid_add = topological_space + monoid_add + | |
| 618 | assumes tendsto_add_Pair: "LIM x (nhds a \<times>\<^sub>F nhds b). fst x + snd x :> nhds (a + b)" | |
| 619 | ||
| 620 | 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 | 621 | |
| 31565 | 622 | lemma tendsto_add [tendsto_intros]: | 
| 62368 | 623 | fixes a b :: "'a::topological_monoid_add" | 
| 624 | shows "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. f x + g x) \<longlongrightarrow> a + b) F" | |
| 625 | using filterlim_compose[OF tendsto_add_Pair, of "\<lambda>x. (f x, g x)" a b F] | |
| 626 | 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 | 627 | |
| 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 | 628 | lemma continuous_add [continuous_intros]: | 
| 62368 | 629 | 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 | 630 | 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 | 631 | 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 | 632 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 633 | lemma continuous_on_add [continuous_intros]: | 
| 62368 | 634 | 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 | 635 | 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 | 636 | 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 | 637 | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 638 | lemma tendsto_add_zero: | 
| 62368 | 639 | fixes f g :: "_ \<Rightarrow> 'b::topological_monoid_add" | 
| 63546 | 640 | shows "(f \<longlongrightarrow> 0) F \<Longrightarrow> (g \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. f x + g x) \<longlongrightarrow> 0) F" | 
| 641 | by (drule (1) tendsto_add) simp | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 642 | |
| 64267 | 643 | lemma tendsto_sum [tendsto_intros]: | 
| 62368 | 644 | fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 63915 | 645 | 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" | 
| 646 | by (induct I rule: infinite_finite_induct) (simp_all add: tendsto_add) | |
| 62368 | 647 | |
| 67673 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 648 | lemma tendsto_null_sum: | 
| 
c8caefb20564
lots of new material, ultimately related to measure theory
 paulson <lp15@cam.ac.uk> parents: 
67399diff
changeset | 649 | 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 | 650 | 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 | 651 | 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 | 652 | 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 | 653 | |
| 64267 | 654 | lemma continuous_sum [continuous_intros]: | 
| 62368 | 655 | fixes f :: "'a \<Rightarrow> 'b::t2_space \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 63301 | 656 | shows "(\<And>i. i \<in> I \<Longrightarrow> continuous F (f i)) \<Longrightarrow> continuous F (\<lambda>x. \<Sum>i\<in>I. f i x)" | 
| 64267 | 657 | unfolding continuous_def by (rule tendsto_sum) | 
| 658 | ||
| 659 | lemma continuous_on_sum [continuous_intros]: | |
| 62368 | 660 | fixes f :: "'a \<Rightarrow> 'b::topological_space \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 63301 | 661 | 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 | 662 | unfolding continuous_on_def by (auto intro: tendsto_sum) | 
| 62368 | 663 | |
| 62369 | 664 | instance nat :: topological_comm_monoid_add | 
| 63546 | 665 | by standard | 
| 666 | (simp add: nhds_discrete principal_prod_principal filterlim_principal eventually_principal) | |
| 62369 | 667 | |
| 668 | instance int :: topological_comm_monoid_add | |
| 63546 | 669 | by standard | 
| 670 | (simp add: nhds_discrete principal_prod_principal filterlim_principal eventually_principal) | |
| 671 | ||
| 62369 | 672 | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 673 | subsubsection \<open>Topological group\<close> | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 674 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 675 | 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 | 676 | 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 | 677 | begin | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 678 | |
| 63546 | 679 | 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 | 680 | by (rule filterlim_compose[OF tendsto_uminus_nhds]) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 681 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 682 | end | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 683 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 684 | 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 | 685 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 686 | 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 | 687 | |
| 63546 | 688 | lemma continuous_minus [continuous_intros]: "continuous F f \<Longrightarrow> continuous F (\<lambda>x. - f x)" | 
| 689 | 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 | 690 | unfolding continuous_def by (rule tendsto_minus) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 691 | |
| 63546 | 692 | lemma continuous_on_minus [continuous_intros]: "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. - f x)" | 
| 693 | for f :: "_ \<Rightarrow> 'b::topological_group_add" | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 694 | unfolding continuous_on_def by (auto intro: tendsto_minus) | 
| 62368 | 695 | |
| 63546 | 696 | lemma tendsto_minus_cancel: "((\<lambda>x. - f x) \<longlongrightarrow> - a) F \<Longrightarrow> (f \<longlongrightarrow> a) F" | 
| 697 | for a :: "'a::topological_group_add" | |
| 698 | by (drule tendsto_minus) simp | |
| 63081 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 699 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 700 | lemma tendsto_minus_cancel_left: | 
| 63546 | 701 | "(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 | 702 | 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 | 703 | by auto | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 704 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 705 | lemma tendsto_diff [tendsto_intros]: | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 706 | fixes a b :: "'a::topological_group_add" | 
| 63546 | 707 | 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 | 708 | 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 | 709 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 710 | lemma continuous_diff [continuous_intros]: | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 711 | 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 | 712 | 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 | 713 | unfolding continuous_def by (rule tendsto_diff) | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 714 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 715 | lemma continuous_on_diff [continuous_intros]: | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 716 | fixes f g :: "_ \<Rightarrow> 'b::topological_group_add" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 717 | 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 | 718 | 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 | 719 | |
| 67399 | 720 | 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 | 721 | by (rule continuous_intros | simp)+ | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 722 | |
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 723 | instance real_normed_vector < topological_ab_group_add | 
| 62368 | 724 | proof | 
| 63546 | 725 | fix a b :: 'a | 
| 726 | show "((\<lambda>x. fst x + snd x) \<longlongrightarrow> a + b) (nhds a \<times>\<^sub>F nhds b)" | |
| 62368 | 727 | unfolding tendsto_Zfun_iff add_diff_add | 
| 728 | using tendsto_fst[OF filterlim_ident, of "(a,b)"] tendsto_snd[OF filterlim_ident, of "(a,b)"] | |
| 729 | by (intro Zfun_add) | |
| 730 | (auto simp add: 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 | 731 | show "(uminus \<longlongrightarrow> - a) (nhds a)" | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 732 | unfolding tendsto_Zfun_iff minus_diff_minus | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 733 | using filterlim_ident[of "nhds a"] | 
| 
5a5beb3dbe7e
introduced class topological_group between topological_monoid and real_normed_vector
 immler parents: 
63040diff
changeset | 734 | by (intro Zfun_minus) (simp add: tendsto_Zfun_iff) | 
| 62368 | 735 | qed | 
| 736 | ||
| 65204 
d23eded35a33
modernized construction of type bcontfun; base explicit theorems on Uniform_Limit.thy; added some lemmas
 immler parents: 
65036diff
changeset | 737 | lemmas real_tendsto_sandwich = tendsto_sandwich[where 'a=real] | 
| 50999 | 738 | |
| 63546 | 739 | |
| 60758 | 740 | subsubsection \<open>Linear operators and multiplication\<close> | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 741 | |
| 63546 | 742 | lemma linear_times: "linear (\<lambda>x. c * x)" | 
| 743 | 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 | 744 | 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 | 745 | |
| 63546 | 746 | 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 | 747 | 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 | 748 | |
| 63546 | 749 | 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 | 750 | 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 | 751 | |
| 63546 | 752 | 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 | 753 | 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 | 754 | |
| 63546 | 755 | lemma (in bounded_linear) tendsto_zero: "(g \<longlongrightarrow> 0) F \<Longrightarrow> ((\<lambda>x. f (g x)) \<longlongrightarrow> 0) F" | 
| 756 | by (drule tendsto) (simp only: zero) | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 757 | |
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 758 | lemma (in bounded_bilinear) tendsto: | 
| 63546 | 759 | "(f \<longlongrightarrow> a) F \<Longrightarrow> (g \<longlongrightarrow> b) F \<Longrightarrow> ((\<lambda>x. f x ** g x) \<longlongrightarrow> a ** b) F" | 
| 760 | 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 | 761 | |
| 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 | 762 | 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 | 763 | "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 | 764 | 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 | 765 | |
| 
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 | 766 | 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 | 767 | "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 | 768 | 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 | 769 | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 770 | lemma (in bounded_bilinear) tendsto_zero: | 
| 61973 | 771 | assumes f: "(f \<longlongrightarrow> 0) F" | 
| 63546 | 772 | and g: "(g \<longlongrightarrow> 0) F" | 
| 61973 | 773 | shows "((\<lambda>x. f x ** g x) \<longlongrightarrow> 0) F" | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 774 | using tendsto [OF f g] by (simp add: zero_left) | 
| 31355 | 775 | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 776 | lemma (in bounded_bilinear) tendsto_left_zero: | 
| 61973 | 777 | "(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 | 778 | by (rule bounded_linear.tendsto_zero [OF bounded_linear_left]) | 
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 779 | |
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 780 | lemma (in bounded_bilinear) tendsto_right_zero: | 
| 61973 | 781 | "(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 | 782 | by (rule bounded_linear.tendsto_zero [OF bounded_linear_right]) | 
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 783 | |
| 44282 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 784 | lemmas tendsto_of_real [tendsto_intros] = | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 785 | 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 | 786 | |
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 787 | lemmas tendsto_scaleR [tendsto_intros] = | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 788 | bounded_bilinear.tendsto [OF bounded_bilinear_scaleR] | 
| 
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
 huffman parents: 
44253diff
changeset | 789 | |
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 790 | |
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 791 | 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 | 792 | 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 | 793 | 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 | 794 | |
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 795 | instance real_normed_algebra < topological_semigroup_mult | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 796 | proof | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 797 | fix a b :: 'a | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 798 | 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 | 799 | unfolding nhds_prod[symmetric] | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 800 | 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 | 801 | 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 | 802 | qed | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 803 | |
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 804 | lemma tendsto_mult [tendsto_intros]: | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 805 | fixes a b :: "'a::topological_semigroup_mult" | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 806 | 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 | 807 | 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 | 808 | by (simp add: nhds_prod[symmetric] tendsto_Pair) | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 809 | |
| 63546 | 810 | 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 | 811 | for c :: "'a::topological_semigroup_mult" | 
| 63546 | 812 | by (rule tendsto_mult [OF tendsto_const]) | 
| 813 | ||
| 814 | 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 | 815 | for c :: "'a::topological_semigroup_mult" | 
| 63546 | 816 | 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 | 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 | 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 | 819 | 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 | 820 | |
| 
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 | 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 | 822 | 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 | 823 | |
| 
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 | 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 | 825 | 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 | 826 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 827 | 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 | 828 | 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 | 829 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 830 | 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 | 831 | 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 | 832 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 833 | 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 | 834 | 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 | 835 | |
| 44568 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 836 | lemmas tendsto_mult_zero = | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 837 | 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 | 838 | |
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 839 | lemmas tendsto_mult_left_zero = | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 840 | 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 | 841 | |
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 842 | lemmas tendsto_mult_right_zero = | 
| 
e6f291cb5810
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
 huffman parents: 
44342diff
changeset | 843 | 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 | 844 | |
| 68296 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 845 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 846 | lemma continuous_mult_left: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 847 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 848 | 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 | 849 | by (rule continuous_mult [OF continuous_const]) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 850 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 851 | lemma continuous_mult_right: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 852 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 853 | 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 | 854 | by (rule continuous_mult [OF _ continuous_const]) | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 855 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 856 | lemma continuous_on_mult_left: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 857 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 858 | 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 | 859 | 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 | 860 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 861 | lemma continuous_on_mult_right: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 862 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 863 | 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 | 864 | 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 | 865 | |
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 866 | lemma continuous_on_mult_const [simp]: | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 867 | fixes c::"'a::real_normed_algebra" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 868 | shows "continuous_on s (( * ) c)" | 
| 
69d680e94961
tidying and reorganisation around Cauchy Integral Theorem
 paulson <lp15@cam.ac.uk> parents: 
68064diff
changeset | 869 | 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 | 870 | |
| 66793 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 871 | lemma tendsto_divide_zero: | 
| 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 872 | fixes c :: "'a::real_normed_field" | 
| 
deabce3ccf1f
new material about connectedness, etc.
 paulson <lp15@cam.ac.uk> parents: 
66456diff
changeset | 873 | 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 | 874 | 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 | 875 | |
| 63546 | 876 | lemma tendsto_power [tendsto_intros]: "(f \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f x ^ n) \<longlongrightarrow> a ^ n) F" | 
| 877 |   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 | 878 | by (induct n) (simp_all add: tendsto_mult) | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 879 | |
| 65680 
378a2f11bec9
Simplification of some proofs. Also key lemmas using !! rather than ! in premises
 paulson <lp15@cam.ac.uk> parents: 
65578diff
changeset | 880 | 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 | 881 |     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 | 882 | 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 | 883 | |
| 63546 | 884 | lemma continuous_power [continuous_intros]: "continuous F f \<Longrightarrow> continuous F (\<lambda>x. (f x)^n)" | 
| 885 |   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 | 886 | 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 | 887 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 888 | 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 | 889 |   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 | 890 | 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 | 891 | 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 | 892 | |
| 64272 | 893 | lemma tendsto_prod [tendsto_intros]: | 
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 894 |   fixes f :: "'a \<Rightarrow> 'b \<Rightarrow> 'c::{real_normed_algebra,comm_ring_1}"
 | 
| 63915 | 895 | 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" | 
| 896 | 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 | 897 | |
| 64272 | 898 | 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 | 899 |   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 | 900 | shows "(\<And>i. i \<in> S \<Longrightarrow> continuous F (f i)) \<Longrightarrow> continuous F (\<lambda>x. \<Prod>i\<in>S. f i x)" | 
| 64272 | 901 | unfolding continuous_def by (rule tendsto_prod) | 
| 902 | ||
| 903 | 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 | 904 |   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 | 905 | 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 | 906 | 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 | 907 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 908 | lemma tendsto_of_real_iff: | 
| 63546 | 909 | "((\<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 | 910 | unfolding tendsto_iff by simp | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 911 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 912 | lemma tendsto_add_const_iff: | 
| 63546 | 913 | "((\<lambda>x. c + f x :: 'a::real_normed_vector) \<longlongrightarrow> c + d) F \<longleftrightarrow> (f \<longlongrightarrow> d) F" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 914 | using tendsto_add[OF tendsto_const[of c], of f d] | 
| 63546 | 915 | 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 | 916 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 917 | |
| 60758 | 918 | subsubsection \<open>Inverse and division\<close> | 
| 31355 | 919 | |
| 920 | lemma (in bounded_bilinear) Zfun_prod_Bfun: | |
| 44195 | 921 | assumes f: "Zfun f F" | 
| 63546 | 922 | and g: "Bfun g F" | 
| 44195 | 923 | shows "Zfun (\<lambda>x. f x ** g x) F" | 
| 31355 | 924 | proof - | 
| 925 | obtain K where K: "0 \<le> K" | |
| 926 | 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 | 927 | using nonneg_bounded by blast | 
| 31355 | 928 | obtain B where B: "0 < B" | 
| 44195 | 929 | 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 | 930 | using g by (rule BfunE) | 
| 44195 | 931 | have "eventually (\<lambda>x. norm (f x ** g x) \<le> norm (f x) * (B * K)) F" | 
| 46887 | 932 | using norm_g proof eventually_elim | 
| 933 | case (elim x) | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 934 | have "norm (f x ** g x) \<le> norm (f x) * norm (g x) * K" | 
| 31355 | 935 | by (rule norm_le) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 936 | also have "\<dots> \<le> norm (f x) * B * K" | 
| 63546 | 937 | 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 | 938 | 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 | 939 | by (rule mult.assoc) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 940 | finally show "norm (f x ** g x) \<le> norm (f x) * (B * K)" . | 
| 31355 | 941 | qed | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 942 | with f show ?thesis | 
| 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 943 | by (rule Zfun_imp_Zfun) | 
| 31355 | 944 | qed | 
| 945 | ||
| 946 | lemma (in bounded_bilinear) Bfun_prod_Zfun: | |
| 44195 | 947 | assumes f: "Bfun f F" | 
| 63546 | 948 | and g: "Zfun g F" | 
| 44195 | 949 | 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 | 950 | using flip g f by (rule bounded_bilinear.Zfun_prod_Bfun) | 
| 31355 | 951 | |
| 952 | lemma Bfun_inverse_lemma: | |
| 953 | fixes x :: "'a::real_normed_div_algebra" | |
| 63546 | 954 | shows "r \<le> norm x \<Longrightarrow> 0 < r \<Longrightarrow> norm (inverse x) \<le> inverse r" | 
| 955 | apply (subst nonzero_norm_inverse) | |
| 956 | apply clarsimp | |
| 44081 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 957 | apply (erule (1) le_imp_inverse_le) | 
| 
730f7cced3a6
rename type 'a net to 'a filter, following standard mathematical terminology
 huffman parents: 
44079diff
changeset | 958 | done | 
| 31355 | 959 | |
| 960 | lemma Bfun_inverse: | |
| 961 | fixes a :: "'a::real_normed_div_algebra" | |
| 61973 | 962 | assumes f: "(f \<longlongrightarrow> a) F" | 
| 31355 | 963 | assumes a: "a \<noteq> 0" | 
| 44195 | 964 | shows "Bfun (\<lambda>x. inverse (f x)) F" | 
| 31355 | 965 | proof - | 
| 966 | from a have "0 < norm a" by simp | |
| 63546 | 967 | then have "\<exists>r>0. r < norm a" by (rule dense) | 
| 968 | then obtain r where r1: "0 < r" and r2: "r < norm a" | |
| 969 | by blast | |
| 44195 | 970 | 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 | 971 | using tendstoD [OF f r1] by blast | 
| 63546 | 972 | then have "eventually (\<lambda>x. norm (inverse (f x)) \<le> inverse (norm a - r)) F" | 
| 46887 | 973 | proof eventually_elim | 
| 974 | case (elim x) | |
| 63546 | 975 | then have 1: "norm (f x - a) < r" | 
| 31355 | 976 | by (simp add: dist_norm) | 
| 63546 | 977 | then have 2: "f x \<noteq> 0" using r2 by auto | 
| 978 | then have "norm (inverse (f x)) = inverse (norm (f x))" | |
| 31355 | 979 | by (rule nonzero_norm_inverse) | 
| 980 | also have "\<dots> \<le> inverse (norm a - r)" | |
| 981 | proof (rule le_imp_inverse_le) | |
| 63546 | 982 | show "0 < norm a - r" | 
| 983 | using r2 by simp | |
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 984 | have "norm a - norm (f x) \<le> norm (a - f x)" | 
| 31355 | 985 | by (rule norm_triangle_ineq2) | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 986 | also have "\<dots> = norm (f x - a)" | 
| 31355 | 987 | by (rule norm_minus_commute) | 
| 988 | also have "\<dots> < r" using 1 . | |
| 63546 | 989 | finally show "norm a - r \<le> norm (f x)" | 
| 990 | by simp | |
| 31355 | 991 | qed | 
| 31487 
93938cafc0e6
put syntax for tendsto in Limits.thy; rename variables
 huffman parents: 
31447diff
changeset | 992 | finally show "norm (inverse (f x)) \<le> inverse (norm a - r)" . | 
| 31355 | 993 | qed | 
| 63546 | 994 | then show ?thesis by (rule BfunI) | 
| 31355 | 995 | qed | 
| 996 | ||
| 31565 | 997 | lemma tendsto_inverse [tendsto_intros]: | 
| 31355 | 998 | fixes a :: "'a::real_normed_div_algebra" | 
| 61973 | 999 | assumes f: "(f \<longlongrightarrow> a) F" | 
| 63546 | 1000 | and a: "a \<noteq> 0" | 
| 61973 | 1001 | shows "((\<lambda>x. inverse (f x)) \<longlongrightarrow> inverse a) F" | 
| 31355 | 1002 | proof - | 
| 1003 | from a have "0 < norm a" by simp | |
| 44195 | 1004 | with f have "eventually (\<lambda>x. dist (f x) a < norm a) F" | 
| 31355 | 1005 | by (rule tendstoD) | 
| 44195 | 1006 | then have "eventually (\<lambda>x. f x \<noteq> 0) F" | 
| 61810 | 1007 | unfolding dist_norm by (auto elim!: eventually_mono) | 
| 44627 | 1008 | with a have "eventually (\<lambda>x. inverse (f x) - inverse a = | 
| 1009 | - (inverse (f x) * (f x - a) * inverse a)) F" | |
| 61810 | 1010 | by (auto elim!: eventually_mono simp: inverse_diff_inverse) | 
| 44627 | 1011 | moreover have "Zfun (\<lambda>x. - (inverse (f x) * (f x - a) * inverse a)) F" | 
| 1012 | by (intro Zfun_minus Zfun_mult_left | |
| 1013 | bounded_bilinear.Bfun_prod_Zfun [OF bounded_bilinear_mult] | |
| 1014 | Bfun_inverse [OF f a] f [unfolded tendsto_Zfun_iff]) | |
| 1015 | ultimately show ?thesis | |
| 1016 | unfolding tendsto_Zfun_iff by (rule Zfun_ssubst) | |
| 31355 | 1017 | qed | 
| 1018 | ||
| 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 | 1019 | 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 | 1020 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1021 | assumes "continuous F f" | 
| 1022 | 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 | 1023 | 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 | 1024 | 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 | 1025 | |
| 
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 | 1026 | 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 | 1027 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1028 | assumes "continuous (at a within s) f" | 
| 1029 | 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 | 1030 | 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 | 1031 | 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 | 1032 | |
| 66827 
c94531b5007d
Divided Topology_Euclidean_Space in two, creating new theory Connected. Also deleted some duplicate / variant theorems
 paulson <lp15@cam.ac.uk> parents: 
66793diff
changeset | 1033 | lemma continuous_at_inverse[continuous_intros, simp]: | 
| 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 | 1034 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1035 | assumes "isCont f a" | 
| 1036 | 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 | 1037 | shows "isCont (\<lambda>x. inverse (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 | 1038 | using assms unfolding continuous_at 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 | 1039 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 1040 | 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 | 1041 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_div_algebra" | 
| 63546 | 1042 | assumes "continuous_on s f" | 
| 1043 | 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 | 1044 | 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 | 1045 | 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 | 1046 | |
| 31565 | 1047 | lemma tendsto_divide [tendsto_intros]: | 
| 31355 | 1048 | fixes a b :: "'a::real_normed_field" | 
| 63546 | 1049 | 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 | 1050 | by (simp add: tendsto_mult tendsto_inverse divide_inverse) | 
| 31355 | 1051 | |
| 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 | 1052 | 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 | 1053 | fixes f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_field" | 
| 63546 | 1054 | assumes "continuous F f" | 
| 1055 | and "continuous F g" | |
| 1056 | 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 | 1057 | 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 | 1058 | 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 | 1059 | |
| 
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 | 1060 | 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 | 1061 | fixes f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_field" | 
| 63546 | 1062 | assumes "continuous (at a within s) f" "continuous (at a within s) g" | 
| 1063 | 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 | 1064 | 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 | 1065 | 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 | 1066 | |
| 
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 | 1067 | 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 | 1068 | 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 | 1069 | 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 | 1070 | 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 | 1071 | 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 | 1072 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 1073 | 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 | 1074 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_field" | 
| 63546 | 1075 | assumes "continuous_on s f" "continuous_on s g" | 
| 1076 | 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 | 1077 | 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 | 1078 | 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 | 1079 | |
| 63546 | 1080 | lemma tendsto_sgn [tendsto_intros]: "(f \<longlongrightarrow> l) F \<Longrightarrow> l \<noteq> 0 \<Longrightarrow> ((\<lambda>x. sgn (f x)) \<longlongrightarrow> sgn l) F" | 
| 1081 | for l :: "'a::real_normed_vector" | |
| 44194 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 1082 | unfolding sgn_div_norm by (simp add: tendsto_intros) | 
| 
0639898074ae
generalize lemmas about LIM and LIMSEQ to tendsto
 huffman parents: 
44081diff
changeset | 1083 | |
| 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 | 1084 | 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 | 1085 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1086 | assumes "continuous F f" | 
| 1087 | 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 | 1088 | 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 | 1089 | 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 | 1090 | |
| 
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 | 1091 | 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 | 1092 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1093 | assumes "continuous (at a within s) f" | 
| 1094 | 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 | 1095 | 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 | 1096 | 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 | 1097 | |
| 
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 | 1098 | 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 | 1099 | fixes f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1100 | assumes "isCont f a" | 
| 1101 | 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 | 1102 | 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 | 1103 | 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 | 1104 | |
| 56371 
fb9ae0727548
extend continuous_intros; remove continuous_on_intros and isCont_intros
 hoelzl parents: 
56366diff
changeset | 1105 | 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 | 1106 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 1107 | assumes "continuous_on s f" | 
| 1108 | 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 | 1109 | 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 | 1110 | 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 | 1111 | |
| 50325 | 1112 | lemma filterlim_at_infinity: | 
| 61076 | 1113 | fixes f :: "_ \<Rightarrow> 'a::real_normed_vector" | 
| 50325 | 1114 | assumes "0 \<le> c" | 
| 1115 | shows "(LIM x F. f x :> at_infinity) \<longleftrightarrow> (\<forall>r>c. eventually (\<lambda>x. r \<le> norm (f x)) F)" | |
| 1116 | unfolding filterlim_iff eventually_at_infinity | |
| 1117 | proof safe | |
| 63546 | 1118 | fix P :: "'a \<Rightarrow> bool" | 
| 1119 | fix b | |
| 50325 | 1120 | assume *: "\<forall>r>c. eventually (\<lambda>x. r \<le> norm (f x)) F" | 
| 63546 | 1121 | assume P: "\<forall>x. b \<le> norm x \<longrightarrow> P x" | 
| 50325 | 1122 | have "max b (c + 1) > c" by auto | 
| 1123 | with * have "eventually (\<lambda>x. max b (c + 1) \<le> norm (f x)) F" | |
| 1124 | by auto | |
| 1125 | then show "eventually (\<lambda>x. P (f x)) F" | |
| 1126 | proof eventually_elim | |
| 63546 | 1127 | case (elim x) | 
| 50325 | 1128 | with P show "P (f x)" by auto | 
| 1129 | qed | |
| 1130 | qed force | |
| 1131 | ||
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1132 | lemma filterlim_at_infinity_imp_norm_at_top: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1133 | fixes F | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1134 | assumes "filterlim f at_infinity F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1135 | 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 | 1136 | proof - | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1137 |   {
 | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1138 | fix r :: real | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1139 | have "\<forall>\<^sub>F x in F. r \<le> norm (f x)" using filterlim_at_infinity[of 0 f F] assms | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1140 | by (cases "r > 0") | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1141 | (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 | 1142 | } | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1143 | thus ?thesis by (auto simp: filterlim_at_top) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1144 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1145 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1146 | lemma filterlim_norm_at_top_imp_at_infinity: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1147 | fixes F | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1148 | 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 | 1149 | shows "filterlim f at_infinity F" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1150 | 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 | 1151 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1152 | 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 | 1153 | 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 | 1154 | |
| 67950 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1155 | lemma filterlim_at_infinity_conv_norm_at_top: | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1156 | "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 | 1157 | 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 | 1158 | |
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1159 | lemma eventually_not_equal_at_infinity: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1160 |   "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 | 1161 | proof - | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1162 | from filterlim_norm_at_top[where 'a = 'a] | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1163 | 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 | 1164 | thus ?thesis by eventually_elim auto | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1165 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1166 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1167 | lemma filterlim_int_of_nat_at_topD: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1168 | fixes F | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1169 | 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 | 1170 | shows "filterlim f F at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1171 | proof - | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1172 | 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 | 1173 | 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 | 1174 | 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 | 1175 | 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 | 1176 | finally show ?thesis . | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1177 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1178 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1179 | lemma filterlim_int_sequentially [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1180 | "filterlim int at_top sequentially" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1181 | unfolding filterlim_at_top | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1182 | proof | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1183 | fix C :: int | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1184 | 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 | 1185 | 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 | 1186 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1187 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1188 | 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 | 1189 | "filterlim real_of_int at_top at_top" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1190 | unfolding filterlim_at_top | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1191 | proof | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1192 | fix C :: real | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1193 | 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 | 1194 | 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 | 1195 | qed | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1196 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1197 | 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 | 1198 | proof (subst filterlim_cong[OF refl refl]) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1199 | 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 | 1200 | by eventually_elim simp | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1201 | qed (simp_all add: filterlim_ident) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1202 | |
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1203 | lemma filterlim_of_real_at_infinity [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1204 | "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 | 1205 | by (intro filterlim_norm_at_top_imp_at_infinity) (auto simp: filterlim_abs_real) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1206 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1207 | lemma not_tendsto_and_filterlim_at_infinity: | 
| 63546 | 1208 | fixes c :: "'a::real_normed_vector" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1209 | assumes "F \<noteq> bot" | 
| 63546 | 1210 | and "(f \<longlongrightarrow> c) F" | 
| 1211 | and "filterlim f at_infinity F" | |
| 1212 | shows False | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1213 | proof - | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 1214 | from tendstoD[OF assms(2), of "1/2"] | 
| 63546 | 1215 | have "eventually (\<lambda>x. dist (f x) c < 1/2) F" | 
| 1216 | by simp | |
| 1217 | moreover | |
| 1218 | from filterlim_at_infinity[of "norm c" f F] assms(3) | |
| 1219 | 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 | 1220 | ultimately have "eventually (\<lambda>x. False) F" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1221 | proof eventually_elim | 
| 63546 | 1222 | fix x | 
| 1223 | assume A: "dist (f x) c < 1/2" | |
| 1224 | 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 | 1225 | also have "norm (f x) = dist (f x) 0" by simp | 
| 63546 | 1226 | 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 | 1227 | finally show False using A by simp | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1228 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1229 | with assms show False by simp | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1230 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1231 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1232 | lemma filterlim_at_infinity_imp_not_convergent: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1233 | assumes "filterlim f at_infinity sequentially" | 
| 63546 | 1234 | shows "\<not> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1235 | by (rule notI, rule not_tendsto_and_filterlim_at_infinity[OF _ _ assms]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1236 | (simp_all add: convergent_LIMSEQ_iff) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1237 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1238 | lemma filterlim_at_infinity_imp_eventually_ne: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1239 | assumes "filterlim f at_infinity F" | 
| 63546 | 1240 | shows "eventually (\<lambda>z. f z \<noteq> c) F" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1241 | proof - | 
| 63546 | 1242 | have "norm c + 1 > 0" | 
| 1243 | by (intro add_nonneg_pos) simp_all | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1244 | with filterlim_at_infinity[OF order.refl, of f F] assms | 
| 63546 | 1245 | have "eventually (\<lambda>z. norm (f z) \<ge> norm c + 1) F" | 
| 1246 | by blast | |
| 1247 | then show ?thesis | |
| 1248 | by eventually_elim auto | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1249 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1250 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 1251 | lemma tendsto_of_nat [tendsto_intros]: | 
| 63546 | 1252 | "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 | 1253 | proof (subst filterlim_at_infinity[OF order.refl], intro allI impI) | 
| 63040 | 1254 | fix r :: real | 
| 1255 | assume r: "r > 0" | |
| 1256 | define n where "n = nat \<lceil>r\<rceil>" | |
| 63546 | 1257 | from r have n: "\<forall>m\<ge>n. of_nat m \<ge> r" | 
| 1258 | unfolding n_def by linarith | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1259 | from eventually_ge_at_top[of n] show "eventually (\<lambda>m. norm (of_nat m :: 'a) \<ge> r) sequentially" | 
| 63546 | 1260 | by eventually_elim (use n in simp_all) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1261 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1262 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1263 | |
| 60758 | 1264 | subsection \<open>Relate @{const at}, @{const at_left} and @{const at_right}\<close>
 | 
| 50347 | 1265 | |
| 60758 | 1266 | text \<open> | 
| 63546 | 1267 |   This lemmas are useful for conversion between @{term "at x"} to @{term "at_left x"} and
 | 
| 1268 |   @{term "at_right x"} and also @{term "at_right 0"}.
 | |
| 60758 | 1269 | \<close> | 
| 50347 | 1270 | |
| 51471 | 1271 | lemmas filterlim_split_at_real = filterlim_split_at[where 'a=real] | 
| 50323 | 1272 | |
| 63546 | 1273 | lemma filtermap_nhds_shift: "filtermap (\<lambda>x. x - d) (nhds a) = nhds (a - d)" | 
| 1274 | 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 | 1275 | by (rule filtermap_fun_inverse[where g="\<lambda>x. x + d"]) | 
| 63546 | 1276 | (auto intro!: tendsto_eq_intros filterlim_ident) | 
| 1277 | ||
| 1278 | lemma filtermap_nhds_minus: "filtermap (\<lambda>x. - x) (nhds a) = nhds (- a)" | |
| 1279 | 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 | 1280 | by (rule filtermap_fun_inverse[where g=uminus]) | 
| 63546 | 1281 | (auto intro!: tendsto_eq_intros filterlim_ident) | 
| 1282 | ||
| 1283 | lemma filtermap_at_shift: "filtermap (\<lambda>x. x - d) (at a) = at (a - d)" | |
| 1284 | 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 | 1285 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_shift[symmetric]) | 
| 50347 | 1286 | |
| 63546 | 1287 | lemma filtermap_at_right_shift: "filtermap (\<lambda>x. x - d) (at_right a) = at_right (a - d)" | 
| 1288 | 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 | 1289 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_shift[symmetric]) | 
| 50323 | 1290 | |
| 63546 | 1291 | lemma at_right_to_0: "at_right a = filtermap (\<lambda>x. x + a) (at_right 0)" | 
| 1292 | for a :: real | |
| 50347 | 1293 | using filtermap_at_right_shift[of "-a" 0] by simp | 
| 1294 | ||
| 1295 | lemma filterlim_at_right_to_0: | |
| 63546 | 1296 | "filterlim f F (at_right a) \<longleftrightarrow> filterlim (\<lambda>x. f (x + a)) F (at_right 0)" | 
| 1297 | for a :: real | |
| 50347 | 1298 | unfolding filterlim_def filtermap_filtermap at_right_to_0[of a] .. | 
| 1299 | ||
| 1300 | lemma eventually_at_right_to_0: | |
| 63546 | 1301 | "eventually P (at_right a) \<longleftrightarrow> eventually (\<lambda>x. P (x + a)) (at_right 0)" | 
| 1302 | for a :: real | |
| 50347 | 1303 | unfolding at_right_to_0[of a] by (simp add: eventually_filtermap) | 
| 1304 | ||
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1305 | 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 | 1306 | for a :: "'a::real_normed_vector" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1307 | 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 | 1308 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1309 | lemma filterlim_at_to_0: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1310 | "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 | 1311 | for a :: "'a::real_normed_vector" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1312 | 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 | 1313 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1314 | lemma eventually_at_to_0: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1315 | "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 | 1316 | for a :: "'a::real_normed_vector" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1317 | 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 | 1318 | |
| 63546 | 1319 | lemma filtermap_at_minus: "filtermap (\<lambda>x. - x) (at a) = at (- a)" | 
| 1320 | 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 | 1321 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_minus[symmetric]) | 
| 50347 | 1322 | |
| 63546 | 1323 | lemma at_left_minus: "at_left a = filtermap (\<lambda>x. - x) (at_right (- a))" | 
| 1324 | 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 | 1325 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_minus[symmetric]) | 
| 50323 | 1326 | |
| 63546 | 1327 | lemma at_right_minus: "at_right a = filtermap (\<lambda>x. - x) (at_left (- a))" | 
| 1328 | 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 | 1329 | by (simp add: filter_eq_iff eventually_filtermap eventually_at_filter filtermap_nhds_minus[symmetric]) | 
| 50347 | 1330 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1331 | |
| 50347 | 1332 | lemma filterlim_at_left_to_right: | 
| 63546 | 1333 | "filterlim f F (at_left a) \<longleftrightarrow> filterlim (\<lambda>x. f (- x)) F (at_right (-a))" | 
| 1334 | for a :: real | |
| 50347 | 1335 | unfolding filterlim_def filtermap_filtermap at_left_minus[of a] .. | 
| 1336 | ||
| 1337 | lemma eventually_at_left_to_right: | |
| 63546 | 1338 | "eventually P (at_left a) \<longleftrightarrow> eventually (\<lambda>x. P (- x)) (at_right (-a))" | 
| 1339 | for a :: real | |
| 50347 | 1340 | unfolding at_left_minus[of a] by (simp add: eventually_filtermap) | 
| 1341 | ||
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1342 | 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 | 1343 | 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 | 1344 | 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 | 1345 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1346 | 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 | 1347 | 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 | 1348 | 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 | 1349 | |
| 68532 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1350 | lemma at_bot_mirror : | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1351 |   shows "(at_bot::('a::{ordered_ab_group_add,linorder} filter)) = filtermap uminus at_top" 
 | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1352 | apply (rule filtermap_fun_inverse[of uminus, symmetric]) | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1353 | subgoal unfolding filterlim_at_top eventually_at_bot_linorder using le_minus_iff by auto | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1354 | subgoal unfolding filterlim_at_bot eventually_at_top_linorder using minus_le_iff by auto | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1355 | by auto | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1356 | |
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1357 | lemma at_top_mirror : | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1358 |   shows "(at_top::('a::{ordered_ab_group_add,linorder} filter)) = filtermap uminus at_bot"  
 | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1359 | apply (subst at_bot_mirror) | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68296diff
changeset | 1360 | by (auto simp add: 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 | 1361 | |
| 
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 | 1362 | 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 | 1363 | 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 | 1364 | |
| 
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 | 1365 | 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 | 1366 | 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 | 1367 | |
| 
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 | 1368 | 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 | 1369 | using filterlim_compose[OF filterlim_uminus_at_bot_at_top, of f F] | 
| 63546 | 1370 | 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 | 1371 | 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 | 1372 | |
| 67950 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1373 | lemma filterlim_at_infinity_imp_filterlim_at_top: | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1374 | 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 | 1375 | assumes "eventually (\<lambda>x. f x > 0) F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1376 | shows "filterlim f at_top F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1377 | proof - | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1378 | 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 | 1379 | 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 | 1380 | by (subst (asm) filterlim_cong[OF refl refl *]) | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1381 | qed | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1382 | |
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1383 | lemma filterlim_at_infinity_imp_filterlim_at_bot: | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1384 | 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 | 1385 | assumes "eventually (\<lambda>x. f x < 0) F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1386 | shows "filterlim f at_bot F" | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1387 | proof - | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1388 | 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 | 1389 | 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 | 1390 | unfolding filterlim_at_infinity_conv_norm_at_top | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1391 | by (subst (asm) filterlim_cong[OF refl refl *]) | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1392 | 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 | 1393 | qed | 
| 
99eaa5cedbb7
Added some simple facts about limits
 Manuel Eberl <eberlm@in.tum.de> parents: 
67707diff
changeset | 1394 | |
| 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 | 1395 | 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 | 1396 | unfolding filterlim_uminus_at_top by simp | 
| 50323 | 1397 | |
| 50347 | 1398 | 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 | 1399 | unfolding filterlim_at_top_gt[where c=0] eventually_at_filter | 
| 50347 | 1400 | proof safe | 
| 63546 | 1401 | fix Z :: real | 
| 1402 | assume [arith]: "0 < Z" | |
| 50347 | 1403 | then have "eventually (\<lambda>x. x < inverse Z) (nhds 0)" | 
| 1404 | by (auto simp add: 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 | 1405 |   then show "eventually (\<lambda>x. x \<noteq> 0 \<longrightarrow> x \<in> {0<..} \<longrightarrow> Z \<le> inverse x) (nhds 0)"
 | 
| 61810 | 1406 | by (auto elim!: eventually_mono simp: inverse_eq_divide field_simps) | 
| 50347 | 1407 | qed | 
| 1408 | ||
| 50325 | 1409 | lemma tendsto_inverse_0: | 
| 61076 | 1410 | fixes x :: "_ \<Rightarrow> 'a::real_normed_div_algebra" | 
| 61973 | 1411 | shows "(inverse \<longlongrightarrow> (0::'a)) at_infinity" | 
| 50325 | 1412 | unfolding tendsto_Zfun_iff diff_0_right Zfun_def eventually_at_infinity | 
| 1413 | proof safe | |
| 63546 | 1414 | fix r :: real | 
| 1415 | assume "0 < r" | |
| 50325 | 1416 | show "\<exists>b. \<forall>x. b \<le> norm x \<longrightarrow> norm (inverse x :: 'a) < r" | 
| 1417 | proof (intro exI[of _ "inverse (r / 2)"] allI impI) | |
| 1418 | fix x :: 'a | |
| 60758 | 1419 | from \<open>0 < r\<close> have "0 < inverse (r / 2)" by simp | 
| 50325 | 1420 | also assume *: "inverse (r / 2) \<le> norm x" | 
| 1421 | finally show "norm (inverse x) < r" | |
| 63546 | 1422 | using * \<open>0 < r\<close> | 
| 1423 | by (subst nonzero_norm_inverse) (simp_all add: inverse_eq_divide field_simps) | |
| 50325 | 1424 | qed | 
| 1425 | qed | |
| 1426 | ||
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1427 | lemma tendsto_add_filterlim_at_infinity: | 
| 63546 | 1428 | fixes c :: "'b::real_normed_vector" | 
| 1429 | and F :: "'a filter" | |
| 1430 | assumes "(f \<longlongrightarrow> c) F" | |
| 1431 | and "filterlim g at_infinity F" | |
| 1432 | 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 | 1433 | proof (subst filterlim_at_infinity[OF order_refl], safe) | 
| 63546 | 1434 | fix r :: real | 
| 1435 | assume r: "r > 0" | |
| 1436 | from assms(1) have "((\<lambda>x. norm (f x)) \<longlongrightarrow> norm c) F" | |
| 1437 | by (rule tendsto_norm) | |
| 1438 | then have "eventually (\<lambda>x. norm (f x) < norm c + 1) F" | |
| 1439 | by (rule order_tendstoD) simp_all | |
| 1440 | moreover from r have "r + norm c + 1 > 0" | |
| 1441 | by (intro add_pos_nonneg) simp_all | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1442 | with assms(2) have "eventually (\<lambda>x. norm (g x) \<ge> r + norm c + 1) F" | 
| 63546 | 1443 | unfolding filterlim_at_infinity[OF order_refl] | 
| 1444 | 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 | 1445 | 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 | 1446 | proof eventually_elim | 
| 63546 | 1447 | fix x :: 'a | 
| 1448 | assume A: "norm (f x) < norm c + 1" and B: "r + norm c + 1 \<le> norm (g x)" | |
| 1449 | from A B have "r \<le> norm (g x) - norm (f x)" | |
| 1450 | by simp | |
| 1451 | also have "norm (g x) - norm (f x) \<le> norm (g x + f x)" | |
| 1452 | by (rule norm_diff_ineq) | |
| 1453 | finally show "r \<le> norm (f x + g x)" | |
| 1454 | by (simp add: add_ac) | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1455 | qed | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1456 | qed | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1457 | |
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1458 | lemma tendsto_add_filterlim_at_infinity': | 
| 63546 | 1459 | fixes c :: "'b::real_normed_vector" | 
| 1460 | and F :: "'a filter" | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
61531diff
changeset | 1461 | assumes "filterlim f at_infinity F" | 
| 63546 | 1462 | and "(g \<longlongrightarrow> c) F" | 
| 1463 | 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 | 1464 | 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 | 1465 | |
| 60721 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1466 | 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 | 1467 | unfolding filterlim_at | 
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1468 | 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 | 1469 | (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 | 1470 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1471 | lemma filterlim_inverse_at_top: | 
| 61973 | 1472 | "(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 | 1473 | by (intro filterlim_compose[OF filterlim_inverse_at_top_right]) | 
| 61810 | 1474 | (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 | 1475 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1476 | 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 | 1477 | "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 | 1478 | 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 | 1479 | |
| 
c1b7793c23a3
generalized filtermap_homeomorph to filtermap_fun_inverse; add eventually_at_top/bot_not_equal
 hoelzl parents: 
60182diff
changeset | 1480 | lemma filterlim_inverse_at_bot: | 
| 61973 | 1481 | "(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 | 1482 | 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 | 1483 | 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 | 1484 | |
| 50347 | 1485 | 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 | 1486 | 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 | 1487 | (auto intro: filterlim_inverse_at_top_right filterlim_inverse_at_right_top) | 
| 50347 | 1488 | |
| 1489 | lemma eventually_at_right_to_top: | |
| 1490 | "eventually P (at_right (0::real)) \<longleftrightarrow> eventually (\<lambda>x. P (inverse x)) at_top" | |
| 1491 | unfolding at_right_to_top eventually_filtermap .. | |
| 1492 | ||
| 1493 | lemma filterlim_at_right_to_top: | |
| 1494 | "filterlim f F (at_right (0::real)) \<longleftrightarrow> (LIM x at_top. f (inverse x) :> F)" | |
| 1495 | unfolding filterlim_def at_right_to_top filtermap_filtermap .. | |
| 1496 | ||
| 1497 | lemma at_top_to_right: "at_top = filtermap inverse (at_right (0::real))" | |
| 1498 | unfolding at_right_to_top filtermap_filtermap inverse_inverse_eq filtermap_ident .. | |
| 1499 | ||
| 1500 | lemma eventually_at_top_to_right: | |
| 1501 | "eventually P at_top \<longleftrightarrow> eventually (\<lambda>x. P (inverse x)) (at_right (0::real))" | |
| 1502 | unfolding at_top_to_right eventually_filtermap .. | |
| 1503 | ||
| 1504 | lemma filterlim_at_top_to_right: | |
| 1505 | "filterlim f F at_top \<longleftrightarrow> (LIM x (at_right (0::real)). f (inverse x) :> F)" | |
| 1506 | unfolding filterlim_def at_top_to_right filtermap_filtermap .. | |
| 1507 | ||
| 50325 | 1508 | lemma filterlim_inverse_at_infinity: | 
| 61076 | 1509 |   fixes x :: "_ \<Rightarrow> 'a::{real_normed_div_algebra, division_ring}"
 | 
| 50325 | 1510 | shows "filterlim inverse at_infinity (at (0::'a))" | 
| 1511 | unfolding filterlim_at_infinity[OF order_refl] | |
| 1512 | proof safe | |
| 63546 | 1513 | fix r :: real | 
| 1514 | assume "0 < r" | |
| 50325 | 1515 | then show "eventually (\<lambda>x::'a. r \<le> norm (inverse x)) (at 0)" | 
| 1516 | unfolding eventually_at norm_inverse | |
| 1517 | by (intro exI[of _ "inverse r"]) | |
| 1518 | (auto simp: norm_conv_dist[symmetric] field_simps inverse_eq_divide) | |
| 1519 | qed | |
| 1520 | ||
| 1521 | lemma filterlim_inverse_at_iff: | |
| 61076 | 1522 |   fixes g :: "'a \<Rightarrow> 'b::{real_normed_div_algebra, division_ring}"
 | 
| 50325 | 1523 | shows "(LIM x F. inverse (g x) :> at 0) \<longleftrightarrow> (LIM x F. g x :> at_infinity)" | 
| 1524 | unfolding filterlim_def filtermap_filtermap[symmetric] | |
| 1525 | proof | |
| 1526 | assume "filtermap g F \<le> at_infinity" | |
| 1527 | then have "filtermap inverse (filtermap g F) \<le> filtermap inverse at_infinity" | |
| 1528 | by (rule filtermap_mono) | |
| 1529 | 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 | 1530 | 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 | 1531 | by (auto intro!: exI[of _ 1] | 
| 63546 | 1532 | simp: le_principal eventually_filtermap filterlim_def at_within_def eventually_at_infinity) | 
| 50325 | 1533 | finally show "filtermap inverse (filtermap g F) \<le> at 0" . | 
| 1534 | next | |
| 1535 | assume "filtermap inverse (filtermap g F) \<le> at 0" | |
| 1536 | then have "filtermap inverse (filtermap inverse (filtermap g F)) \<le> filtermap inverse (at 0)" | |
| 1537 | by (rule filtermap_mono) | |
| 1538 | with filterlim_inverse_at_infinity show "filtermap g F \<le> at_infinity" | |
| 1539 | by (auto intro: order_trans simp: filterlim_def filtermap_filtermap) | |
| 1540 | qed | |
| 1541 | ||
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1542 | lemma tendsto_mult_filterlim_at_infinity: | 
| 63546 | 1543 | fixes c :: "'a::real_normed_field" | 
| 64394 | 1544 | assumes "(f \<longlongrightarrow> c) F" "c \<noteq> 0" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1545 | assumes "filterlim g at_infinity F" | 
| 63546 | 1546 | shows "filterlim (\<lambda>x. f x * g x) at_infinity F" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1547 | proof - | 
| 61973 | 1548 | 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 | 1549 | by (intro tendsto_mult tendsto_inverse assms filterlim_compose[OF tendsto_inverse_0]) | 
| 63546 | 1550 | then have "filterlim (\<lambda>x. inverse (f x) * inverse (g x)) (at (inverse c * 0)) F" | 
| 1551 | unfolding filterlim_at | |
| 1552 | using assms | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1553 | by (auto intro: filterlim_at_infinity_imp_eventually_ne tendsto_imp_eventually_ne eventually_conj) | 
| 63546 | 1554 | then show ?thesis | 
| 1555 | by (subst filterlim_inverse_at_iff[symmetric]) simp_all | |
| 64394 | 1556 | qed | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 1557 | |
| 61973 | 1558 | lemma tendsto_inverse_0_at_top: "LIM x F. f x :> at_top \<Longrightarrow> ((\<lambda>x. inverse (f x) :: real) \<longlongrightarrow> 0) F" | 
| 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 | 1559 | by (metis filterlim_at filterlim_mono[OF _ at_top_le_at_infinity order_refl] filterlim_inverse_at_iff) | 
| 50419 | 1560 | |
| 63556 | 1561 | lemma real_tendsto_divide_at_top: | 
| 1562 | fixes c::"real" | |
| 1563 | assumes "(f \<longlongrightarrow> c) F" | |
| 1564 | assumes "filterlim g at_top F" | |
| 1565 | shows "((\<lambda>x. f x / g x) \<longlongrightarrow> 0) F" | |
| 1566 | by (auto simp: divide_inverse_commute | |
| 1567 | intro!: tendsto_mult[THEN tendsto_eq_rhs] tendsto_inverse_0_at_top assms) | |
| 1568 | ||
| 63546 | 1569 | lemma mult_nat_left_at_top: "c > 0 \<Longrightarrow> filterlim (\<lambda>x. c * x) at_top sequentially" | 
| 1570 | for c :: nat | |
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 1571 | 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 | 1572 | |
| 63546 | 1573 | lemma mult_nat_right_at_top: "c > 0 \<Longrightarrow> filterlim (\<lambda>x. x * c) at_top sequentially" | 
| 1574 | for c :: nat | |
| 66447 
a1f5c5c26fa6
Replaced subseq with strict_mono
 eberlm <eberlm@in.tum.de> parents: 
65680diff
changeset | 1575 | by (rule filterlim_subseq) (auto simp: strict_mono_def) | 
| 63546 | 1576 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1577 | lemma filterlim_times_pos: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1578 | "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 | 1579 | 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 | 1580 |   for c::"'a::{linordered_field, linorder_topology}"
 | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1581 | unfolding filterlim_iff | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1582 | proof safe | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1583 | fix P | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1584 | 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 | 1585 | 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 | 1586 | unfolding \<open>l = _ \<close> eventually_at_right_field | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1587 | by auto | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1588 | 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 | 1589 | 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 | 1590 | 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 | 1591 | 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 | 1592 | qed | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1593 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1594 | 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 | 1595 | for a c :: "'a::real_normed_field" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1596 | 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 | 1597 | (auto intro!: tendsto_eq_intros filterlim_ident) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1598 | |
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1599 | lemma filtermap_times_pos_at_right: | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1600 |   fixes c::"'a::{linordered_field, linorder_topology}"
 | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1601 | assumes "c > 0" | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1602 | 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 | 1603 | using assms | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1604 | 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 | 1605 | (auto intro!: filterlim_ident filterlim_times_pos) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 1606 | |
| 63546 | 1607 | 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 | 1608 | proof (rule antisym) | 
| 61973 | 1609 | 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 | 1610 | 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 | 1611 | then show "filtermap inverse at_infinity \<le> at (0::'a)" | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1612 | apply (simp add: le_principal eventually_filtermap eventually_at_infinity filterlim_def at_within_def) | 
| 63546 | 1613 | apply (rule_tac x="1" in exI) | 
| 1614 | apply auto | |
| 59613 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1615 | done | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1616 | next | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1617 | 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 | 1618 | 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 | 1619 | 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 | 1620 | 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 | 1621 | 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 | 1622 | qed | 
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1623 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1624 | lemma lim_at_infinity_0: | 
| 63546 | 1625 |   fixes l :: "'a::{real_normed_field,field}"
 | 
| 1626 | shows "(f \<longlongrightarrow> l) at_infinity \<longleftrightarrow> ((f \<circ> inverse) \<longlongrightarrow> l) (at (0::'a))" | |
| 1627 | 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 | 1628 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1629 | lemma lim_zero_infinity: | 
| 63546 | 1630 |   fixes l :: "'a::{real_normed_field,field}"
 | 
| 61973 | 1631 | shows "((\<lambda>x. f(1 / x)) \<longlongrightarrow> l) (at (0::'a)) \<Longrightarrow> (f \<longlongrightarrow> l) at_infinity" | 
| 63546 | 1632 | 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 | 1633 | |
| 
7103019278f0
The function frac. Various lemmas about limits, series, the exp function, etc.
 paulson <lp15@cam.ac.uk> parents: 
58889diff
changeset | 1634 | |
| 60758 | 1635 | text \<open> | 
| 63546 | 1636 | We only show rules for multiplication and addition when the functions are either against a real | 
| 1637 |   value or against infinity. Further rules are easy to derive by using @{thm
 | |
| 1638 | filterlim_uminus_at_top}. | |
| 60758 | 1639 | \<close> | 
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1640 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1641 | lemma filterlim_tendsto_pos_mult_at_top: | 
| 63546 | 1642 | assumes f: "(f \<longlongrightarrow> c) F" | 
| 1643 | and c: "0 < c" | |
| 1644 | 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 | 1645 | 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 | 1646 | 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 | 1647 | proof safe | 
| 63546 | 1648 | fix Z :: real | 
| 1649 | assume "0 < Z" | |
| 60758 | 1650 | from f \<open>0 < c\<close> have "eventually (\<lambda>x. c / 2 < f x) F" | 
| 61810 | 1651 | by (auto dest!: tendstoD[where e="c / 2"] elim!: eventually_mono | 
| 63546 | 1652 | 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 | 1653 | 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 | 1654 | 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 | 1655 | 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 | 1656 | proof eventually_elim | 
| 63546 | 1657 | case (elim x) | 
| 60758 | 1658 | 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 | 1659 | by (intro mult_mono) (auto simp: zero_le_divide_iff) | 
| 60758 | 1660 | 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 | 1661 | by simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1662 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1663 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1664 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1665 | 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 | 1666 | assumes f: "LIM x F. f x :> at_top" | 
| 63546 | 1667 | 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 | 1668 | 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 | 1669 | 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 | 1670 | proof safe | 
| 63546 | 1671 | fix Z :: real | 
| 1672 | 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 | 1673 | 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 | 1674 | 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 | 1675 | 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 | 1676 | 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 | 1677 | 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 | 1678 | proof eventually_elim | 
| 63546 | 1679 | case (elim x) | 
| 60758 | 1680 | 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 | 1681 | 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 | 1682 | 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 | 1683 | by simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1684 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1685 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1686 | |
| 63556 | 1687 | lemma filterlim_at_top_mult_tendsto_pos: | 
| 1688 | assumes f: "(f \<longlongrightarrow> c) F" | |
| 1689 | and c: "0 < c" | |
| 1690 | and g: "LIM x F. g x :> at_top" | |
| 1691 | shows "LIM x F. (g x * f x:: real) :> at_top" | |
| 1692 | by (auto simp: mult.commute intro!: filterlim_tendsto_pos_mult_at_top f c g) | |
| 1693 | ||
| 50419 | 1694 | lemma filterlim_tendsto_pos_mult_at_bot: | 
| 63546 | 1695 | fixes c :: real | 
| 1696 | assumes "(f \<longlongrightarrow> c) F" "0 < c" "filterlim g at_bot F" | |
| 50419 | 1697 | shows "LIM x F. f x * g x :> at_bot" | 
| 1698 | using filterlim_tendsto_pos_mult_at_top[OF assms(1,2), of "\<lambda>x. - g x"] assms(3) | |
| 1699 | unfolding filterlim_uminus_at_bot by simp | |
| 1700 | ||
| 60182 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1701 | lemma filterlim_tendsto_neg_mult_at_bot: | 
| 63546 | 1702 | fixes c :: real | 
| 1703 | 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 | 1704 | shows "LIM x F. f x * g x :> at_bot" | 
| 
e1ea5a6379c9
generalized tends over powr; added DERIV rule for powr
 hoelzl parents: 
60141diff
changeset | 1705 | 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 | 1706 | 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 | 1707 | |
| 56330 | 1708 | lemma filterlim_pow_at_top: | 
| 63721 | 1709 | fixes f :: "'a \<Rightarrow> real" | 
| 63546 | 1710 | assumes "0 < n" | 
| 1711 | and f: "LIM x F. f x :> at_top" | |
| 56330 | 1712 | shows "LIM x F. (f x)^n :: real :> at_top" | 
| 63546 | 1713 | using \<open>0 < n\<close> | 
| 1714 | proof (induct n) | |
| 1715 | case 0 | |
| 1716 | then show ?case by simp | |
| 1717 | next | |
| 56330 | 1718 | case (Suc n) with f show ?case | 
| 1719 | by (cases "n = 0") (auto intro!: filterlim_at_top_mult_at_top) | |
| 63546 | 1720 | qed | 
| 56330 | 1721 | |
| 1722 | lemma filterlim_pow_at_bot_even: | |
| 1723 | fixes f :: "real \<Rightarrow> real" | |
| 1724 | shows "0 < n \<Longrightarrow> LIM x F. f x :> at_bot \<Longrightarrow> even n \<Longrightarrow> LIM x F. (f x)^n :> at_top" | |
| 1725 | using filterlim_pow_at_top[of n "\<lambda>x. - f x" F] by (simp add: filterlim_uminus_at_top) | |
| 1726 | ||
| 1727 | lemma filterlim_pow_at_bot_odd: | |
| 1728 | fixes f :: "real \<Rightarrow> real" | |
| 1729 | shows "0 < n \<Longrightarrow> LIM x F. f x :> at_bot \<Longrightarrow> odd n \<Longrightarrow> LIM x F. (f x)^n :> at_bot" | |
| 1730 | using filterlim_pow_at_top[of n "\<lambda>x. - f x" F] by (simp add: filterlim_uminus_at_bot) | |
| 1731 | ||
| 67371 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1732 | lemma filterlim_power_at_infinity [tendsto_intros]: | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1733 | 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 | 1734 | assumes "filterlim f at_infinity F" "n > 0" | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1735 | 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 | 1736 | by (rule filterlim_norm_at_top_imp_at_infinity) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1737 | (auto simp: norm_power intro!: filterlim_pow_at_top assms | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1738 | intro: filterlim_at_infinity_imp_norm_at_top) | 
| 
2d9cf74943e1
moved in some material from Euler-MacLaurin
 paulson <lp15@cam.ac.uk> parents: 
67091diff
changeset | 1739 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1740 | lemma filterlim_tendsto_add_at_top: | 
| 61973 | 1741 | assumes f: "(f \<longlongrightarrow> c) F" | 
| 63546 | 1742 | 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 | 1743 | 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 | 1744 | 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 | 1745 | proof safe | 
| 63546 | 1746 | fix Z :: real | 
| 1747 | assume "0 < Z" | |
| 50324 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1748 | from f have "eventually (\<lambda>x. c - 1 < f x) F" | 
| 61810 | 1749 | 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 | 1750 | 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 | 1751 | 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 | 1752 | 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 | 1753 | by eventually_elim simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1754 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1755 | |
| 50347 | 1756 | lemma LIM_at_top_divide: | 
| 1757 | fixes f g :: "'a \<Rightarrow> real" | |
| 61973 | 1758 | assumes f: "(f \<longlongrightarrow> a) F" "0 < a" | 
| 63546 | 1759 | and g: "(g \<longlongrightarrow> 0) F" "eventually (\<lambda>x. 0 < g x) F" | 
| 50347 | 1760 | shows "LIM x F. f x / g x :> at_top" | 
| 1761 | unfolding divide_inverse | |
| 1762 | by (rule filterlim_tendsto_pos_mult_at_top[OF f]) (rule filterlim_inverse_at_top[OF g]) | |
| 1763 | ||
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1764 | 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 | 1765 | assumes f: "LIM x F. f x :> at_top" | 
| 63546 | 1766 | 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 | 1767 | 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 | 1768 | 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 | 1769 | proof safe | 
| 63546 | 1770 | fix Z :: real | 
| 1771 | 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 | 1772 | 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 | 1773 | 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 | 1774 | 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 | 1775 | 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 | 1776 | 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 | 1777 | by eventually_elim simp | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1778 | qed | 
| 
0a1242d5e7d4
add filterlim rules for diverging multiplication and addition; move at_infinity to the HOL image
 hoelzl parents: 
50323diff
changeset | 1779 | |
| 50331 | 1780 | lemma tendsto_divide_0: | 
| 61076 | 1781 |   fixes f :: "_ \<Rightarrow> 'a::{real_normed_div_algebra, division_ring}"
 | 
| 61973 | 1782 | assumes f: "(f \<longlongrightarrow> c) F" | 
| 63546 | 1783 | and g: "LIM x F. g x :> at_infinity" | 
| 61973 | 1784 | shows "((\<lambda>x. f x / g x) \<longlongrightarrow> 0) F" | 
| 63546 | 1785 | using tendsto_mult[OF f filterlim_compose[OF tendsto_inverse_0 g]] | 
| 1786 | by (simp add: divide_inverse) | |
| 50331 | 1787 | |
| 1788 | lemma linear_plus_1_le_power: | |
| 1789 | fixes x :: real | |
| 1790 | assumes x: "0 \<le> x" | |
| 1791 | shows "real n * x + 1 \<le> (x + 1) ^ n" | |
| 1792 | proof (induct n) | |
| 63546 | 1793 | case 0 | 
| 1794 | then show ?case by simp | |
| 1795 | next | |
| 50331 | 1796 | case (Suc n) | 
| 63546 | 1797 | from x have "real (Suc n) * x + 1 \<le> (x + 1) * (real n * x + 1)" | 
| 1798 | by (simp add: field_simps) | |
| 50331 | 1799 | also have "\<dots> \<le> (x + 1)^Suc n" | 
| 1800 | using Suc x by (simp add: mult_left_mono) | |
| 1801 | finally show ?case . | |
| 63546 | 1802 | qed | 
| 50331 | 1803 | |
| 1804 | lemma filterlim_realpow_sequentially_gt1: | |
| 1805 | fixes x :: "'a :: real_normed_div_algebra" | |
| 1806 | assumes x[arith]: "1 < norm x" | |
| 1807 | shows "LIM n sequentially. x ^ n :> at_infinity" | |
| 1808 | proof (intro filterlim_at_infinity[THEN iffD2] allI impI) | |
| 63546 | 1809 | fix y :: real | 
| 1810 | assume "0 < y" | |
| 50331 | 1811 | have "0 < norm x - 1" by simp | 
| 63546 | 1812 | then obtain N :: nat where "y < real N * (norm x - 1)" | 
| 1813 | by (blast dest: reals_Archimedean3) | |
| 1814 | also have "\<dots> \<le> real N * (norm x - 1) + 1" | |
| 1815 | by simp | |
| 1816 | also have "\<dots> \<le> (norm x - 1 + 1) ^ N" | |
| 1817 | by (rule linear_plus_1_le_power) simp | |
| 1818 | also have "\<dots> = norm x ^ N" | |
| 1819 | by simp | |
| 50331 | 1820 | finally have "\<forall>n\<ge>N. y \<le> norm x ^ n" | 
| 1821 | by (metis order_less_le_trans power_increasing order_less_imp_le x) | |
| 1822 | then show "eventually (\<lambda>n. y \<le> norm (x ^ n)) sequentially" | |
| 1823 | unfolding eventually_sequentially | |
| 1824 | by (auto simp: norm_power) | |
| 1825 | qed simp | |
| 1826 | ||
| 51471 | 1827 | |
| 66456 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1828 | lemma filterlim_divide_at_infinity: | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1829 | fixes f g :: "'a \<Rightarrow> 'a :: real_normed_field" | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1830 | 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 | 1831 | 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 | 1832 | proof - | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1833 | 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 | 1834 | 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 | 1835 | filterlim_compose [OF filterlim_inverse_at_infinity assms(2)]) | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1836 | thus ?thesis by (simp add: field_simps) | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1837 | qed | 
| 
621897f47fab
Various lemmas for HOL-Analysis
 Manuel Eberl <eberlm@in.tum.de> parents: 
66447diff
changeset | 1838 | |
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1839 | subsection \<open>Floor and Ceiling\<close> | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1840 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1841 | lemma eventually_floor_less: | 
| 63546 | 1842 |   fixes f :: "'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1843 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 1844 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1845 | 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 | 1846 | 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 | 1847 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1848 | lemma eventually_less_ceiling: | 
| 63546 | 1849 |   fixes f :: "'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1850 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 1851 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1852 | 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 | 1853 | 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 | 1854 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1855 | lemma eventually_floor_eq: | 
| 63546 | 1856 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1857 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 1858 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1859 | 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 | 1860 | using eventually_floor_less[OF assms] eventually_less_ceiling[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1861 | 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 | 1862 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1863 | lemma eventually_ceiling_eq: | 
| 63546 | 1864 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1865 | assumes f: "(f \<longlongrightarrow> l) F" | 
| 63546 | 1866 | and l: "l \<notin> \<int>" | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1867 | 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 | 1868 | using eventually_floor_less[OF assms] eventually_less_ceiling[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1869 | 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 | 1870 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1871 | lemma tendsto_of_int_floor: | 
| 63546 | 1872 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1873 | assumes "(f \<longlongrightarrow> l) F" | 
| 63546 | 1874 | and "l \<notin> \<int>" | 
| 1875 |   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 | 1876 | using eventually_floor_eq[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1877 | by (simp add: eventually_mono topological_tendstoI) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1878 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1879 | lemma tendsto_of_int_ceiling: | 
| 63546 | 1880 |   fixes f::"'a \<Rightarrow> 'b::{order_topology,floor_ceiling}"
 | 
| 63263 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1881 | assumes "(f \<longlongrightarrow> l) F" | 
| 63546 | 1882 | and "l \<notin> \<int>" | 
| 1883 |   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 | 1884 | using eventually_ceiling_eq[OF assms] | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1885 | by (simp add: eventually_mono topological_tendstoI) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1886 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1887 | lemma continuous_on_of_int_floor: | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1888 |   "continuous_on (UNIV - \<int>::'a::{order_topology, floor_ceiling} set)
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1889 |     (\<lambda>x. of_int (floor x)::'b::{ring_1, topological_space})"
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1890 | unfolding continuous_on_def | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1891 | by (auto intro!: tendsto_of_int_floor) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1892 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1893 | lemma continuous_on_of_int_ceiling: | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1894 |   "continuous_on (UNIV - \<int>::'a::{order_topology, floor_ceiling} set)
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1895 |     (\<lambda>x. of_int (ceiling x)::'b::{ring_1, topological_space})"
 | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1896 | unfolding continuous_on_def | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1897 | by (auto intro!: tendsto_of_int_ceiling) | 
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1898 | |
| 
c6c95d64607a
approximation, derivative, and continuity of floor and ceiling
 immler parents: 
63104diff
changeset | 1899 | |
| 60758 | 1900 | subsection \<open>Limits of Sequences\<close> | 
| 51526 | 1901 | |
| 62368 | 1902 | lemma [trans]: "X = Y \<Longrightarrow> Y \<longlonglongrightarrow> z \<Longrightarrow> X \<longlonglongrightarrow> z" | 
| 51526 | 1903 | by simp | 
| 1904 | ||
| 1905 | lemma LIMSEQ_iff: | |
| 1906 | fixes L :: "'a::real_normed_vector" | |
| 61969 | 1907 | 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 | 1908 | unfolding lim_sequentially dist_norm .. | 
| 51526 | 1909 | |
| 63546 | 1910 | lemma LIMSEQ_I: "(\<And>r. 0 < r \<Longrightarrow> \<exists>no. \<forall>n\<ge>no. norm (X n - L) < r) \<Longrightarrow> X \<longlonglongrightarrow> L" | 
| 1911 | for L :: "'a::real_normed_vector" | |
| 1912 | by (simp add: LIMSEQ_iff) | |
| 1913 | ||
| 1914 | lemma LIMSEQ_D: "X \<longlonglongrightarrow> L \<Longrightarrow> 0 < r \<Longrightarrow> \<exists>no. \<forall>n\<ge>no. norm (X n - L) < r" | |
| 1915 | for L :: "'a::real_normed_vector" | |
| 1916 | by (simp add: LIMSEQ_iff) | |
| 1917 | ||
| 1918 | lemma LIMSEQ_linear: "X \<longlonglongrightarrow> x \<Longrightarrow> l > 0 \<Longrightarrow> (\<lambda> n. X (n * l)) \<longlonglongrightarrow> x" | |
| 51526 | 1919 | unfolding tendsto_def eventually_sequentially | 
| 57512 
cc97b347b301
reduced name variants for assoc and commute on plus and mult
 haftmann parents: 
57447diff
changeset | 1920 | by (metis div_le_dividend div_mult_self1_is_m le_trans mult.commute) | 
| 51526 | 1921 | |
| 65036 
ab7e11730ad8
Some new lemmas. Existing lemmas modified to use uniform_limit rather than its expansion
 paulson <lp15@cam.ac.uk> parents: 
64394diff
changeset | 1922 | lemma norm_inverse_le_norm: "r \<le> norm x \<Longrightarrow> 0 < r \<Longrightarrow> norm (inverse x) \<le> inverse r" | 
| 63546 | 1923 | for x :: "'a::real_normed_div_algebra" | 
| 1924 | apply (subst nonzero_norm_inverse, clarsimp) | |
| 1925 | apply (erule (1) le_imp_inverse_le) | |
| 1926 | done | |
| 1927 | ||
| 1928 | lemma Bseq_inverse: "X \<longlonglongrightarrow> a \<Longrightarrow> a \<noteq> 0 \<Longrightarrow> Bseq (\<lambda>n. inverse (X n))" | |
| 1929 | for a :: "'a::real_normed_div_algebra" | |
| 51526 | 1930 | by (rule Bfun_inverse) | 
| 1931 | ||
| 63546 | 1932 | |
| 1933 | text \<open>Transformation of limit.\<close> | |
| 1934 | ||
| 1935 | lemma Lim_transform: "(g \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f x - g x) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> a) F" | |
| 1936 | for a b :: "'a::real_normed_vector" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1937 | 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 | 1938 | |
| 63546 | 1939 | lemma Lim_transform2: "(f \<longlongrightarrow> a) F \<Longrightarrow> ((\<lambda>x. f x - g x) \<longlongrightarrow> 0) F \<Longrightarrow> (g \<longlongrightarrow> a) F" | 
| 1940 | for a b :: "'a::real_normed_vector" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1941 | by (erule Lim_transform) (simp add: tendsto_minus_cancel) | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1942 | |
| 63546 | 1943 | proposition Lim_transform_eq: "((\<lambda>x. f x - g x) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> a) F \<longleftrightarrow> (g \<longlongrightarrow> a) F" | 
| 1944 | for a :: "'a::real_normed_vector" | |
| 1945 | 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 | 1946 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1947 | lemma Lim_transform_eventually: | 
| 61973 | 1948 | "eventually (\<lambda>x. f x = g x) net \<Longrightarrow> (f \<longlongrightarrow> l) net \<Longrightarrow> (g \<longlongrightarrow> l) net" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1949 | apply (rule topological_tendstoI) | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1950 | apply (drule (2) topological_tendstoD) | 
| 63546 | 1951 | apply (erule (1) eventually_elim2) | 
| 1952 | apply simp | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1953 | done | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1954 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1955 | lemma Lim_transform_within: | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 1956 | assumes "(f \<longlongrightarrow> l) (at x within S)" | 
| 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 1957 | and "0 < d" | 
| 63546 | 1958 | and "\<And>x'. x'\<in>S \<Longrightarrow> 0 < dist x' x \<Longrightarrow> dist x' x < d \<Longrightarrow> f x' = g x'" | 
| 61973 | 1959 | shows "(g \<longlongrightarrow> l) (at x within S)" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1960 | proof (rule Lim_transform_eventually) | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1961 | 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 | 1962 | using assms by (auto simp: eventually_at) | 
| 63546 | 1963 | show "(f \<longlongrightarrow> l) (at x within S)" | 
| 1964 | by fact | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1965 | qed | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1966 | |
| 67706 
4ddc49205f5d
Unified the order of zeros and poles; improved reasoning around non-essential singularites
 Wenda Li <wl302@cam.ac.uk> parents: 
67673diff
changeset | 1967 | 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 | 1968 | 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 | 1969 | 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 | 1970 | 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 | 1971 | 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 | 1972 | 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 | 1973 | 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 | 1974 | |
| 63546 | 1975 | 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 | 1976 | lemma Lim_transform_away_within: | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1977 | fixes a b :: "'a::t1_space" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1978 | assumes "a \<noteq> b" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1979 | and "\<forall>x\<in>S. x \<noteq> a \<and> x \<noteq> b \<longrightarrow> f x = g x" | 
| 61973 | 1980 | and "(f \<longlongrightarrow> l) (at a within S)" | 
| 1981 | shows "(g \<longlongrightarrow> l) (at a within S)" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1982 | proof (rule Lim_transform_eventually) | 
| 63546 | 1983 | show "(f \<longlongrightarrow> l) (at a within S)" | 
| 1984 | by fact | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1985 | 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 | 1986 | unfolding eventually_at_topological | 
| 63546 | 1987 |     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 | 1988 | qed | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1989 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1990 | lemma Lim_transform_away_at: | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1991 | fixes a b :: "'a::t1_space" | 
| 63546 | 1992 | assumes ab: "a \<noteq> b" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1993 | and fg: "\<forall>x. x \<noteq> a \<and> x \<noteq> b \<longrightarrow> f x = g x" | 
| 61973 | 1994 | and fl: "(f \<longlongrightarrow> l) (at a)" | 
| 1995 | shows "(g \<longlongrightarrow> l) (at a)" | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1996 | 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 | 1997 | |
| 63546 | 1998 | text \<open>Alternatively, within an open set.\<close> | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 1999 | lemma Lim_transform_within_open: | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2000 | assumes "(f \<longlongrightarrow> l) (at a within T)" | 
| 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2001 | and "open s" and "a \<in> s" | 
| 63546 | 2002 | 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 | 2003 | shows "(g \<longlongrightarrow> l) (at a within T)" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2004 | proof (rule Lim_transform_eventually) | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2005 | 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 | 2006 | unfolding eventually_at_topological | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2007 | using assms by auto | 
| 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2008 | 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 | 2009 | qed | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2010 | |
| 63546 | 2011 | |
| 2012 | 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 | 2013 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2014 | (* FIXME: Only one congruence rule for tendsto can be used at a time! *) | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2015 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2016 | lemma Lim_cong_within(*[cong add]*): | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2017 | assumes "a = b" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2018 | and "x = y" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2019 | and "S = T" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2020 | and "\<And>x. x \<noteq> b \<Longrightarrow> x \<in> T \<Longrightarrow> f x = g x" | 
| 61973 | 2021 | 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 | 2022 | unfolding tendsto_def eventually_at_topological | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2023 | using assms by simp | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2024 | |
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2025 | lemma Lim_cong_at(*[cong add]*): | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2026 | assumes "a = b" "x = y" | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2027 | and "\<And>x. x \<noteq> a \<Longrightarrow> f x = g x" | 
| 61973 | 2028 | shows "((\<lambda>x. f x) \<longlongrightarrow> x) (at a) \<longleftrightarrow> ((g \<longlongrightarrow> y) (at a))" | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2029 | unfolding tendsto_def eventually_at_topological | 
| 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2030 | using assms by simp | 
| 63546 | 2031 | |
| 2032 | 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 | 2033 | 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 | 2034 | 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 | 2035 | shows "(\<lambda>n. inverse (X n)) \<longlonglongrightarrow> 0" | 
| 51526 | 2036 | apply (rule filterlim_compose[OF tendsto_inverse_0]) | 
| 2037 | apply (simp add: filterlim_at_infinity[OF order_refl] eventually_sequentially) | |
| 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 | 2038 | apply (metis assms abs_le_D1 linorder_le_cases linorder_not_le) | 
| 51526 | 2039 | done | 
| 2040 | ||
| 63546 | 2041 | text \<open>The sequence @{term "1/n"} tends to 0 as @{term n} tends to infinity.\<close>
 | 
| 2042 | lemma LIMSEQ_inverse_real_of_nat: "(\<lambda>n. inverse (real (Suc n))) \<longlonglongrightarrow> 0" | |
| 51526 | 2043 | by (metis filterlim_compose tendsto_inverse_0 filterlim_mono order_refl filterlim_Suc | 
| 63546 | 2044 | filterlim_compose[OF filterlim_real_sequentially] at_top_le_at_infinity) | 
| 2045 | ||
| 2046 | text \<open> | |
| 2047 |   The sequence @{term "r + 1/n"} tends to @{term r} as @{term n} tends to
 | |
| 2048 | infinity is now easily proved. | |
| 2049 | \<close> | |
| 2050 | ||
| 2051 | lemma LIMSEQ_inverse_real_of_nat_add: "(\<lambda>n. r + inverse (real (Suc n))) \<longlonglongrightarrow> r" | |
| 51526 | 2052 | using tendsto_add [OF tendsto_const LIMSEQ_inverse_real_of_nat] by auto | 
| 2053 | ||
| 63546 | 2054 | lemma LIMSEQ_inverse_real_of_nat_add_minus: "(\<lambda>n. r + -inverse (real (Suc n))) \<longlonglongrightarrow> r" | 
| 51526 | 2055 | using tendsto_add [OF tendsto_const tendsto_minus [OF LIMSEQ_inverse_real_of_nat]] | 
| 2056 | by auto | |
| 2057 | ||
| 63546 | 2058 | lemma LIMSEQ_inverse_real_of_nat_add_minus_mult: "(\<lambda>n. r * (1 + - inverse (real (Suc n)))) \<longlonglongrightarrow> r" | 
| 51526 | 2059 | using tendsto_mult [OF tendsto_const LIMSEQ_inverse_real_of_nat_add_minus [of 1]] | 
| 2060 | by auto | |
| 2061 | ||
| 61973 | 2062 | 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 | 2063 | using lim_1_over_n by (simp add: inverse_eq_divide) | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2064 | |
| 67685 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2065 | 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 | 2066 | using lim_inverse_n | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2067 | by (simp add: inverse_eq_divide) | 
| 
bdff8bf0a75b
moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
 immler parents: 
67673diff
changeset | 2068 | |
| 61969 | 2069 | 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 | 2070 | proof (rule Lim_transform_eventually) | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2071 | show "eventually (\<lambda>n. 1 + inverse (of_nat n :: 'a) = of_nat (Suc n) / of_nat n) sequentially" | 
| 63546 | 2072 | using eventually_gt_at_top[of "0::nat"] | 
| 2073 | by eventually_elim (simp add: field_simps) | |
| 61969 | 2074 | 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 | 2075 | by (intro tendsto_add tendsto_const lim_inverse_n) | 
| 63546 | 2076 | then show "(\<lambda>n. 1 + inverse (of_nat n) :: 'a) \<longlonglongrightarrow> 1" | 
| 2077 | by simp | |
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2078 | qed | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2079 | |
| 61969 | 2080 | 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 | 2081 | proof (rule Lim_transform_eventually) | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2082 | show "eventually (\<lambda>n. inverse (of_nat (Suc n) / of_nat n :: 'a) = | 
| 63546 | 2083 | of_nat n / of_nat (Suc n)) sequentially" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2084 | using eventually_gt_at_top[of "0::nat"] | 
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2085 | by eventually_elim (simp add: field_simps del: of_nat_Suc) | 
| 61969 | 2086 | 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 | 2087 | by (intro tendsto_inverse LIMSEQ_Suc_n_over_n) simp_all | 
| 63546 | 2088 | then show "(\<lambda>n. inverse (of_nat (Suc n) / of_nat n :: 'a)) \<longlonglongrightarrow> 1" | 
| 2089 | by simp | |
| 61524 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2090 | qed | 
| 
f2e51e704a96
added many small lemmas about setsum/setprod/powr/...
 eberlm parents: 
61169diff
changeset | 2091 | |
| 63546 | 2092 | |
| 60758 | 2093 | subsection \<open>Convergence on sequences\<close> | 
| 51526 | 2094 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2095 | lemma convergent_cong: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2096 | assumes "eventually (\<lambda>x. f x = g x) sequentially" | 
| 63546 | 2097 | shows "convergent f \<longleftrightarrow> convergent g" | 
| 2098 | unfolding convergent_def | |
| 2099 | by (subst filterlim_cong[OF refl refl assms]) (rule refl) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2100 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2101 | lemma convergent_Suc_iff: "convergent (\<lambda>n. f (Suc n)) \<longleftrightarrow> convergent f" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2102 | by (auto simp: convergent_def LIMSEQ_Suc_iff) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2103 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2104 | lemma convergent_ignore_initial_segment: "convergent (\<lambda>n. f (n + m)) = convergent f" | 
| 63546 | 2105 | proof (induct m arbitrary: f) | 
| 2106 | case 0 | |
| 2107 | then show ?case by simp | |
| 2108 | next | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2109 | case (Suc m) | 
| 63546 | 2110 | have "convergent (\<lambda>n. f (n + Suc m)) \<longleftrightarrow> convergent (\<lambda>n. f (Suc n + m))" | 
| 2111 | by simp | |
| 2112 | also have "\<dots> \<longleftrightarrow> convergent (\<lambda>n. f (n + m))" | |
| 2113 | by (rule convergent_Suc_iff) | |
| 2114 | also have "\<dots> \<longleftrightarrow> convergent f" | |
| 2115 | by (rule Suc) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2116 | finally show ?case . | 
| 63546 | 2117 | qed | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2118 | |
| 51526 | 2119 | lemma convergent_add: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2120 | fixes X Y :: "nat \<Rightarrow> 'a::topological_monoid_add" | 
| 51526 | 2121 | assumes "convergent (\<lambda>n. X n)" | 
| 63546 | 2122 | and "convergent (\<lambda>n. Y n)" | 
| 51526 | 2123 | 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 | 2124 | using assms unfolding convergent_def by (blast intro: tendsto_add) | 
| 51526 | 2125 | |
| 64267 | 2126 | lemma convergent_sum: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2127 | fixes X :: "'a \<Rightarrow> nat \<Rightarrow> 'b::topological_comm_monoid_add" | 
| 63915 | 2128 | shows "(\<And>i. i \<in> A \<Longrightarrow> convergent (\<lambda>n. X i n)) \<Longrightarrow> convergent (\<lambda>n. \<Sum>i\<in>A. X i n)" | 
| 2129 | by (induct A rule: infinite_finite_induct) (simp_all add: convergent_const convergent_add) | |
| 51526 | 2130 | |
| 2131 | lemma (in bounded_linear) convergent: | |
| 2132 | assumes "convergent (\<lambda>n. X n)" | |
| 2133 | 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 | 2134 | using assms unfolding convergent_def by (blast intro: tendsto) | 
| 51526 | 2135 | |
| 2136 | lemma (in bounded_bilinear) convergent: | |
| 63546 | 2137 | assumes "convergent (\<lambda>n. X n)" | 
| 2138 | and "convergent (\<lambda>n. Y n)" | |
| 51526 | 2139 | 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 | 2140 | using assms unfolding convergent_def by (blast intro: tendsto) | 
| 51526 | 2141 | |
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2142 | lemma convergent_minus_iff: | 
| 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2143 | 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 | 2144 | 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 | 2145 | unfolding convergent_def by (force dest: tendsto_minus) | 
| 51526 | 2146 | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2147 | lemma convergent_diff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2148 | fixes X Y :: "nat \<Rightarrow> 'a::topological_group_add" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2149 | assumes "convergent (\<lambda>n. X n)" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2150 | assumes "convergent (\<lambda>n. Y n)" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2151 | 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 | 2152 | using assms unfolding convergent_def by (blast intro: tendsto_diff) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2153 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2154 | lemma convergent_norm: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2155 | assumes "convergent f" | 
| 63546 | 2156 | shows "convergent (\<lambda>n. norm (f n))" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2157 | proof - | 
| 63546 | 2158 | from assms have "f \<longlonglongrightarrow> lim f" | 
| 2159 | by (simp add: convergent_LIMSEQ_iff) | |
| 2160 | then have "(\<lambda>n. norm (f n)) \<longlonglongrightarrow> norm (lim f)" | |
| 2161 | by (rule tendsto_norm) | |
| 2162 | then show ?thesis | |
| 2163 | by (auto simp: convergent_def) | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2164 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2165 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2166 | lemma convergent_of_real: | 
| 63546 | 2167 | "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 | 2168 | unfolding convergent_def by (blast intro!: tendsto_of_real) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2169 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2170 | lemma convergent_add_const_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2171 | "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 | 2172 | proof | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2173 | assume "convergent (\<lambda>n. c + f n)" | 
| 63546 | 2174 | from convergent_diff[OF this convergent_const[of c]] show "convergent f" | 
| 2175 | by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2176 | next | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2177 | assume "convergent f" | 
| 63546 | 2178 | from convergent_add[OF convergent_const[of c] this] show "convergent (\<lambda>n. c + f n)" | 
| 2179 | by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2180 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2181 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2182 | lemma convergent_add_const_right_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2183 | "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 | 2184 | 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 | 2185 | |
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2186 | lemma convergent_diff_const_right_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2187 | "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 | 2188 | 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 | 2189 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2190 | lemma convergent_mult: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2191 | fixes X Y :: "nat \<Rightarrow> 'a::topological_semigroup_mult" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2192 | assumes "convergent (\<lambda>n. X n)" | 
| 63546 | 2193 | and "convergent (\<lambda>n. Y n)" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2194 | 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 | 2195 | using assms unfolding convergent_def by (blast intro: tendsto_mult) | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2196 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2197 | lemma convergent_mult_const_iff: | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2198 | assumes "c \<noteq> 0" | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2199 |   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 | 2200 | proof | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2201 | assume "convergent (\<lambda>n. c * f n)" | 
| 62087 
44841d07ef1d
revisions to limits and derivatives, plus new lemmas
 paulson parents: 
61976diff
changeset | 2202 | from assms convergent_mult[OF this convergent_const[of "inverse c"]] | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2203 | show "convergent f" by (simp add: field_simps) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2204 | next | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2205 | assume "convergent f" | 
| 63546 | 2206 | from convergent_mult[OF convergent_const[of c] this] show "convergent (\<lambda>n. c * f n)" | 
| 2207 | by simp | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2208 | qed | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2209 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2210 | lemma convergent_mult_const_right_iff: | 
| 68064 
b249fab48c76
type class generalisations; some work on infinite products
 paulson <lp15@cam.ac.uk> parents: 
67958diff
changeset | 2211 |   fixes c :: "'a::{field,topological_semigroup_mult}"
 | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2212 | assumes "c \<noteq> 0" | 
| 63546 | 2213 | shows "convergent (\<lambda>n. f n * c) \<longleftrightarrow> convergent f" | 
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2214 | 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 | 2215 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2216 | lemma convergent_imp_Bseq: "convergent f \<Longrightarrow> Bseq f" | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2217 | by (simp add: Cauchy_Bseq convergent_Cauchy) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2218 | |
| 51526 | 2219 | |
| 60758 | 2220 | text \<open>A monotone sequence converges to its least upper bound.\<close> | 
| 51526 | 2221 | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2222 | lemma LIMSEQ_incseq_SUP: | 
| 63546 | 2223 |   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 | 2224 | assumes u: "bdd_above (range X)" | 
| 63546 | 2225 | and X: "incseq X" | 
| 61969 | 2226 | 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 | 2227 | by (rule order_tendstoI) | 
| 63546 | 2228 | (auto simp: eventually_sequentially u less_cSUP_iff | 
| 2229 | intro: X[THEN incseqD] less_le_trans cSUP_lessD[OF u]) | |
| 51526 | 2230 | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2231 | lemma LIMSEQ_decseq_INF: | 
| 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2232 |   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 | 2233 | assumes u: "bdd_below (range X)" | 
| 63546 | 2234 | and X: "decseq X" | 
| 61969 | 2235 | 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 | 2236 | by (rule order_tendstoI) | 
| 63546 | 2237 | (auto simp: eventually_sequentially u cINF_less_iff | 
| 2238 | intro: X[THEN decseqD] le_less_trans less_cINF_D[OF u]) | |
| 2239 | ||
| 2240 | text \<open>Main monotonicity theorem.\<close> | |
| 2241 | ||
| 2242 | lemma Bseq_monoseq_convergent: "Bseq X \<Longrightarrow> monoseq X \<Longrightarrow> convergent X" | |
| 2243 | for X :: "nat \<Rightarrow> real" | |
| 2244 | by (auto simp: monoseq_iff convergent_def intro: LIMSEQ_decseq_INF LIMSEQ_incseq_SUP | |
| 2245 | dest: Bseq_bdd_above Bseq_bdd_below) | |
| 2246 | ||
| 2247 | lemma Bseq_mono_convergent: "Bseq X \<Longrightarrow> (\<forall>m n. m \<le> n \<longrightarrow> X m \<le> X n) \<Longrightarrow> convergent X" | |
| 2248 | for X :: "nat \<Rightarrow> real" | |
| 54263 
c4159fe6fa46
move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
 hoelzl parents: 
54230diff
changeset | 2249 | by (auto intro!: Bseq_monoseq_convergent incseq_imp_monoseq simp: incseq_def) | 
| 51526 | 2250 | |
| 63546 | 2251 | lemma monoseq_imp_convergent_iff_Bseq: "monoseq f \<Longrightarrow> convergent f \<longleftrightarrow> Bseq f" | 
| 2252 | for f :: "nat \<Rightarrow> real" | |
| 61531 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2253 | 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 | 2254 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2255 | lemma Bseq_monoseq_convergent'_inc: | 
| 63546 | 2256 | fixes f :: "nat \<Rightarrow> real" | 
| 2257 | 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 | 2258 | by (subst convergent_ignore_initial_segment [symmetric, of _ M]) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2259 | (auto intro!: Bseq_monoseq_convergent simp: monoseq_def) | 
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2260 | |
| 
ab2e862263e7
Rounding function, uniform limits, cotangent, binomial identities
 eberlm parents: 
61524diff
changeset | 2261 | lemma Bseq_monoseq_convergent'_dec: | 
| 63546 | 2262 | fixes f :: "nat \<Rightarrow> real" | 
| 2263 | 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 | 2264 | by (subst convergent_ignore_initial_segment [symmetric, of _ M]) | 
| 63546 | 2265 | (auto intro!: Bseq_monoseq_convergent simp: monoseq_def) | 
| 2266 | ||
| 2267 | 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)" | |
| 2268 | for X :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 51526 | 2269 | unfolding Cauchy_def dist_norm .. | 
| 2270 | ||
| 63546 | 2271 | 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" | 
| 2272 | for X :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 2273 | by (simp add: Cauchy_iff) | |
| 2274 | ||
| 2275 | lemma CauchyD: "Cauchy X \<Longrightarrow> 0 < e \<Longrightarrow> \<exists>M. \<forall>m\<ge>M. \<forall>n\<ge>M. norm (X m - X n) < e" | |
| 2276 | for X :: "nat \<Rightarrow> 'a::real_normed_vector" | |
| 2277 | by (simp add: Cauchy_iff) | |
| 51526 | 2278 | |
| 2279 | lemma incseq_convergent: | |
| 2280 | fixes X :: "nat \<Rightarrow> real" | |
| 63546 | 2281 | assumes "incseq X" | 
| 2282 | and "\<forall>i. X i \<le> B" | |
| 61969 | 2283 | obtains L where "X \<longlonglongrightarrow> L" "\<forall>i. X i \<le> L" | 
| 51526 | 2284 | proof atomize_elim | 
| 60758 | 2285 | from incseq_bounded[OF assms] \<open>incseq X\<close> Bseq_monoseq_convergent[of X] | 
| 61969 | 2286 | obtain L where "X \<longlonglongrightarrow> L" | 
| 51526 | 2287 | by (auto simp: convergent_def monoseq_def incseq_def) | 
| 61969 | 2288 | with \<open>incseq X\<close> show "\<exists>L. X \<longlonglongrightarrow> L \<and> (\<forall>i. X i \<le> L)" | 
| 51526 | 2289 | by (auto intro!: exI[of _ L] incseq_le) | 
| 2290 | qed | |
| 2291 | ||
| 2292 | lemma decseq_convergent: | |
| 2293 | fixes X :: "nat \<Rightarrow> real" | |
| 63546 | 2294 | assumes "decseq X" | 
| 2295 | and "\<forall>i. B \<le> X i" | |
| 61969 | 2296 | obtains L where "X \<longlonglongrightarrow> L" "\<forall>i. L \<le> X i" | 
| 51526 | 2297 | proof atomize_elim | 
| 60758 | 2298 | from decseq_bounded[OF assms] \<open>decseq X\<close> Bseq_monoseq_convergent[of X] | 
| 61969 | 2299 | obtain L where "X \<longlonglongrightarrow> L" | 
| 51526 | 2300 | by (auto simp: convergent_def monoseq_def decseq_def) | 
| 61969 | 2301 | 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 | 2302 | by (auto intro!: exI[of _ L] decseq_ge) | 
| 51526 | 2303 | qed | 
| 2304 | ||
| 63546 | 2305 | |
| 60758 | 2306 | subsection \<open>Power Sequences\<close> | 
| 51526 | 2307 | |
| 63546 | 2308 | lemma Bseq_realpow: "0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> Bseq (\<lambda>n. x ^ n)" | 
| 2309 | for x :: real | |
| 2310 | apply (simp add: Bseq_def) | |
| 2311 | apply (rule_tac x = 1 in exI) | |
| 2312 | apply (simp add: power_abs) | |
| 2313 | apply (auto dest: power_mono) | |
| 2314 | done | |
| 2315 | ||
| 2316 | lemma monoseq_realpow: "0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> monoseq (\<lambda>n. x ^ n)" | |
| 2317 | for x :: real | |
| 2318 | apply (clarify intro!: mono_SucI2) | |
| 2319 | apply (cut_tac n = n and N = "Suc n" and a = x in power_decreasing) | |
| 2320 | apply auto | |
| 2321 | done | |
| 2322 | ||
| 2323 | lemma convergent_realpow: "0 \<le> x \<Longrightarrow> x \<le> 1 \<Longrightarrow> convergent (\<lambda>n. x ^ n)" | |
| 2324 | for x :: real | |
| 2325 | by (blast intro!: Bseq_monoseq_convergent Bseq_realpow monoseq_realpow) | |
| 2326 | ||
| 2327 | lemma LIMSEQ_inverse_realpow_zero: "1 < x \<Longrightarrow> (\<lambda>n. inverse (x ^ n)) \<longlonglongrightarrow> 0" | |
| 2328 | for x :: real | |
| 51526 | 2329 | by (rule filterlim_compose[OF tendsto_inverse_0 filterlim_realpow_sequentially_gt1]) simp | 
| 2330 | ||
| 2331 | lemma LIMSEQ_realpow_zero: | |
| 63546 | 2332 | fixes x :: real | 
| 2333 | assumes "0 \<le> x" "x < 1" | |
| 2334 | shows "(\<lambda>n. x ^ n) \<longlonglongrightarrow> 0" | |
| 2335 | proof (cases "x = 0") | |
| 2336 | case False | |
| 2337 | with \<open>0 \<le> x\<close> have x0: "0 < x" by simp | |
| 2338 | then have "1 < inverse x" | |
| 2339 | using \<open>x < 1\<close> by (rule one_less_inverse) | |
| 2340 | then have "(\<lambda>n. inverse (inverse x ^ n)) \<longlonglongrightarrow> 0" | |
| 51526 | 2341 | by (rule LIMSEQ_inverse_realpow_zero) | 
| 63546 | 2342 | then show ?thesis by (simp add: power_inverse) | 
| 2343 | next | |
| 2344 | case True | |
| 2345 | show ?thesis | |
| 2346 | by (rule LIMSEQ_imp_Suc) (simp add: True) | |
| 2347 | qed | |
| 2348 | ||
| 2349 | lemma LIMSEQ_power_zero: "norm x < 1 \<Longrightarrow> (\<lambda>n. x ^ n) \<longlonglongrightarrow> 0" | |
| 2350 | for x :: "'a::real_normed_algebra_1" | |
| 2351 | apply (drule LIMSEQ_realpow_zero [OF norm_ge_zero]) | |
| 2352 | apply (simp only: tendsto_Zfun_iff, erule Zfun_le) | |
| 2353 | apply (simp add: power_abs norm_power_ineq) | |
| 2354 | done | |
| 51526 | 2355 | |
| 61969 | 2356 | lemma LIMSEQ_divide_realpow_zero: "1 < x \<Longrightarrow> (\<lambda>n. a / (x ^ n) :: real) \<longlonglongrightarrow> 0" | 
| 51526 | 2357 | by (rule tendsto_divide_0 [OF tendsto_const filterlim_realpow_sequentially_gt1]) simp | 
| 2358 | ||
| 63556 | 2359 | lemma | 
| 2360 | tendsto_power_zero: | |
| 2361 | fixes x::"'a::real_normed_algebra_1" | |
| 2362 | assumes "filterlim f at_top F" | |
| 2363 | assumes "norm x < 1" | |
| 2364 | shows "((\<lambda>y. x ^ (f y)) \<longlongrightarrow> 0) F" | |
| 2365 | proof (rule tendstoI) | |
| 2366 | fix e::real assume "0 < e" | |
| 2367 | from tendstoD[OF LIMSEQ_power_zero[OF \<open>norm x < 1\<close>] \<open>0 < e\<close>] | |
| 2368 | have "\<forall>\<^sub>F xa in sequentially. norm (x ^ xa) < e" | |
| 2369 | by simp | |
| 2370 | then obtain N where N: "norm (x ^ n) < e" if "n \<ge> N" for n | |
| 2371 | by (auto simp: eventually_sequentially) | |
| 2372 | have "\<forall>\<^sub>F i in F. f i \<ge> N" | |
| 2373 | using \<open>filterlim f sequentially F\<close> | |
| 2374 | by (simp add: filterlim_at_top) | |
| 2375 | then show "\<forall>\<^sub>F i in F. dist (x ^ f i) 0 < e" | |
| 2376 | by (eventually_elim) (auto simp: N) | |
| 2377 | qed | |
| 2378 | ||
| 63546 | 2379 | text \<open>Limit of @{term "c^n"} for @{term"\<bar>c\<bar> < 1"}.\<close>
 | 
| 51526 | 2380 | |
| 61969 | 2381 | lemma LIMSEQ_rabs_realpow_zero: "\<bar>c\<bar> < 1 \<Longrightarrow> (\<lambda>n. \<bar>c\<bar> ^ n :: real) \<longlonglongrightarrow> 0" | 
| 51526 | 2382 | by (rule LIMSEQ_realpow_zero [OF abs_ge_zero]) | 
| 2383 | ||
| 61969 | 2384 | lemma LIMSEQ_rabs_realpow_zero2: "\<bar>c\<bar> < 1 \<Longrightarrow> (\<lambda>n. c ^ n :: real) \<longlonglongrightarrow> 0" | 
| 51526 | 2385 | by (rule LIMSEQ_power_zero) simp | 
| 2386 | ||
| 2387 | ||
| 60758 | 2388 | subsection \<open>Limits of Functions\<close> | 
| 51526 | 2389 | |
| 63546 | 2390 | 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)" | 
| 2391 | for a :: "'a::real_normed_vector" and L :: "'b::real_normed_vector" | |
| 2392 | by (simp add: LIM_def dist_norm) | |
| 51526 | 2393 | |
| 2394 | lemma LIM_I: | |
| 63546 | 2395 | "(\<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" | 
| 2396 | for a :: "'a::real_normed_vector" and L :: "'b::real_normed_vector" | |
| 2397 | by (simp add: LIM_eq) | |
| 2398 | ||
| 2399 | 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" | |
| 2400 | for a :: "'a::real_normed_vector" and L :: "'b::real_normed_vector" | |
| 2401 | by (simp add: LIM_eq) | |
| 2402 | ||
| 2403 | lemma LIM_offset: "f \<midarrow>a\<rightarrow> L \<Longrightarrow> (\<lambda>x. f (x + k)) \<midarrow>(a - k)\<rightarrow> L" | |
| 2404 | for a :: "'a::real_normed_vector" | |
| 2405 | by (simp add: filtermap_at_shift[symmetric, of a k] filterlim_def filtermap_filtermap) | |
| 2406 | ||
| 2407 | lemma LIM_offset_zero: "f \<midarrow>a\<rightarrow> L \<Longrightarrow> (\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> L" | |
| 2408 | for a :: "'a::real_normed_vector" | |
| 2409 | by (drule LIM_offset [where k = a]) (simp add: add.commute) | |
| 2410 | ||
| 2411 | lemma LIM_offset_zero_cancel: "(\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> L \<Longrightarrow> f \<midarrow>a\<rightarrow> L" | |
| 2412 | for a :: "'a::real_normed_vector" | |
| 2413 | by (drule LIM_offset [where k = "- a"]) simp | |
| 2414 | ||
| 2415 | lemma LIM_offset_zero_iff: "f \<midarrow>a\<rightarrow> L \<longleftrightarrow> (\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> L" | |
| 2416 | 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 | 2417 | 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 | 2418 | |
| 63546 | 2419 | 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 | 2420 | for f :: "'a \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 2421 | unfolding tendsto_iff dist_norm by simp | 
| 51526 | 2422 | |
| 2423 | 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 | 2424 | fixes f :: "'a \<Rightarrow> 'b::real_normed_vector" | 
| 61973 | 2425 | shows "((\<lambda>x. f x - l) \<longlongrightarrow> 0) F \<Longrightarrow> (f \<longlongrightarrow> l) F" | 
| 51526 | 2426 | unfolding tendsto_iff dist_norm by simp | 
| 2427 | ||
| 63546 | 2428 | 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 | 2429 | for f :: "'a \<Rightarrow> 'b::real_normed_vector" | 
| 63546 | 2430 | unfolding tendsto_iff dist_norm by simp | 
| 51526 | 2431 | |
| 2432 | lemma LIM_imp_LIM: | |
| 2433 | fixes f :: "'a::topological_space \<Rightarrow> 'b::real_normed_vector" | |
| 2434 | fixes g :: "'a::topological_space \<Rightarrow> 'c::real_normed_vector" | |
| 61976 | 2435 | assumes f: "f \<midarrow>a\<rightarrow> l" | 
| 63546 | 2436 | and le: "\<And>x. x \<noteq> a \<Longrightarrow> norm (g x - m) \<le> norm (f x - l)" | 
| 61976 | 2437 | shows "g \<midarrow>a\<rightarrow> m" | 
| 63546 | 2438 | by (rule metric_LIM_imp_LIM [OF f]) (simp add: dist_norm le) | 
| 51526 | 2439 | |
| 2440 | lemma LIM_equal2: | |
| 2441 | fixes f g :: "'a::real_normed_vector \<Rightarrow> 'b::topological_space" | |
| 63546 | 2442 | assumes "0 < R" | 
| 2443 | and "\<And>x. x \<noteq> a \<Longrightarrow> norm (x - a) < R \<Longrightarrow> f x = g x" | |
| 61976 | 2444 | shows "g \<midarrow>a\<rightarrow> l \<Longrightarrow> f \<midarrow>a\<rightarrow> l" | 
| 63546 | 2445 | by (rule metric_LIM_equal2 [OF assms]) (simp_all add: dist_norm) | 
| 51526 | 2446 | |
| 2447 | lemma LIM_compose2: | |
| 2448 | fixes a :: "'a::real_normed_vector" | |
| 61976 | 2449 | assumes f: "f \<midarrow>a\<rightarrow> b" | 
| 63546 | 2450 | and g: "g \<midarrow>b\<rightarrow> c" | 
| 2451 | and inj: "\<exists>d>0. \<forall>x. x \<noteq> a \<and> norm (x - a) < d \<longrightarrow> f x \<noteq> b" | |
| 61976 | 2452 | shows "(\<lambda>x. g (f x)) \<midarrow>a\<rightarrow> c" | 
| 63546 | 2453 | by (rule metric_LIM_compose2 [OF f g inj [folded dist_norm]]) | 
| 51526 | 2454 | |
| 2455 | lemma real_LIM_sandwich_zero: | |
| 2456 | fixes f g :: "'a::topological_space \<Rightarrow> real" | |
| 61976 | 2457 | assumes f: "f \<midarrow>a\<rightarrow> 0" | 
| 63546 | 2458 | and 1: "\<And>x. x \<noteq> a \<Longrightarrow> 0 \<le> g x" | 
| 2459 | and 2: "\<And>x. x \<noteq> a \<Longrightarrow> g x \<le> f x" | |
| 61976 | 2460 | shows "g \<midarrow>a\<rightarrow> 0" | 
| 51526 | 2461 | proof (rule LIM_imp_LIM [OF f]) (* FIXME: use tendsto_sandwich *) | 
| 63546 | 2462 | fix x | 
| 2463 | assume x: "x \<noteq> a" | |
| 2464 | with 1 have "norm (g x - 0) = g x" by simp | |
| 51526 | 2465 | also have "g x \<le> f x" by (rule 2 [OF x]) | 
| 2466 | also have "f x \<le> \<bar>f x\<bar>" by (rule abs_ge_self) | |
| 2467 | also have "\<bar>f x\<bar> = norm (f x - 0)" by simp | |
| 2468 | finally show "norm (g x - 0) \<le> norm (f x - 0)" . | |
| 2469 | qed | |
| 2470 | ||
| 2471 | ||
| 60758 | 2472 | subsection \<open>Continuity\<close> | 
| 51526 | 2473 | |
| 63546 | 2474 | lemma LIM_isCont_iff: "(f \<midarrow>a\<rightarrow> f a) = ((\<lambda>h. f (a + h)) \<midarrow>0\<rightarrow> f a)" | 
| 2475 | for f :: "'a::real_normed_vector \<Rightarrow> 'b::topological_space" | |
| 2476 | by (rule iffI [OF LIM_offset_zero LIM_offset_zero_cancel]) | |
| 2477 | ||
| 2478 | lemma isCont_iff: "isCont f x = (\<lambda>h. f (x + h)) \<midarrow>0\<rightarrow> f x" | |
| 2479 | for f :: "'a::real_normed_vector \<Rightarrow> 'b::topological_space" | |
| 2480 | by (simp add: isCont_def LIM_isCont_iff) | |
| 51526 | 2481 | |
| 2482 | lemma isCont_LIM_compose2: | |
| 2483 | fixes a :: "'a::real_normed_vector" | |
| 2484 | assumes f [unfolded isCont_def]: "isCont f a" | |
| 63546 | 2485 | and g: "g \<midarrow>f a\<rightarrow> l" | 
| 2486 | and inj: "\<exists>d>0. \<forall>x. x \<noteq> a \<and> norm (x - a) < d \<longrightarrow> f x \<noteq> f a" | |
| 61976 | 2487 | shows "(\<lambda>x. g (f x)) \<midarrow>a\<rightarrow> l" | 
| 63546 | 2488 | by (rule LIM_compose2 [OF f g inj]) | 
| 2489 | ||
| 2490 | lemma isCont_norm [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. norm (f x)) a" | |
| 2491 | for f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | |
| 51526 | 2492 | by (fact continuous_norm) | 
| 2493 | ||
| 63546 | 2494 | lemma isCont_rabs [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. \<bar>f x\<bar>) a" | 
| 2495 | for f :: "'a::t2_space \<Rightarrow> real" | |
| 51526 | 2496 | by (fact continuous_rabs) | 
| 2497 | ||
| 63546 | 2498 | lemma isCont_add [simp]: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x + g x) a" | 
| 2499 | for f :: "'a::t2_space \<Rightarrow> 'b::topological_monoid_add" | |
| 51526 | 2500 | by (fact continuous_add) | 
| 2501 | ||
| 63546 | 2502 | lemma isCont_minus [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. - f x) a" | 
| 2503 | for f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | |
| 51526 | 2504 | by (fact continuous_minus) | 
| 2505 | ||
| 63546 | 2506 | lemma isCont_diff [simp]: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x - g x) a" | 
| 2507 | for f :: "'a::t2_space \<Rightarrow> 'b::real_normed_vector" | |
| 51526 | 2508 | by (fact continuous_diff) | 
| 2509 | ||
| 63546 | 2510 | lemma isCont_mult [simp]: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x * g x) a" | 
| 2511 | for f g :: "'a::t2_space \<Rightarrow> 'b::real_normed_algebra" | |
| 51526 | 2512 | by (fact continuous_mult) | 
| 2513 | ||
| 63546 | 2514 | lemma (in bounded_linear) isCont: "isCont g a \<Longrightarrow> isCont (\<lambda>x. f (g x)) a" | 
| 51526 | 2515 | by (fact continuous) | 
| 2516 | ||
| 63546 | 2517 | lemma (in bounded_bilinear) isCont: "isCont f a \<Longrightarrow> isCont g a \<Longrightarrow> isCont (\<lambda>x. f x ** g x) a" | 
| 51526 | 2518 | by (fact continuous) | 
| 2519 | ||
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2520 | lemmas isCont_scaleR [simp] = | 
| 51526 | 2521 | bounded_bilinear.isCont [OF bounded_bilinear_scaleR] | 
| 2522 | ||
| 2523 | lemmas isCont_of_real [simp] = | |
| 2524 | bounded_linear.isCont [OF bounded_linear_of_real] | |
| 2525 | ||
| 63546 | 2526 | lemma isCont_power [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. f x ^ n) a" | 
| 2527 |   for f :: "'a::t2_space \<Rightarrow> 'b::{power,real_normed_algebra}"
 | |
| 51526 | 2528 | by (fact continuous_power) | 
| 2529 | ||
| 64267 | 2530 | 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 | 2531 | for f :: "'a \<Rightarrow> 'b::t2_space \<Rightarrow> 'c::topological_comm_monoid_add" | 
| 64267 | 2532 | by (auto intro: continuous_sum) | 
| 51526 | 2533 | |
| 63546 | 2534 | |
| 60758 | 2535 | subsection \<open>Uniform Continuity\<close> | 
| 51526 | 2536 | |
| 63104 | 2537 | lemma uniformly_continuous_on_def: | 
| 2538 | fixes f :: "'a::metric_space \<Rightarrow> 'b::metric_space" | |
| 2539 | shows "uniformly_continuous_on s f \<longleftrightarrow> | |
| 2540 | (\<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)" | |
| 2541 | unfolding uniformly_continuous_on_uniformity | |
| 2542 | uniformity_dist filterlim_INF filterlim_principal eventually_inf_principal | |
| 2543 | by (force simp: Ball_def uniformity_dist[symmetric] eventually_uniformity_metric) | |
| 2544 | ||
| 63546 | 2545 | abbreviation isUCont :: "['a::metric_space \<Rightarrow> 'b::metric_space] \<Rightarrow> bool" | 
| 2546 | where "isUCont f \<equiv> uniformly_continuous_on UNIV f" | |
| 2547 | ||
| 2548 | 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 | 2549 | 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 | 2550 | |
| 63546 | 2551 | lemma isUCont_isCont: "isUCont f \<Longrightarrow> isCont f x" | 
| 63104 | 2552 | by (drule uniformly_continuous_imp_continuous) (simp add: continuous_on_eq_continuous_at) | 
| 2553 | ||
| 2554 | lemma uniformly_continuous_on_Cauchy: | |
| 63546 | 2555 | fixes f :: "'a::metric_space \<Rightarrow> 'b::metric_space" | 
| 63104 | 2556 | assumes "uniformly_continuous_on S f" "Cauchy X" "\<And>n. X n \<in> S" | 
| 2557 | shows "Cauchy (\<lambda>n. f (X n))" | |
| 2558 | using assms | |
| 63546 | 2559 | apply (simp only: uniformly_continuous_on_def) | 
| 63104 | 2560 | apply (rule metric_CauchyI) | 
| 63546 | 2561 | apply (drule_tac x=e in spec) | 
| 2562 | apply safe | |
| 2563 | apply (drule_tac e=d in metric_CauchyD) | |
| 2564 | apply safe | |
| 2565 | apply (rule_tac x=M in exI) | |
| 2566 | apply simp | |
| 63104 | 2567 | done | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 2568 | |
| 63546 | 2569 | lemma isUCont_Cauchy: "isUCont f \<Longrightarrow> Cauchy X \<Longrightarrow> Cauchy (\<lambda>n. f (X n))" | 
| 63104 | 2570 | by (rule uniformly_continuous_on_Cauchy[where S=UNIV and f=f]) simp_all | 
| 64287 | 2571 | |
| 2572 | lemma uniformly_continuous_imp_Cauchy_continuous: | |
| 2573 | fixes f :: "'a::metric_space \<Rightarrow> 'b::metric_space" | |
| 67091 | 2574 | shows "\<lbrakk>uniformly_continuous_on S f; Cauchy \<sigma>; \<And>n. (\<sigma> n) \<in> S\<rbrakk> \<Longrightarrow> Cauchy(f \<circ> \<sigma>)" | 
| 64287 | 2575 | by (simp add: uniformly_continuous_on_def Cauchy_def) meson | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 2576 | |
| 51526 | 2577 | lemma (in bounded_linear) isUCont: "isUCont f" | 
| 63546 | 2578 | unfolding isUCont_def dist_norm | 
| 51526 | 2579 | proof (intro allI impI) | 
| 63546 | 2580 | fix r :: real | 
| 2581 | assume r: "0 < r" | |
| 2582 | 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 | 2583 | using pos_bounded by blast | 
| 51526 | 2584 | show "\<exists>s>0. \<forall>x y. norm (x - y) < s \<longrightarrow> norm (f x - f y) < r" | 
| 2585 | proof (rule exI, safe) | |
| 56541 | 2586 | from r K show "0 < r / K" by simp | 
| 51526 | 2587 | next | 
| 2588 | fix x y :: 'a | |
| 2589 | assume xy: "norm (x - y) < r / K" | |
| 2590 | have "norm (f x - f y) = norm (f (x - y))" by (simp only: diff) | |
| 2591 | also have "\<dots> \<le> norm (x - y) * K" by (rule norm_le) | |
| 2592 | also from K xy have "\<dots> < r" by (simp only: pos_less_divide_eq) | |
| 2593 | finally show "norm (f x - f y) < r" . | |
| 2594 | qed | |
| 2595 | qed | |
| 2596 | ||
| 2597 | lemma (in bounded_linear) Cauchy: "Cauchy X \<Longrightarrow> Cauchy (\<lambda>n. f (X n))" | |
| 63546 | 2598 | by (rule isUCont [THEN isUCont_Cauchy]) | 
| 51526 | 2599 | |
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2600 | lemma LIM_less_bound: | 
| 51526 | 2601 | fixes f :: "real \<Rightarrow> real" | 
| 2602 |   assumes ev: "b < x" "\<forall> x' \<in> { b <..< x}. 0 \<le> f x'" and "isCont f x"
 | |
| 2603 | 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 | 2604 | proof (rule tendsto_lowerbound) | 
| 61973 | 2605 | show "(f \<longlongrightarrow> f x) (at_left x)" | 
| 60758 | 2606 | using \<open>isCont f x\<close> by (simp add: filterlim_at_split isCont_def) | 
| 51526 | 2607 | 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 | 2608 | using ev by (auto simp: eventually_at dist_real_def intro!: exI[of _ "x - b"]) | 
| 51526 | 2609 | qed simp | 
| 51471 | 2610 | |
| 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 | 2611 | |
| 60758 | 2612 | 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 | 2613 | |
| 
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 | 2614 | lemma nested_sequence_unique: | 
| 61969 | 2615 | 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" | 
| 2616 | 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 | 2617 | 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 | 2618 | 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 | 2619 | have "decseq g" unfolding decseq_Suc_iff by fact | 
| 63546 | 2620 | have "f n \<le> g 0" for n | 
| 2621 | proof - | |
| 2622 | from \<open>decseq g\<close> have "g n \<le> g 0" | |
| 2623 | by (rule decseqD) simp | |
| 2624 | with \<open>\<forall>n. f n \<le> g n\<close>[THEN spec, of n] show ?thesis | |
| 2625 | by auto | |
| 2626 | qed | |
| 61969 | 2627 | then obtain u where "f \<longlonglongrightarrow> u" "\<forall>i. f i \<le> u" | 
| 60758 | 2628 | using incseq_convergent[OF \<open>incseq f\<close>] by auto | 
| 63546 | 2629 | moreover have "f 0 \<le> g n" for n | 
| 2630 | proof - | |
| 60758 | 2631 | from \<open>incseq f\<close> have "f 0 \<le> f n" by (rule incseqD) simp | 
| 63546 | 2632 | with \<open>\<forall>n. f n \<le> g n\<close>[THEN spec, of n] show ?thesis | 
| 2633 | by simp | |
| 2634 | qed | |
| 61969 | 2635 | then obtain l where "g \<longlonglongrightarrow> l" "\<forall>i. l \<le> g i" | 
| 60758 | 2636 | using decseq_convergent[OF \<open>decseq g\<close>] by auto | 
| 61969 | 2637 | 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 | 2638 | 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 | 2639 | 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 | 2640 | |
| 
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 | 2641 | 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 | 2642 | 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 | 2643 | assumes [arith]: "a \<le> b" | 
| 63546 | 2644 | 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" | 
| 2645 | 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 | 2646 | 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 | 2647 | proof - | 
| 63040 | 2648 | define bisect where "bisect = | 
| 2649 | rec_nat (a, b) (\<lambda>n (x, y). if P x ((x+y) / 2) then ((x+y)/2, y) else (x, (x+y)/2))" | |
| 2650 | define l u where "l n = fst (bisect n)" and "u n = snd (bisect n)" 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 | 2651 | 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 | 2652 | 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 | 2653 | 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 | 2654 | |
| 63546 | 2655 | 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 | 2656 | |
| 61969 | 2657 | 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 | 2658 | proof (safe intro!: nested_sequence_unique) | 
| 63546 | 2659 | show "l n \<le> l (Suc n)" "u (Suc n) \<le> u n" for n | 
| 2660 | 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 | 2661 | next | 
| 63546 | 2662 | have "l n - u n = (a - b) / 2^n" for n | 
| 2663 | by (induct n) (auto simp: field_simps) | |
| 2664 | then show "(\<lambda>n. l n - u n) \<longlonglongrightarrow> 0" | |
| 2665 | 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 | 2666 | qed fact | 
| 63546 | 2667 | then obtain x where x: "\<And>n. l n \<le> x" "\<And>n. x \<le> u n" and "l \<longlonglongrightarrow> x" "u \<longlonglongrightarrow> x" | 
| 2668 | by auto | |
| 2669 | 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 | 2670 | 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 | 2671 | |
| 
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 | 2672 | 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 | 2673 | proof (rule ccontr) | 
| 60141 
833adf7db7d8
New material, mostly about limits. Consolidation.
 paulson <lp15@cam.ac.uk> parents: 
60017diff
changeset | 2674 | assume "\<not> P a b" | 
| 63546 | 2675 | have "\<not> P (l n) (u n)" for n | 
| 2676 | proof (induct n) | |
| 2677 | case 0 | |
| 2678 | then show ?case | |
| 2679 | by (simp add: \<open>\<not> P a b\<close>) | |
| 2680 | next | |
| 2681 | case (Suc n) | |
| 2682 | with trans[of "l n" "(l n + u n) / 2" "u n"] show ?case | |
| 2683 | by auto | |
| 2684 | 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 | 2685 | moreover | 
| 63546 | 2686 |     {
 | 
| 2687 | have "eventually (\<lambda>n. x - d / 2 < l n) sequentially" | |
| 61969 | 2688 | 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 | 2689 | moreover have "eventually (\<lambda>n. u n < x + d / 2) sequentially" | 
| 61969 | 2690 | 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 | 2691 | 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 | 2692 | proof eventually_elim | 
| 63546 | 2693 | 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 | 2694 | 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 | 2695 | with x show "P (l n) (u n)" by (rule d) | 
| 63546 | 2696 | qed | 
| 2697 | } | |
| 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 | 2698 | 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 | 2699 | 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 | 2700 | 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 | 2701 | |
| 
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 | 2702 | 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 | 2703 | proof (cases "a \<le> b", rule compactI) | 
| 63546 | 2704 | fix C | 
| 2705 |   assume C: "a \<le> b" "\<forall>t\<in>C. open t" "{a..b} \<subseteq> \<Union>C"
 | |
| 63040 | 2706 |   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 | 2707 |   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 | 2708 | 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 | 2709 | case (trans a b c) | 
| 63546 | 2710 |     then have *: "{a..c} = {a..b} \<union> {b..c}"
 | 
| 2711 | by auto | |
| 2712 | with trans obtain C1 C2 | |
| 2713 |       where "C1\<subseteq>C" "finite C1" "{a..b} \<subseteq> \<Union>C1" "C2\<subseteq>C" "finite C2" "{b..c} \<subseteq> \<Union>C2"
 | |
| 2714 | 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 | 2715 | 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 | 2716 | 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 | 2717 | 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 | 2718 | case (local x) | 
| 63546 | 2719 | with C have "x \<in> \<Union>C" by auto | 
| 2720 | with C(2) obtain c where "x \<in> c" "open c" "c \<in> C" | |
| 2721 | 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 | 2722 |     then obtain e where "0 < e" "{x - e <..< x + e} \<subseteq> c"
 | 
| 62101 | 2723 | by (auto simp: open_dist dist_real_def subset_eq Ball_def abs_less_iff) | 
| 60758 | 2724 | 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 | 2725 |       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 | 2726 | 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 | 2727 | 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 | 2728 | |
| 
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 | 2729 | |
| 57447 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 2730 | 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 | 2731 | 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 | 2732 |   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 | 2733 | 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 | 2734 |   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 | 2735 | proof - | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 2736 |   have S: "compact S" "S \<noteq> {}"
 | 
| 60758 | 2737 | 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 | 2738 | 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 | 2739 | 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 | 2740 | 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 | 2741 | 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 | 2742 | 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 | 2743 | 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 | 2744 |   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 | 2745 | 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 | 2746 | 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 | 2747 | by auto | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 2748 | qed | 
| 
87429bdecad5
import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
 hoelzl parents: 
57276diff
changeset | 2749 | |
| 60974 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 2750 | lemma open_Collect_positive: | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 2751 | fixes f :: "'a::topological_space \<Rightarrow> real" | 
| 63546 | 2752 | assumes f: "continuous_on s f" | 
| 2753 |   shows "\<exists>A. open A \<and> A \<inter> s = {x\<in>s. 0 < f x}"
 | |
| 2754 |   using continuous_on_open_invariant[THEN iffD1, OF f, rule_format, of "{0 <..}"]
 | |
| 2755 | 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 | 2756 | |
| 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 2757 | lemma open_Collect_less_Int: | 
| 67958 
732c0b059463
tuned proofs and generalized some lemmas about limits
 huffman parents: 
67950diff
changeset | 2758 | fixes f g :: "'a::topological_space \<Rightarrow> real" | 
| 63546 | 2759 | assumes f: "continuous_on s f" | 
| 2760 | and g: "continuous_on s g" | |
| 2761 |   shows "\<exists>A. open A \<and> A \<inter> s = {x\<in>s. f x < g x}"
 | |
| 2762 | 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 | 2763 | |
| 
6a6f15d8fbc4
New material and fixes related to the forthcoming Stone-Weierstrass development
 paulson <lp15@cam.ac.uk> parents: 
60758diff
changeset | 2764 | |
| 60758 | 2765 | 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 | 2766 | |
| 60758 | 2767 | 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 | 2768 | |
| 
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 | 2769 | 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 | 2770 | 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 | 2771 | 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 | 2772 | \<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 | 2773 |   using continuous_attains_sup[of "{a..b}" f]
 | 
| 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 | 2774 | by (auto simp add: continuous_at_imp_continuous_on Ball_def Bex_def) | 
| 
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 | 2775 | |
| 
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 | 2776 | 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 | 2777 | 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 | 2778 | 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 | 2779 | \<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 | 2780 |   using continuous_attains_inf[of "{a..b}" f]
 | 
| 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 | 2781 | by (auto simp add: continuous_at_imp_continuous_on Ball_def Bex_def) | 
| 
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 | 2782 | |
| 
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 | 2783 | 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 | 2784 | 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 | 2785 | 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 | 2786 | 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 | 2787 | |
| 
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 | 2788 | 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 | 2789 | 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 | 2790 | 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 | 2791 | \<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 | 2792 | 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 | 2793 | |
| 
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 | 2794 | (*HOL style here: object-level formulations*) | 
| 63546 | 2795 | lemma IVT_objl: | 
| 2796 | "(f a \<le> y \<and> y \<le> f b \<and> a \<le> b \<and> (\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x)) \<longrightarrow> | |
| 2797 | (\<exists>x. a \<le> x \<and> x \<le> b \<and> f x = y)" | |
| 2798 | for a y :: real | |
| 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 | 2799 | by (blast intro: IVT) | 
| 
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 | 2800 | |
| 63546 | 2801 | lemma IVT2_objl: | 
| 2802 | "(f b \<le> y \<and> y \<le> f a \<and> a \<le> b \<and> (\<forall>x. a \<le> x \<and> x \<le> b \<longrightarrow> isCont f x)) \<longrightarrow> | |
| 2803 | (\<exists>x. a \<le> x \<and> x \<le> b \<and> f x = y)" | |
| 2804 | for b y :: real | |
| 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 | 2805 | by (blast intro: IVT2) | 
| 
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 | 2806 | |
| 
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 | 2807 | 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 | 2808 | 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 | 2809 | 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 | 2810 | 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 | 2811 | (\<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 | 2812 | 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 | 2813 | 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 | 2814 | 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 | 2815 | 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 | 2816 | using isCont_eq_Lb[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 | 2817 | show ?thesis | 
| 
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 | 2818 | using IVT[of f L _ M] IVT2[of f L _ M] M L assms | 
| 
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 | 2819 | apply (rule_tac x="f L" in exI) | 
| 
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 | 2820 | apply (rule_tac x="f M" in exI) | 
| 
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 | 2821 | apply (cases "L \<le> M") | 
| 63546 | 2822 | apply simp | 
| 2823 | apply (metis order_trans) | |
| 2824 | apply simp | |
| 2825 | apply (metis order_trans) | |
| 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 | 2826 | done | 
| 
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 | 2827 | 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 | 2828 | |
| 
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 | 2829 | |
| 63546 | 2830 | 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 | 2831 | |
| 
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 | 2832 | 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 | 2833 | 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 | 2834 | assumes d: "0 < d" | 
| 63546 | 2835 | and inj: "\<forall>z. \<bar>z-x\<bar> \<le> d \<longrightarrow> g (f z) = z" | 
| 2836 | and cont: "\<forall>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 | 2837 | 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 | 2838 | proof - | 
| 63546 | 2839 | let ?A = "f (x - d)" | 
| 2840 | let ?B = "f (x + d)" | |
| 2841 |   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 | 2842 | |
| 
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 | 2843 | 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 | 2844 | 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 | 2845 | 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 | 2846 | 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 | 2847 | |
| 
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 | 2848 |   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 | 2849 | 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 | 2850 |   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 | 2851 | 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 | 2852 | 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 | 2853 | 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 | 2854 | 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 | 2855 |   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 | 2856 | 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 | 2857 | ultimately | 
| 
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 | 2858 | show ?thesis | 
| 
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 | 2859 | 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 | 2860 | 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 | 2861 | |
| 
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 | 2862 | lemma isCont_inverse_function2: | 
| 63546 | 2863 | fixes f g :: "real \<Rightarrow> real" | 
| 2864 | shows | |
| 2865 | "a < x \<Longrightarrow> x < b \<Longrightarrow> | |
| 2866 | \<forall>z. a \<le> z \<and> z \<le> b \<longrightarrow> g (f z) = z \<Longrightarrow> | |
| 2867 | \<forall>z. a \<le> z \<and> z \<le> b \<longrightarrow> isCont f z \<Longrightarrow> isCont g (f x)" | |
| 2868 | apply (rule isCont_inverse_function [where f=f and d="min (x - a) (b - x)"]) | |
| 2869 | apply (simp_all add: abs_le_iff) | |
| 2870 | 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 | 2871 | |
| 66827 
c94531b5007d
Divided Topology_Euclidean_Space in two, creating new theory Connected. Also deleted some duplicate / variant theorems
 paulson <lp15@cam.ac.uk> parents: 
66793diff
changeset | 2872 | (* need to rename second continuous_at_inverse *) | 
| 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 | 2873 | lemma isCont_inv_fun: | 
| 
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 | 2874 | fixes f g :: "real \<Rightarrow> real" | 
| 63546 | 2875 | shows "0 < d \<Longrightarrow> (\<forall>z. \<bar>z - x\<bar> \<le> d \<longrightarrow> g (f z) = z) \<Longrightarrow> | 
| 2876 | \<forall>z. \<bar>z - x\<bar> \<le> d \<longrightarrow> isCont f z \<Longrightarrow> isCont g (f x)" | |
| 2877 | by (rule isCont_inverse_function) | |
| 2878 | ||
| 2879 | text \<open>Bartle/Sherbert: Introduction to Real Analysis, Theorem 4.2.9, p. 110.\<close> | |
| 2880 | 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)" | |
| 2881 | for f :: "real \<Rightarrow> real" | |
| 2882 | apply (drule (1) LIM_D) | |
| 2883 | apply clarify | |
| 2884 | apply (rule_tac x = s in exI) | |
| 2885 | apply (simp add: abs_less_iff) | |
| 2886 | done | |
| 2887 | ||
| 2888 | 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)" | |
| 2889 | for f :: "real \<Rightarrow> real" | |
| 2890 | apply (drule LIM_D [where r="-l"]) | |
| 2891 | apply simp | |
| 2892 | apply clarify | |
| 2893 | apply (rule_tac x = s in exI) | |
| 2894 | apply (simp add: abs_less_iff) | |
| 2895 | done | |
| 2896 | ||
| 2897 | 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)" | |
| 2898 | for f :: "real \<Rightarrow> real" | |
| 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 | 2899 | using LIM_fun_gt_zero[of f l c] LIM_fun_less_zero[of f l c] by (auto simp add: neq_iff) | 
| 51531 
f415febf4234
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
 hoelzl parents: 
51529diff
changeset | 2900 | |
| 31349 
2261c8781f73
new theory of filters and limits; prove LIMSEQ and LIM lemmas using filters
 huffman parents: diff
changeset | 2901 | end |