Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 7130d75

Browse files
committed
chore(*): introduce notation for left/right/punctured nhds (#10694)
New notation: * `𝓝[≤] x`: the filter `nhds_within x (set.Iic x)` of left-neighborhoods of `x`; * `𝓝[≥] x`: the filter `nhds_within x (set.Ici x)` of right-neighborhoods of `x`; * `𝓝[<] x`: the filter `nhds_within x (set.Iio x)` of punctured left-neighborhoods of `x`; * `𝓝[>] x`: the filter `nhds_within x (set.Ioi x)` of punctured right-neighborhoods of `x`; * `𝓝[≠] x`: the filter `nhds_within x {x}ᶜ` of punctured neighborhoods of `x`.
1 parent 6043522 commit 7130d75

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

45 files changed

+343
-333
lines changed

src/analysis/ODE/gronwall.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -106,7 +106,7 @@ See also `norm_le_gronwall_bound_of_norm_deriv_right_le` for a version bounding
106106
theorem le_gronwall_bound_of_liminf_deriv_right_le {f f' : ℝ → ℝ} {δ K ε : ℝ} {a b : ℝ}
107107
(hf : continuous_on f (Icc a b))
108108
(hf' : ∀ x ∈ Ico a b, ∀ r, f' x < r →
109-
∃ᶠ z in 𝓝[Ioi x] x, (z - x)⁻¹ * (f z - f x) < r)
109+
∃ᶠ z in 𝓝[>] x, (z - x)⁻¹ * (f z - f x) < r)
110110
(ha : f a ≤ δ) (bound : ∀ x ∈ Ico a b, f' x ≤ K * f x + ε) :
111111
∀ x ∈ Icc a b, f x ≤ gronwall_bound δ K ε (x - a) :=
112112
begin

src/analysis/analytic/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -358,7 +358,7 @@ lemma has_fpower_series_on_ball.mono
358358
⟨le_trans hr hf.1, r'_pos, λ y hy, hf.has_sum (emetric.ball_subset_ball hr hy)⟩
359359

360360
protected lemma has_fpower_series_at.eventually (hf : has_fpower_series_at f p x) :
361-
∀ᶠ r : ℝ≥0in 𝓝[Ioi 0] 0, has_fpower_series_on_ball f p x r :=
361+
∀ᶠ r : ℝ≥0in 𝓝[>] 0, has_fpower_series_on_ball f p x r :=
362362
let ⟨r, hr⟩ := hf in
363363
mem_of_superset (Ioo_mem_nhds_within_Ioi (left_mem_Ico.2 hr.r_pos)) $
364364
λ r' hr', hr.mono hr'.1 hr'.2.le

src/analysis/analytic/inverse.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -477,7 +477,7 @@ begin
477477
(𝓝 (r * (I + 1) * 0)) := tendsto_const_nhds.mul tendsto_id,
478478
have B : ∀ᶠ a in 𝓝 0, r * (I + 1) * a < 1/2,
479479
by { apply (tendsto_order.1 this).2, simp [zero_lt_one] },
480-
have C : ∀ᶠ a in 𝓝[set.Ioi (0 : ℝ)] (0 : ℝ), (0 : ℝ) < a,
480+
have C : ∀ᶠ a in 𝓝[>] (0 : ℝ), (0 : ℝ) < a,
481481
by { filter_upwards [self_mem_nhds_within], exact λ a ha, ha },
482482
rcases (C.and ((A.and B).filter_mono inf_le_left)).exists with ⟨a, ha⟩,
483483
exact ⟨a, ha.1, ha.2.1.le, ha.2.2.le⟩ },

src/analysis/asymptotics/asymptotics.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -755,7 +755,7 @@ begin
755755
refine ⟨_, λ h, (is_o_zero g' ⊤).congr (λ x, (h x).symm) (λ x, rfl)⟩,
756756
simp only [is_o_iff, eventually_top],
757757
refine λ h x, norm_le_zero_iff.1 _,
758-
have : tendsto (λ c : ℝ, c * ∥g' x∥) (𝓝[Ioi 0] 0) (𝓝 0) :=
758+
have : tendsto (λ c : ℝ, c * ∥g' x∥) (𝓝[>] 0) (𝓝 0) :=
759759
((continuous_id.mul continuous_const).tendsto' _ _ (zero_mul _)).mono_left inf_le_left,
760760
exact le_of_tendsto_of_tendsto tendsto_const_nhds this
761761
(eventually_nhds_within_iff.2 $ eventually_of_forall $ λ c hc, h hc x)

src/analysis/box_integral/divergence_theorem.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -170,7 +170,7 @@ begin
170170
`volume J ≤ (2 * δ) ^ (n + 1)` is small, and the difference of the integrals is small
171171
because each of the integrals is close to `volume (J.face i) • f x`.
172172
TODO: there should be a shorter and more readable way to formalize this simple proof. -/
173-
have : ∀ᶠ δ in 𝓝[Ioi 0] (0 : ℝ), δ ∈ Ioc (0 : ℝ) (1 / 2) ∧
173+
have : ∀ᶠ δ in 𝓝[>] (0 : ℝ), δ ∈ Ioc (0 : ℝ) (1 / 2) ∧
174174
(∀ y₁ y₂ ∈ closed_ball x δ ∩ I.Icc, ∥f y₁ - f y₂∥ ≤ ε / 2) ∧
175175
((2 * δ) ^ (n + 1) * ∥f' x (pi.single i 1)∥ ≤ ε / 2),
176176
{ refine eventually.and _ (eventually.and _ _),

src/analysis/calculus/deriv.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -275,7 +275,7 @@ end
275275

276276
lemma has_deriv_at_iff_tendsto_slope :
277277
has_deriv_at f f' x ↔
278-
tendsto (λ y, (y - x)⁻¹ • (f y - f x)) (𝓝[{x}ᶜ] x) (𝓝 f') :=
278+
tendsto (λ y, (y - x)⁻¹ • (f y - f x)) (𝓝[] x) (𝓝 f') :=
279279
has_deriv_at_filter_iff_tendsto_slope
280280

281281
theorem has_deriv_within_at_congr_set {s t u : set 𝕜}
@@ -1724,7 +1724,7 @@ lemma local_homeomorph.has_deriv_at_symm (f : local_homeomorph 𝕜 𝕜) {a f'
17241724
htff'.of_local_left_inverse (f.symm.continuous_at ha) hf' (f.eventually_right_inverse ha)
17251725

17261726
lemma has_deriv_at.eventually_ne (h : has_deriv_at f f' x) (hf' : f' ≠ 0) :
1727-
∀ᶠ z in 𝓝[{x}ᶜ] x, f z ≠ f x :=
1727+
∀ᶠ z in 𝓝[] x, f z ≠ f x :=
17281728
(has_deriv_at_iff_has_fderiv_at.1 h).eventually_ne
17291729
⟨∥f'∥⁻¹, λ z, by field_simp [norm_smul, mt norm_eq_zero.1 hf']⟩
17301730

@@ -2015,7 +2015,7 @@ lemma has_deriv_within_at.limsup_slope_le' (hf : has_deriv_within_at f f' s x)
20152015

20162016
lemma has_deriv_within_at.liminf_right_slope_le
20172017
(hf : has_deriv_within_at f f' (Ici x) x) (hr : f' < r) :
2018-
∃ᶠ z in 𝓝[Ioi x] x, (z - x)⁻¹ * (f z - f x) < r :=
2018+
∃ᶠ z in 𝓝[>] x, (z - x)⁻¹ * (f z - f x) < r :=
20192019
(hf.Ioi_of_Ici.limsup_slope_le' (lt_irrefl x) hr).frequently
20202020

20212021
end real
@@ -2072,7 +2072,7 @@ is less than or equal to `∥f'∥`. See also `has_deriv_within_at.limsup_norm_s
20722072
for a stronger version using limit superior and any set `s`. -/
20732073
lemma has_deriv_within_at.liminf_right_norm_slope_le
20742074
(hf : has_deriv_within_at f f' (Ici x) x) (hr : ∥f'∥ < r) :
2075-
∃ᶠ z in 𝓝[Ioi x] x, ∥z - x∥⁻¹ * ∥f z - f x∥ < r :=
2075+
∃ᶠ z in 𝓝[>] x, ∥z - x∥⁻¹ * ∥f z - f x∥ < r :=
20762076
(hf.Ioi_of_Ici.limsup_norm_slope_le hr).frequently
20772077

20782078
/-- If `f` has derivative `f'` within `(x, +∞)` at `x`, then for any `r > ∥f'∥` the ratio
@@ -2088,7 +2088,7 @@ See also
20882088
`∥f z - f x∥` instead of `∥f z∥ - ∥f x∥`. -/
20892089
lemma has_deriv_within_at.liminf_right_slope_norm_le
20902090
(hf : has_deriv_within_at f f' (Ici x) x) (hr : ∥f'∥ < r) :
2091-
∃ᶠ z in 𝓝[Ioi x] x, (z - x)⁻¹ * (∥f z∥ - ∥f x∥) < r :=
2091+
∃ᶠ z in 𝓝[>] x, (z - x)⁻¹ * (∥f z∥ - ∥f x∥) < r :=
20922092
begin
20932093
have := (hf.Ioi_of_Ici.limsup_slope_norm_le hr).frequently,
20942094
refine this.mp (eventually.mono self_mem_nhds_within _),

src/analysis/calculus/extend_deriv.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -99,8 +99,8 @@ end
9999
its derivative also converges at `a`, then `f` is differentiable on the right at `a`. -/
100100
lemma has_deriv_at_interval_left_endpoint_of_tendsto_deriv {s : set ℝ} {e : E} {a : ℝ} {f : ℝ → E}
101101
(f_diff : differentiable_on ℝ f s) (f_lim : continuous_within_at f s a)
102-
(hs : s ∈ 𝓝[Ioi a] a)
103-
(f_lim' : tendsto (λx, deriv f x) (𝓝[Ioi a] a) (𝓝 e)) :
102+
(hs : s ∈ 𝓝[>] a)
103+
(f_lim' : tendsto (λx, deriv f x) (𝓝[>] a) (𝓝 e)) :
104104
has_deriv_within_at f e (Ici a) a :=
105105
begin
106106
/- This is a specialization of `has_fderiv_at_boundary_of_tendsto_fderiv`. To be in the setting of
@@ -136,8 +136,8 @@ end
136136
its derivative also converges at `a`, then `f` is differentiable on the left at `a`. -/
137137
lemma has_deriv_at_interval_right_endpoint_of_tendsto_deriv {s : set ℝ} {e : E} {a : ℝ} {f : ℝ → E}
138138
(f_diff : differentiable_on ℝ f s) (f_lim : continuous_within_at f s a)
139-
(hs : s ∈ 𝓝[Iio a] a)
140-
(f_lim' : tendsto (λx, deriv f x) (𝓝[Iio a] a) (𝓝 e)) :
139+
(hs : s ∈ 𝓝[<] a)
140+
(f_lim' : tendsto (λx, deriv f x) (𝓝[<] a) (𝓝 e)) :
141141
has_deriv_within_at f e (Iic a) a :=
142142
begin
143143
/- This is a specialization of `has_fderiv_at_boundary_of_differentiable`. To be in the setting of
@@ -183,7 +183,7 @@ begin
183183
-- extension results.
184184
apply has_deriv_at_interval_left_endpoint_of_tendsto_deriv diff hf.continuous_within_at
185185
self_mem_nhds_within,
186-
have : tendsto g (𝓝[Ioi x] x) (𝓝 (g x)) := tendsto_inf_left hg,
186+
have : tendsto g (𝓝[>] x) (𝓝 (g x)) := tendsto_inf_left hg,
187187
apply this.congr' _,
188188
apply mem_of_superset self_mem_nhds_within (λy hy, _),
189189
exact (f_diff y (ne_of_gt hy)).deriv.symm },
@@ -194,7 +194,7 @@ begin
194194
-- extension results.
195195
apply has_deriv_at_interval_right_endpoint_of_tendsto_deriv diff hf.continuous_within_at
196196
self_mem_nhds_within,
197-
have : tendsto g (𝓝[Iio x] x) (𝓝 (g x)) := tendsto_inf_left hg,
197+
have : tendsto g (𝓝[<] x) (𝓝 (g x)) := tendsto_inf_left hg,
198198
apply this.congr' _,
199199
apply mem_of_superset self_mem_nhds_within (λy hy, _),
200200
exact (f_diff y (ne_of_lt hy)).deriv.symm },

src/analysis/calculus/fderiv.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2780,7 +2780,7 @@ begin
27802780
end
27812781

27822782
lemma has_fderiv_at.eventually_ne (h : has_fderiv_at f f' x) (hf' : ∃ C, ∀ z, ∥z∥ ≤ C * ∥f' z∥) :
2783-
∀ᶠ z in 𝓝[{x}ᶜ] x, f z ≠ f x :=
2783+
∀ᶠ z in 𝓝[] x, f z ≠ f x :=
27842784
by simpa only [compl_eq_univ_diff] using (has_fderiv_within_at_univ.2 h).eventually_ne hf'
27852785

27862786
end

src/analysis/calculus/fderiv_symmetric.lean

Lines changed: 9 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -70,7 +70,7 @@ This is a technical statement used to show that the second derivative is symmetr
7070
lemma convex.taylor_approx_two_segment
7171
{v w : E} (hv : x + v ∈ interior s) (hw : x + v + w ∈ interior s) :
7272
is_o (λ (h : ℝ), f (x + h • v + h • w) - f (x + h • v) - h • f' x w
73-
- h^2 • f'' v w - (h^2/2) • f'' w w) (λ h, h^2) (𝓝[Ioi (0 : ℝ)] 0) :=
73+
- h^2 • f'' v w - (h^2/2) • f'' w w) (λ h, h^2) (𝓝[>] (0 : ℝ)) :=
7474
begin
7575
-- it suffices to check that the expression is bounded by `ε * ((∥v∥ + ∥w∥) * ∥w∥) * h^2` for
7676
-- small enough `h`, for any positive `ε`.
@@ -79,12 +79,12 @@ begin
7979
-- good up to `δ`.
8080
rw [has_fderiv_within_at, has_fderiv_at_filter, is_o_iff] at hx,
8181
rcases metric.mem_nhds_within_iff.1 (hx εpos) with ⟨δ, δpos, sδ⟩,
82-
have E1 : ∀ᶠ h in 𝓝[Ioi (0:ℝ)] 0, h * (∥v∥ + ∥w∥) < δ,
83-
{ have : filter.tendsto (λ h, h * (∥v∥ + ∥w∥)) (𝓝[Ioi (0:ℝ)] 0) (𝓝 (0 * (∥v∥ + ∥w∥))) :=
82+
have E1 : ∀ᶠ h in 𝓝[>] (0:ℝ), h * (∥v∥ + ∥w∥) < δ,
83+
{ have : filter.tendsto (λ h, h * (∥v∥ + ∥w∥)) (𝓝[>] (0:ℝ)) (𝓝 (0 * (∥v∥ + ∥w∥))) :=
8484
(continuous_id.mul continuous_const).continuous_within_at,
8585
apply (tendsto_order.1 this).2 δ,
8686
simpa only [zero_mul] using δpos },
87-
have E2 : ∀ᶠ h in 𝓝[Ioi (0:ℝ)] 0, (h : ℝ) < 1 :=
87+
have E2 : ∀ᶠ h in 𝓝[>] (0:ℝ), (h : ℝ) < 1 :=
8888
mem_nhds_within_Ioi_iff_exists_Ioo_subset.2
8989
⟨(1 : ℝ), by simp only [mem_Ioi, zero_lt_one], λ x hx, hx.2⟩,
9090
filter_upwards [E1, E2, self_mem_nhds_within],
@@ -194,7 +194,7 @@ lemma convex.is_o_alternate_sum_square
194194
{v w : E} (h4v : x + (4 : ℝ) • v ∈ interior s) (h4w : x + (4 : ℝ) • w ∈ interior s) :
195195
is_o (λ (h : ℝ), f (x + h • (2 • v + 2 • w)) + f (x + h • (v + w))
196196
- f (x + h • (2 • v + w)) - f (x + h • (v + 2 • w)) - h^2 • f'' v w)
197-
(λ h, h^2) (𝓝[Ioi (0 : ℝ)] 0) :=
197+
(λ h, h^2) (𝓝[>] (0 : ℝ)) :=
198198
begin
199199
have A : (1 : ℝ)/2 ∈ Ioc (0 : ℝ) 1 := ⟨by norm_num, by norm_num⟩,
200200
have B : (1 : ℝ)/2 ∈ Icc (0 : ℝ) 1 := ⟨by norm_num, by norm_num⟩,
@@ -252,14 +252,14 @@ lemma convex.second_derivative_within_at_symmetric_of_mem_interior
252252
{v w : E} (h4v : x + (4 : ℝ) • v ∈ interior s) (h4w : x + (4 : ℝ) • w ∈ interior s) :
253253
f'' w v = f'' v w :=
254254
begin
255-
have A : is_o (λ (h : ℝ), h^2 • (f'' w v- f'' v w)) (λ h, h^2) (𝓝[Ioi (0 : ℝ)] 0),
255+
have A : is_o (λ (h : ℝ), h^2 • (f'' w v- f'' v w)) (λ h, h^2) (𝓝[>] (0 : ℝ)),
256256
{ convert (s_conv.is_o_alternate_sum_square hf xs hx h4v h4w).sub
257257
(s_conv.is_o_alternate_sum_square hf xs hx h4w h4v),
258258
ext h,
259259
simp only [add_comm, smul_add, smul_sub],
260260
abel },
261-
have B : is_o (λ (h : ℝ), f'' w v - f'' v w) (λ h, (1 : ℝ)) (𝓝[Ioi (0 : ℝ)] 0),
262-
{ have : is_O (λ (h : ℝ), 1/h^2) (λ h, 1/h^2) (𝓝[Ioi (0 : ℝ)] 0) := is_O_refl _ _,
261+
have B : is_o (λ (h : ℝ), f'' w v - f'' v w) (λ h, (1 : ℝ)) (𝓝[>] (0 : ℝ)),
262+
{ have : is_O (λ (h : ℝ), 1/h^2) (λ h, 1/h^2) (𝓝[>] (0 : ℝ)) := is_O_refl _ _,
263263
have C := this.smul_is_o A,
264264
apply C.congr' _ _,
265265
{ filter_upwards [self_mem_nhds_within],
@@ -298,7 +298,7 @@ begin
298298
refine tendsto_const_nhds.smul _,
299299
refine tendsto_const_nhds.add _,
300300
exact continuous_at_id.smul continuous_at_const },
301-
have B : ∀ (m : E), ∀ᶠ t in 𝓝[Ioi (0 : ℝ)] (0 : ℝ), x + (4 : ℝ) • (z + t • m) ∈ interior s,
301+
have B : ∀ (m : E), ∀ᶠ t in 𝓝[>] (0 : ℝ), x + (4 : ℝ) • (z + t • m) ∈ interior s,
302302
{ assume m,
303303
apply nhds_within_le_nhds,
304304
apply A m,

src/analysis/calculus/lhopital.lean

Lines changed: 37 additions & 37 deletions
Original file line numberDiff line numberDiff line change
@@ -47,14 +47,14 @@ include hab
4747
theorem lhopital_zero_right_on_Ioo
4848
(hff' : ∀ x ∈ Ioo a b, has_deriv_at f (f' x) x) (hgg' : ∀ x ∈ Ioo a b, has_deriv_at g (g' x) x)
4949
(hg' : ∀ x ∈ Ioo a b, g' x ≠ 0)
50-
(hfa : tendsto f (𝓝[Ioi a] a) (𝓝 0)) (hga : tendsto g (𝓝[Ioi a] a) (𝓝 0))
51-
(hdiv : tendsto (λ x, (f' x) / (g' x)) (𝓝[Ioi a] a) l) :
52-
tendsto (λ x, (f x) / (g x)) (𝓝[Ioi a] a) l :=
50+
(hfa : tendsto f (𝓝[>] a) (𝓝 0)) (hga : tendsto g (𝓝[>] a) (𝓝 0))
51+
(hdiv : tendsto (λ x, (f' x) / (g' x)) (𝓝[>] a) l) :
52+
tendsto (λ x, (f x) / (g x)) (𝓝[>] a) l :=
5353
begin
5454
have sub : ∀ x ∈ Ioo a b, Ioo a x ⊆ Ioo a b := λ x hx, Ioo_subset_Ioo (le_refl a) (le_of_lt hx.2),
5555
have hg : ∀ x ∈ (Ioo a b), g x ≠ 0,
5656
{ intros x hx h,
57-
have : tendsto g (𝓝[Iio x] x) (𝓝 0),
57+
have : tendsto g (𝓝[<] x) (𝓝 0),
5858
{ rw [← h, ← nhds_within_Ioo_eq_nhds_within_Iio hx.1],
5959
exact ((hgg' x hx).continuous_at.continuous_within_at.mono $ sub x hx).tendsto },
6060
obtain ⟨y, hyx, hy⟩ : ∃ c ∈ Ioo a x, g' c = 0,
@@ -220,9 +220,9 @@ include hab
220220

221221
theorem lhopital_zero_right_on_Ioo
222222
(hdf : differentiable_on ℝ f (Ioo a b)) (hg' : ∀ x ∈ Ioo a b, deriv g x ≠ 0)
223-
(hfa : tendsto f (𝓝[Ioi a] a) (𝓝 0)) (hga : tendsto g (𝓝[Ioi a] a) (𝓝 0))
224-
(hdiv : tendsto (λ x, ((deriv f) x) / ((deriv g) x)) (𝓝[Ioi a] a) l) :
225-
tendsto (λ x, (f x) / (g x)) (𝓝[Ioi a] a) l :=
223+
(hfa : tendsto f (𝓝[>] a) (𝓝 0)) (hga : tendsto g (𝓝[>] a) (𝓝 0))
224+
(hdiv : tendsto (λ x, ((deriv f) x) / ((deriv g) x)) (𝓝[>] a) l) :
225+
tendsto (λ x, (f x) / (g x)) (𝓝[>] a) l :=
226226
begin
227227
have hdf : ∀ x ∈ Ioo a b, differentiable_at ℝ f x,
228228
from λ x hx, (hdf x hx).differentiable_at (Ioo_mem_nhds hx.1 hx.2),
@@ -307,19 +307,19 @@ namespace has_deriv_at
307307

308308
/-- L'Hôpital's rule for approaching a real from the right, `has_deriv_at` version -/
309309
theorem lhopital_zero_nhds_right
310-
(hff' : ∀ᶠ x in 𝓝[Ioi a] a, has_deriv_at f (f' x) x)
311-
(hgg' : ∀ᶠ x in 𝓝[Ioi a] a, has_deriv_at g (g' x) x)
312-
(hg' : ∀ᶠ x in 𝓝[Ioi a] a, g' x ≠ 0)
313-
(hfa : tendsto f (𝓝[Ioi a] a) (𝓝 0)) (hga : tendsto g (𝓝[Ioi a] a) (𝓝 0))
314-
(hdiv : tendsto (λ x, (f' x) / (g' x)) (𝓝[Ioi a] a) l) :
315-
tendsto (λ x, (f x) / (g x)) (𝓝[Ioi a] a) l :=
310+
(hff' : ∀ᶠ x in 𝓝[>] a, has_deriv_at f (f' x) x)
311+
(hgg' : ∀ᶠ x in 𝓝[>] a, has_deriv_at g (g' x) x)
312+
(hg' : ∀ᶠ x in 𝓝[>] a, g' x ≠ 0)
313+
(hfa : tendsto f (𝓝[>] a) (𝓝 0)) (hga : tendsto g (𝓝[>] a) (𝓝 0))
314+
(hdiv : tendsto (λ x, (f' x) / (g' x)) (𝓝[>] a) l) :
315+
tendsto (λ x, (f x) / (g x)) (𝓝[>] a) l :=
316316
begin
317317
rw eventually_iff_exists_mem at *,
318318
rcases hff' with ⟨s₁, hs₁, hff'⟩,
319319
rcases hgg' with ⟨s₂, hs₂, hgg'⟩,
320320
rcases hg' with ⟨s₃, hs₃, hg'⟩,
321321
let s := s₁ ∩ s₂ ∩ s₃,
322-
have hs : s ∈ 𝓝[Ioi a] a := inter_mem (inter_mem hs₁ hs₂) hs₃,
322+
have hs : s ∈ 𝓝[>] a := inter_mem (inter_mem hs₁ hs₂) hs₃,
323323
rw mem_nhds_within_Ioi_iff_exists_Ioo_subset at hs,
324324
rcases hs with ⟨u, hau, hu⟩,
325325
refine lhopital_zero_right_on_Ioo hau _ _ _ hfa hga hdiv;
@@ -330,19 +330,19 @@ end
330330

331331
/-- L'Hôpital's rule for approaching a real from the left, `has_deriv_at` version -/
332332
theorem lhopital_zero_nhds_left
333-
(hff' : ∀ᶠ x in 𝓝[Iio a] a, has_deriv_at f (f' x) x)
334-
(hgg' : ∀ᶠ x in 𝓝[Iio a] a, has_deriv_at g (g' x) x)
335-
(hg' : ∀ᶠ x in 𝓝[Iio a] a, g' x ≠ 0)
336-
(hfa : tendsto f (𝓝[Iio a] a) (𝓝 0)) (hga : tendsto g (𝓝[Iio a] a) (𝓝 0))
337-
(hdiv : tendsto (λ x, (f' x) / (g' x)) (𝓝[Iio a] a) l) :
338-
tendsto (λ x, (f x) / (g x)) (𝓝[Iio a] a) l :=
333+
(hff' : ∀ᶠ x in 𝓝[<] a, has_deriv_at f (f' x) x)
334+
(hgg' : ∀ᶠ x in 𝓝[<] a, has_deriv_at g (g' x) x)
335+
(hg' : ∀ᶠ x in 𝓝[<] a, g' x ≠ 0)
336+
(hfa : tendsto f (𝓝[<] a) (𝓝 0)) (hga : tendsto g (𝓝[<] a) (𝓝 0))
337+
(hdiv : tendsto (λ x, (f' x) / (g' x)) (𝓝[<] a) l) :
338+
tendsto (λ x, (f x) / (g x)) (𝓝[<] a) l :=
339339
begin
340340
rw eventually_iff_exists_mem at *,
341341
rcases hff' with ⟨s₁, hs₁, hff'⟩,
342342
rcases hgg' with ⟨s₂, hs₂, hgg'⟩,
343343
rcases hg' with ⟨s₃, hs₃, hg'⟩,
344344
let s := s₁ ∩ s₂ ∩ s₃,
345-
have hs : s ∈ 𝓝[Iio a] a := inter_mem (inter_mem hs₁ hs₂) hs₃,
345+
have hs : s ∈ 𝓝[<] a := inter_mem (inter_mem hs₁ hs₂) hs₃,
346346
rw mem_nhds_within_Iio_iff_exists_Ioo_subset at hs,
347347
rcases hs with ⟨l, hal, hl⟩,
348348
refine lhopital_zero_left_on_Ioo hal _ _ _ hfa hga hdiv;
@@ -436,36 +436,36 @@ namespace deriv
436436

437437
/-- **L'Hôpital's rule** for approaching a real from the right, `deriv` version -/
438438
theorem lhopital_zero_nhds_right
439-
(hdf : ∀ᶠ x in 𝓝[Ioi a] a, differentiable_at ℝ f x)
440-
(hg' : ∀ᶠ x in 𝓝[Ioi a] a, deriv g x ≠ 0)
441-
(hfa : tendsto f (𝓝[Ioi a] a) (𝓝 0)) (hga : tendsto g (𝓝[Ioi a] a) (𝓝 0))
442-
(hdiv : tendsto (λ x, ((deriv f) x) / ((deriv g) x)) (𝓝[Ioi a] a) l) :
443-
tendsto (λ x, (f x) / (g x)) (𝓝[Ioi a] a) l :=
439+
(hdf : ∀ᶠ x in 𝓝[>] a, differentiable_at ℝ f x)
440+
(hg' : ∀ᶠ x in 𝓝[>] a, deriv g x ≠ 0)
441+
(hfa : tendsto f (𝓝[>] a) (𝓝 0)) (hga : tendsto g (𝓝[>] a) (𝓝 0))
442+
(hdiv : tendsto (λ x, ((deriv f) x) / ((deriv g) x)) (𝓝[>] a) l) :
443+
tendsto (λ x, (f x) / (g x)) (𝓝[>] a) l :=
444444
begin
445-
have hdg : ∀ᶠ x in 𝓝[Ioi a] a, differentiable_at ℝ g x,
445+
have hdg : ∀ᶠ x in 𝓝[>] a, differentiable_at ℝ g x,
446446
from hg'.mp (eventually_of_forall $
447447
λ _ hg', classical.by_contradiction (λ h, hg' (deriv_zero_of_not_differentiable_at h))),
448-
have hdf' : ∀ᶠ x in 𝓝[Ioi a] a, has_deriv_at f (deriv f x) x,
448+
have hdf' : ∀ᶠ x in 𝓝[>] a, has_deriv_at f (deriv f x) x,
449449
from hdf.mp (eventually_of_forall $ λ _, differentiable_at.has_deriv_at),
450-
have hdg' : ∀ᶠ x in 𝓝[Ioi a] a, has_deriv_at g (deriv g x) x,
450+
have hdg' : ∀ᶠ x in 𝓝[>] a, has_deriv_at g (deriv g x) x,
451451
from hdg.mp (eventually_of_forall $ λ _, differentiable_at.has_deriv_at),
452452
exact has_deriv_at.lhopital_zero_nhds_right hdf' hdg' hg' hfa hga hdiv
453453
end
454454

455455
/-- **L'Hôpital's rule** for approaching a real from the left, `deriv` version -/
456456
theorem lhopital_zero_nhds_left
457-
(hdf : ∀ᶠ x in 𝓝[Iio a] a, differentiable_at ℝ f x)
458-
(hg' : ∀ᶠ x in 𝓝[Iio a] a, deriv g x ≠ 0)
459-
(hfa : tendsto f (𝓝[Iio a] a) (𝓝 0)) (hga : tendsto g (𝓝[Iio a] a) (𝓝 0))
460-
(hdiv : tendsto (λ x, ((deriv f) x) / ((deriv g) x)) (𝓝[Iio a] a) l) :
461-
tendsto (λ x, (f x) / (g x)) (𝓝[Iio a] a) l :=
457+
(hdf : ∀ᶠ x in 𝓝[<] a, differentiable_at ℝ f x)
458+
(hg' : ∀ᶠ x in 𝓝[<] a, deriv g x ≠ 0)
459+
(hfa : tendsto f (𝓝[<] a) (𝓝 0)) (hga : tendsto g (𝓝[<] a) (𝓝 0))
460+
(hdiv : tendsto (λ x, ((deriv f) x) / ((deriv g) x)) (𝓝[<] a) l) :
461+
tendsto (λ x, (f x) / (g x)) (𝓝[<] a) l :=
462462
begin
463-
have hdg : ∀ᶠ x in 𝓝[Iio a] a, differentiable_at ℝ g x,
463+
have hdg : ∀ᶠ x in 𝓝[<] a, differentiable_at ℝ g x,
464464
from hg'.mp (eventually_of_forall $
465465
λ _ hg', classical.by_contradiction (λ h, hg' (deriv_zero_of_not_differentiable_at h))),
466-
have hdf' : ∀ᶠ x in 𝓝[Iio a] a, has_deriv_at f (deriv f x) x,
466+
have hdf' : ∀ᶠ x in 𝓝[<] a, has_deriv_at f (deriv f x) x,
467467
from hdf.mp (eventually_of_forall $ λ _, differentiable_at.has_deriv_at),
468-
have hdg' : ∀ᶠ x in 𝓝[Iio a] a, has_deriv_at g (deriv g x) x,
468+
have hdg' : ∀ᶠ x in 𝓝[<] a, has_deriv_at g (deriv g x) x,
469469
from hdg.mp (eventually_of_forall $ λ _, differentiable_at.has_deriv_at),
470470
exact has_deriv_at.lhopital_zero_nhds_left hdf' hdg' hg' hfa hga hdiv
471471
end

0 commit comments

Comments
 (0)