Skip to content

Commit 20c7b4b

Browse files
grunwegsgouezelurkud
committed
chore(Topology/Basic): re-use variables; rename a : X to x : X (#9993)
Co-authored-by: sgouezel <sebastien.gouezel@univ-rennes1.fr> Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
1 parent e3b6818 commit 20c7b4b

File tree

15 files changed

+334
-333
lines changed

15 files changed

+334
-333
lines changed

Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -141,10 +141,10 @@ theorem isEquivalent_const_iff_tendsto {c : β} (h : c ≠ 0) :
141141
u ~[l] const _ c ↔ Tendsto u l (𝓝 c) := by
142142
simp (config := { unfoldPartialApp := true }) only [IsEquivalent, const, isLittleO_const_iff h]
143143
constructor <;> intro h
144-
· have := h.sub (tendsto_const_nhds (a := -c))
144+
· have := h.sub (tendsto_const_nhds (x := -c))
145145
simp only [Pi.sub_apply, sub_neg_eq_add, sub_add_cancel, zero_add] at this
146146
exact this
147-
· have := h.sub (tendsto_const_nhds (a := c))
147+
· have := h.sub (tendsto_const_nhds (x := c))
148148
rwa [sub_self] at this
149149
#align asymptotics.is_equivalent_const_iff_tendsto Asymptotics.isEquivalent_const_iff_tendsto
150150

Mathlib/Analysis/Calculus/FDeriv/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -779,7 +779,7 @@ theorem HasFDerivAtFilter.tendsto_nhds (hL : L ≤ 𝓝 x) (h : HasFDerivAtFilte
779779
refine' h.isBigO_sub.trans_tendsto (Tendsto.mono_left _ hL)
780780
rw [← sub_self x]
781781
exact tendsto_id.sub tendsto_const_nhds
782-
have := this.add (@tendsto_const_nhds _ _ _ (f x) _)
782+
have := this.add (tendsto_const_nhds (x := f x))
783783
rw [zero_add (f x)] at this
784784
exact this.congr (by simp only [sub_add_cancel, eq_self_iff_true, forall_const])
785785
#align has_fderiv_at_filter.tendsto_nhds HasFDerivAtFilter.tendsto_nhds

Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -216,7 +216,7 @@ variable (f)
216216
theorem tendsto_integral_exp_inner_smul_cocompact :
217217
Tendsto (fun w : V => ∫ v, e[-⟪v, w⟫] • f v) (cocompact V) (𝓝 0) := by
218218
by_cases hfi : Integrable f; swap
219-
· convert tendsto_const_nhds (a := (0 : E)) with w
219+
· convert tendsto_const_nhds (x := (0 : E)) with w
220220
apply integral_undef
221221
rwa [← fourier_integrand_integrable w]
222222
refine' Metric.tendsto_nhds.mpr fun ε hε => _

Mathlib/Analysis/InnerProductSpace/Projection.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -172,10 +172,10 @@ theorem exists_norm_eq_iInf_of_complete_convex {K : Set F} (ne : K.Nonempty) (h
172172
convert this
173173
exact sqrt_zero.symm
174174
have eq₁ : Tendsto (fun n : ℕ => 8 * δ * (1 / (n + 1))) atTop (nhds (0 : ℝ)) := by
175-
convert (@tendsto_const_nhds _ _ _ (8 * δ) _).mul tendsto_one_div_add_atTop_nhds_0_nat
175+
convert (tendsto_const_nhds (x := 8 * δ)).mul tendsto_one_div_add_atTop_nhds_0_nat
176176
simp only [mul_zero]
177177
have : Tendsto (fun n : ℕ => (4 : ℝ) * (1 / (n + 1))) atTop (nhds (0 : ℝ)) := by
178-
convert (@tendsto_const_nhds _ _ _ (4 : ℝ) _).mul tendsto_one_div_add_atTop_nhds_0_nat
178+
convert (tendsto_const_nhds (x := 4)).mul tendsto_one_div_add_atTop_nhds_0_nat
179179
simp only [mul_zero]
180180
have eq₂ :
181181
Tendsto (fun n : ℕ => (4 : ℝ) * (1 / (n + 1)) * (1 / (n + 1))) atTop (nhds (0 : ℝ)) := by

Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1311,7 +1311,7 @@ instance completeSpace [CompleteSpace G] : CompleteSpace (ContinuousMultilinearM
13111311
map_smul' := fun v i c x => by
13121312
skip
13131313
have A := hF (Function.update v i (c • x))
1314-
have B := Filter.Tendsto.smul (@tendsto_const_nhds _ ℕ _ c _) (hF (Function.update v i x))
1314+
have B := Filter.Tendsto.smul (tendsto_const_nhds (x := c)) (hF (Function.update v i x))
13151315
simp? at A B says simp only [map_smul] at A B
13161316
exact tendsto_nhds_unique A B }
13171317
-- and that `F` has norm at most `(b 0 + ‖f 0‖)`.

Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -108,7 +108,7 @@ theorem tendsto_rpow_div_mul_add (a b c : ℝ) (hb : 0 ≠ b) :
108108
((tendsto_exp_nhds_0_nhds_1.comp
109109
(by
110110
simpa only [mul_zero, pow_one] using
111-
(@tendsto_const_nhds _ _ _ a _).mul
111+
(tendsto_const_nhds (x := a)).mul
112112
(tendsto_div_pow_mul_exp_add_atTop b c 1 hb))).comp
113113
tendsto_log_atTop)
114114
apply eventuallyEq_of_mem (Ioi_mem_atTop (0 : ℝ))

Mathlib/Topology/Algebra/Algebra.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -111,7 +111,7 @@ theorem Subalgebra.le_topologicalClosure (s : Subalgebra R A) : s ≤ s.topologi
111111
#align subalgebra.le_topological_closure Subalgebra.le_topologicalClosure
112112

113113
theorem Subalgebra.isClosed_topologicalClosure (s : Subalgebra R A) :
114-
IsClosed (s.topologicalClosure : Set A) := by convert @isClosed_closure A _ s
114+
IsClosed (s.topologicalClosure : Set A) := by convert @isClosed_closure A s _
115115
#align subalgebra.is_closed_topological_closure Subalgebra.isClosed_topologicalClosure
116116

117117
theorem Subalgebra.topologicalClosure_minimal (s : Subalgebra R A) {t : Subalgebra R A} (h : s ≤ t)

Mathlib/Topology/Algebra/Order/LiminfLimsup.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -183,7 +183,7 @@ set_option linter.uppercaseLean3 false in
183183

184184
theorem limsSup_nhds (a : α) : limsSup (𝓝 a) = a :=
185185
csInf_eq_of_forall_ge_of_forall_gt_exists_lt (isBounded_le_nhds a)
186-
(fun a' (h : { n : α | n ≤ a' } ∈ 𝓝 a) ↦ show a ≤ a' from @mem_of_mem_nhds α _ a _ h)
186+
(fun a' (h : { n : α | n ≤ a' } ∈ 𝓝 a) ↦ show a ≤ a' from @mem_of_mem_nhds α a _ _ h)
187187
fun b (hba : a < b) ↦
188188
show ∃ c, { n : α | n ≤ c } ∈ 𝓝 a ∧ c < b from
189189
match dense_or_discrete a b with

Mathlib/Topology/Bases.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -130,7 +130,7 @@ theorem isTopologicalBasis_of_isOpen_of_nhds {s : Set (Set α)} (h_open : ∀ u
130130
rcases h_nhds a univ trivial isOpen_univ with ⟨u, h₁, h₂, -⟩
131131
exact ⟨u, h₁, h₂⟩
132132
· refine' (le_generateFrom h_open).antisymm fun u hu => _
133-
refine' (@isOpen_iff_nhds α (generateFrom s) u).mpr fun a ha => _
133+
refine (@isOpen_iff_nhds α u (generateFrom s)).mpr fun a ha ↦ ?_
134134
rcases h_nhds a u ha hu with ⟨v, hvs, hav, hvu⟩
135135
rw [nhds_generateFrom]
136136
exact iInf₂_le_of_le v ⟨hav, hvs⟩ (le_principal_iff.2 hvu)

0 commit comments

Comments
 (0)