Skip to content

Commit f191832

Browse files
james18lpcurkud
andcommitted
chore: Rename eventually_of_forall to Eventually.of_forall (#15444)
… and `frequently_of_forall` to `Frequently.of_forall` Co-authored-by: Yael Dillies <yael.dillies@gmail.com> Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
1 parent 355dce7 commit f191832

File tree

187 files changed

+512
-508
lines changed

Some content is hidden

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

187 files changed

+512
-508
lines changed

Counterexamples/Phillips.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -132,7 +132,7 @@ def boundedIntegrableFunctionsIntegralCLM [MeasurableSpace α] (μ : Measure α)
132132
intro f
133133
rw [mul_comm]
134134
apply norm_integral_le_of_norm_le_const
135-
apply Filter.eventually_of_forall
135+
apply Filter.Eventually.of_forall
136136
intro x
137137
exact BoundedContinuousFunction.norm_coe_le_norm f.1 x)
138138

@@ -434,7 +434,7 @@ theorem toFunctions_toMeasure [MeasurableSpace α] (μ : Measure α) [IsFiniteMe
434434
have : Integrable (fun _ => (1 : ℝ)) μ := integrable_const (1 : ℝ)
435435
apply
436436
this.mono' (Measurable.indicator (@measurable_const _ _ _ _ (1 : ℝ)) hs).aestronglyMeasurable
437-
apply Filter.eventually_of_forall
437+
apply Filter.Eventually.of_forall
438438
exact norm_indicator_le_one _
439439

440440
theorem toFunctions_toMeasure_continuousPart [MeasurableSpace α] [MeasurableSingletonClass α]

Mathlib/Analysis/Analytic/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -330,7 +330,7 @@ theorem radius_le_radius_continuousLinearMap_comp (p : FormalMultilinearSeries
330330
apply le_radius_of_isBigO
331331
apply (IsBigO.trans_isLittleO _ (p.isLittleO_one_of_lt_radius hr)).isBigO
332332
refine IsBigO.mul (@IsBigOWith.isBigO _ _ _ _ _ ‖f‖ _ _ _ ?_) (isBigO_refl _ _)
333-
refine IsBigOWith.of_bound (eventually_of_forall fun n => ?_)
333+
refine IsBigOWith.of_bound (Eventually.of_forall fun n => ?_)
334334
simpa only [norm_norm] using f.norm_compContinuousMultilinearMap_le (p n)
335335

336336
end FormalMultilinearSeries
@@ -829,7 +829,7 @@ theorem HasFPowerSeriesOnBall.tendstoLocallyUniformlyOn' (hf : HasFPowerSeriesOn
829829
protected theorem HasFPowerSeriesOnBall.continuousOn (hf : HasFPowerSeriesOnBall f p x r) :
830830
ContinuousOn f (EMetric.ball x r) :=
831831
hf.tendstoLocallyUniformlyOn'.continuousOn <|
832-
eventually_of_forall fun n =>
832+
Eventually.of_forall fun n =>
833833
((p.partialSum_continuous n).comp (continuous_id.sub continuous_const)).continuousOn
834834

835835
protected theorem HasFPowerSeriesAt.continuousAt (hf : HasFPowerSeriesAt f p x) :

Mathlib/Analysis/Analytic/Constructions.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -221,7 +221,7 @@ lemma formalMultilinearSeries_geometric_radius (𝕜) [NontriviallyNormedField
221221
simp_rw [IsLittleO, IsBigOWith, not_forall, norm_one, mul_one,
222222
not_eventually]
223223
refine ⟨1, one_pos, ?_⟩
224-
refine ((eventually_ne_atTop 0).mp (eventually_of_forall ?_)).frequently
224+
refine ((eventually_ne_atTop 0).mp (Eventually.of_forall ?_)).frequently
225225
intro n hn
226226
push_neg
227227
rwa [norm_pow, one_lt_pow_iff_of_nonneg (norm_nonneg _) hn,

Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -195,7 +195,7 @@ theorem isEquivalent_of_tendsto_one (hz : ∀ᶠ x in l, v x = 0 → u x = 0)
195195

196196
theorem isEquivalent_of_tendsto_one' (hz : ∀ x, v x = 0 → u x = 0) (huv : Tendsto (u / v) l (𝓝 1)) :
197197
u ~[l] v :=
198-
isEquivalent_of_tendsto_one (eventually_of_forall hz) huv
198+
isEquivalent_of_tendsto_one (Eventually.of_forall hz) huv
199199

200200
theorem isEquivalent_iff_tendsto_one (hz : ∀ᶠ x in l, v x ≠ 0) :
201201
u ~[l] v ↔ Tendsto (u / v) l (𝓝 1) := by

Mathlib/Analysis/Asymptotics/Asymptotics.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1077,7 +1077,7 @@ theorem isLittleO_principal {s : Set α} : f'' =o[𝓟 s] g' ↔ ∀ x ∈ s, f'
10771077
((continuous_id.mul continuous_const).tendsto' _ _ (zero_mul _)).mono_left
10781078
inf_le_left
10791079
apply le_of_tendsto_of_tendsto tendsto_const_nhds this
1080-
apply eventually_nhdsWithin_iff.2 (eventually_of_forall (fun c hc ↦ ?_))
1080+
apply eventually_nhdsWithin_iff.2 (Eventually.of_forall (fun c hc ↦ ?_))
10811081
exact eventually_principal.1 (h hc) x hx
10821082
· apply (isLittleO_zero g' _).congr' ?_ EventuallyEq.rfl
10831083
exact fun x hx ↦ (h x hx).symm
@@ -1564,11 +1564,11 @@ theorem isLittleO_iff_tendsto' {f g : α → 𝕜} (hgf : ∀ᶠ x in l, g x = 0
15641564
f =o[l] g ↔ Tendsto (fun x => f x / g x) l (𝓝 0) :=
15651565
⟨IsLittleO.tendsto_div_nhds_zero, fun h =>
15661566
(((isLittleO_one_iff _).mpr h).mul_isBigO (isBigO_refl g l)).congr'
1567-
(hgf.mono fun _x => div_mul_cancel_of_imp) (eventually_of_forall fun _x => one_mul _)⟩
1567+
(hgf.mono fun _x => div_mul_cancel_of_imp) (Eventually.of_forall fun _x => one_mul _)⟩
15681568

15691569
theorem isLittleO_iff_tendsto {f g : α → 𝕜} (hgf : ∀ x, g x = 0 → f x = 0) :
15701570
f =o[l] g ↔ Tendsto (fun x => f x / g x) l (𝓝 0) :=
1571-
isLittleO_iff_tendsto' (eventually_of_forall hgf)
1571+
isLittleO_iff_tendsto' (Eventually.of_forall hgf)
15721572

15731573
alias ⟨_, isLittleO_of_tendsto'⟩ := isLittleO_iff_tendsto'
15741574

Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -159,15 +159,15 @@ theorem SuperpolynomialDecay.trans_eventually_abs_le (hf : SuperpolynomialDecay
159159
rw [superpolynomialDecay_iff_abs_tendsto_zero] at hf ⊢
160160
refine fun z =>
161161
tendsto_of_tendsto_of_tendsto_of_le_of_le' tendsto_const_nhds (hf z)
162-
(eventually_of_forall fun x => abs_nonneg _) (hfg.mono fun x hx => ?_)
162+
(Eventually.of_forall fun x => abs_nonneg _) (hfg.mono fun x hx => ?_)
163163
calc
164164
|k x ^ z * g x| = |k x ^ z| * |g x| := abs_mul (k x ^ z) (g x)
165165
_ ≤ |k x ^ z| * |f x| := by gcongr _ * ?_; exact hx
166166
_ = |k x ^ z * f x| := (abs_mul (k x ^ z) (f x)).symm
167167

168168
theorem SuperpolynomialDecay.trans_abs_le (hf : SuperpolynomialDecay l k f)
169169
(hfg : ∀ x, |g x| ≤ |f x|) : SuperpolynomialDecay l k g :=
170-
hf.trans_eventually_abs_le (eventually_of_forall hfg)
170+
hf.trans_eventually_abs_le (Eventually.of_forall hfg)
171171

172172
end LinearOrderedCommRing
173173

@@ -206,7 +206,7 @@ theorem superpolynomialDecay_iff_abs_isBoundedUnder (hk : Tendsto k l atTop) :
206206
zero_mul m ▸
207207
Tendsto.mul_const m ((tendsto_zero_iff_abs_tendsto_zero _).1 hk.inv_tendsto_atTop)
208208
refine
209-
tendsto_of_tendsto_of_tendsto_of_le_of_le' h1 h2 (eventually_of_forall fun x => abs_nonneg _)
209+
tendsto_of_tendsto_of_tendsto_of_le_of_le' h1 h2 (Eventually.of_forall fun x => abs_nonneg _)
210210
((eventually_map.1 hm).mp ?_)
211211
refine (hk.eventually_ne_atTop 0).mono fun x hk0 hx => ?_
212212
refine Eq.trans_le ?_ (mul_le_mul_of_nonneg_left hx <| abs_nonneg (k x)⁻¹)

Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -151,9 +151,9 @@ theorem subbox_induction_on' {p : Box ι → Prop} (I : Box ι)
151151
simpa [hJsub] using
152152
tendsto_const_nhds.div_atTop (tendsto_pow_atTop_atTop_of_one_lt _root_.one_lt_two)
153153
replace hJlz : Tendsto (fun m ↦ (J m).lower) atTop (𝓝[Icc I.lower I.upper] z) :=
154-
tendsto_nhdsWithin_of_tendsto_nhds_of_eventually_within _ hJlz (eventually_of_forall hJl_mem)
154+
tendsto_nhdsWithin_of_tendsto_nhds_of_eventually_within _ hJlz (Eventually.of_forall hJl_mem)
155155
replace hJuz : Tendsto (fun m ↦ (J m).upper) atTop (𝓝[Icc I.lower I.upper] z) :=
156-
tendsto_nhdsWithin_of_tendsto_nhds_of_eventually_within _ hJuz (eventually_of_forall hJu_mem)
156+
tendsto_nhdsWithin_of_tendsto_nhds_of_eventually_within _ hJuz (Eventually.of_forall hJu_mem)
157157
rcases H_nhds z (h0 ▸ hzJ 0) with ⟨U, hUz, hU⟩
158158
rcases (tendsto_lift'.1 (hJlz.Icc hJuz) U hUz).exists with ⟨m, hUm⟩
159159
exact hJp m (hU (J m) (hJle m) m (hzJ m) hUm (hJsub m))

Mathlib/Analysis/BoxIntegral/Integrability.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -294,7 +294,7 @@ theorem IntegrableOn.hasBoxIntegral [CompleteSpace E] {f : (ι → ℝ) → E} {
294294
integral_finset_biUnion π.boxes (fun J _ => J.measurableSet_coe) π.pairwiseDisjoint (hfgi _)]
295295
refine dist_sum_sum_le_of_le _ fun J hJ => ?_
296296
rw [dist_eq_norm, ← integral_sub (hfi _ J hJ) (hgi J hJ)]
297-
refine norm_integral_le_of_norm_le (hfgi _ J hJ) (eventually_of_forall fun x => ?_)
297+
refine norm_integral_le_of_norm_le (hfgi _ J hJ) (Eventually.of_forall fun x => ?_)
298298
exact hfg_mono x (hNx (π.tag J))
299299

300300
/-- If `f : ℝⁿ → E` is continuous on a rectangular box `I`, then it is Box integrable on `I`

Mathlib/Analysis/BoxIntegral/Partition/Filter.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -518,7 +518,7 @@ theorem eventually_isPartition (l : IntegrationParams) (I : Box ι) :
518518
∀ᶠ π in l.toFilteriUnion I ⊤, TaggedPrepartition.IsPartition π :=
519519
eventually_iSup.2 fun _ =>
520520
eventually_inf_principal.2 <|
521-
eventually_of_forall fun π h =>
521+
Eventually.of_forall fun π h =>
522522
π.isPartition_iff_iUnion_eq.2 (h.trans Prepartition.iUnion_top)
523523

524524
end IntegrationParams

Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -85,16 +85,16 @@ nonrec theorem convolution_tendsto_right {ι} {φ : ι → ContDiffBump (0 : G)}
8585
(hig : ∀ᶠ i in l, AEStronglyMeasurable (g i) μ) (hcg : Tendsto (uncurry g) (l ×ˢ 𝓝 x₀) (𝓝 z₀))
8686
(hk : Tendsto k l (𝓝 x₀)) :
8787
Tendsto (fun i => ((φ i).normed μ ⋆[lsmul ℝ ℝ, μ] g i) (k i)) l (𝓝 z₀) :=
88-
convolution_tendsto_right (eventually_of_forall fun i => (φ i).nonneg_normed)
89-
(eventually_of_forall fun i => (φ i).integral_normed) (tendsto_support_normed_smallSets hφ) hig
88+
convolution_tendsto_right (Eventually.of_forall fun i => (φ i).nonneg_normed)
89+
(Eventually.of_forall fun i => (φ i).integral_normed) (tendsto_support_normed_smallSets hφ) hig
9090
hcg hk
9191

9292
/-- Special case of `ContDiffBump.convolution_tendsto_right` where `g` is continuous,
9393
and the limit is taken only in the first function. -/
9494
theorem convolution_tendsto_right_of_continuous {ι} {φ : ι → ContDiffBump (0 : G)} {l : Filter ι}
9595
(hφ : Tendsto (fun i => (φ i).rOut) l (𝓝 0)) (hg : Continuous g) (x₀ : G) :
9696
Tendsto (fun i => ((φ i).normed μ ⋆[lsmul ℝ ℝ, μ] g) x₀) l (𝓝 (g x₀)) :=
97-
convolution_tendsto_right hφ (eventually_of_forall fun _ => hg.aestronglyMeasurable)
97+
convolution_tendsto_right hφ (Eventually.of_forall fun _ => hg.aestronglyMeasurable)
9898
((hg.tendsto x₀).comp tendsto_snd) tendsto_const_nhds
9999

100100
/-- If a function `g` is locally integrable, then the convolution `φ i * g` converges almost
@@ -112,7 +112,7 @@ theorem ae_convolution_tendsto_right_of_locallyIntegrable
112112
filter_upwards [(Besicovitch.vitaliFamily μ).ae_tendsto_average_norm_sub hg] with x₀ h₀
113113
simp only [convolution_eq_swap, lsmul_apply]
114114
have hφ' : Tendsto (fun i ↦ (φ i).rOut) l (𝓝[>] 0) :=
115-
tendsto_nhdsWithin_iff.2 ⟨hφ, eventually_of_forall (fun i ↦ (φ i).rOut_pos)⟩
115+
tendsto_nhdsWithin_iff.2 ⟨hφ, Eventually.of_forall (fun i ↦ (φ i).rOut_pos)⟩
116116
have := (h₀.comp (Besicovitch.tendsto_filterAt μ x₀)).comp hφ'
117117
simp only [Function.comp] at this
118118
apply tendsto_integral_smul_of_tendsto_average_norm_sub (K ^ (FiniteDimensional.finrank ℝ G)) this

0 commit comments

Comments
 (0)