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