Skip to content

Commit e8f765e

Browse files
author
mathlib4-bot
committed
Merge remote-tracking branch 'origin/master' into bump/v4.22.0
2 parents cea177c + bb38781 commit e8f765e

File tree

37 files changed

+1287
-454
lines changed

37 files changed

+1287
-454
lines changed

Mathlib.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1799,6 +1799,8 @@ import Mathlib.Analysis.SpecialFunctions.Gaussian.FourierTransform
17991799
import Mathlib.Analysis.SpecialFunctions.Gaussian.GaussianIntegral
18001800
import Mathlib.Analysis.SpecialFunctions.Gaussian.PoissonSummation
18011801
import Mathlib.Analysis.SpecialFunctions.ImproperIntegrals
1802+
import Mathlib.Analysis.SpecialFunctions.Integrability.Basic
1803+
import Mathlib.Analysis.SpecialFunctions.Integrability.LogMeromorphic
18021804
import Mathlib.Analysis.SpecialFunctions.Integrals
18031805
import Mathlib.Analysis.SpecialFunctions.JapaneseBracket
18041806
import Mathlib.Analysis.SpecialFunctions.Log.Base
@@ -4249,6 +4251,7 @@ import Mathlib.MeasureTheory.Function.Floor
42494251
import Mathlib.MeasureTheory.Function.Holder
42504252
import Mathlib.MeasureTheory.Function.Intersectivity
42514253
import Mathlib.MeasureTheory.Function.Jacobian
4254+
import Mathlib.MeasureTheory.Function.JacobianOneDim
42524255
import Mathlib.MeasureTheory.Function.L1Space.AEEqFun
42534256
import Mathlib.MeasureTheory.Function.L1Space.HasFiniteIntegral
42544257
import Mathlib.MeasureTheory.Function.L1Space.Integrable

Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -986,7 +986,7 @@ theorem HasFTaylorSeriesUpToOn.comp {n : WithTop ℕ∞} {g : F → G} {f : E
986986
have B : HasFDerivWithinAt (fun x ↦ (q (f x)).taylorComp (p x) m)
987987
(∑ c : OrderedFinpartition m, ∑ i : Option (Fin c.length),
988988
((q (f x)).compAlongOrderedFinpartition (p x) (c.extend i)).curryLeft) s x :=
989-
HasFDerivWithinAt.sum (fun c _ ↦ A c)
989+
HasFDerivWithinAt.fun_sum (fun c _ ↦ A c)
990990
suffices ∑ c : OrderedFinpartition m, ∑ i : Option (Fin c.length),
991991
((q (f x)).compAlongOrderedFinpartition (p x) (c.extend i)) =
992992
(q (f x)).taylorComp (p x) (m + 1) by

Mathlib/Analysis/Calculus/ContDiff/Operations.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -282,7 +282,7 @@ theorem iteratedFDerivWithin_neg_apply {f : E → F} (hu : UniqueDiffOn 𝕜 s)
282282
_ = fderivWithin 𝕜 (-iteratedFDerivWithin 𝕜 i f s) s x (h 0) (Fin.tail h) := by
283283
rw [fderivWithin_congr' (@hi) hx]; rfl
284284
_ = -(fderivWithin 𝕜 (iteratedFDerivWithin 𝕜 i f s) s) x (h 0) (Fin.tail h) := by
285-
rw [Pi.neg_def, fderivWithin_neg (hu x hx)]; rfl
285+
rw [fderivWithin_neg (hu x hx)]; rfl
286286
_ = -(iteratedFDerivWithin 𝕜 (i + 1) f s) x h := rfl
287287

288288
theorem iteratedFDeriv_neg_apply {i : ℕ} {f : E → F} :

Mathlib/Analysis/Calculus/Deriv/Add.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -175,11 +175,11 @@ variable {ι : Type*} {u : Finset ι} {A : ι → 𝕜 → F} {A' : ι → F}
175175

176176
theorem HasDerivAtFilter.sum (h : ∀ i ∈ u, HasDerivAtFilter (A i) (A' i) x L) :
177177
HasDerivAtFilter (fun y => ∑ i ∈ u, A i y) (∑ i ∈ u, A' i) x L := by
178-
simpa [ContinuousLinearMap.sum_apply] using (HasFDerivAtFilter.sum h).hasDerivAtFilter
178+
simpa [ContinuousLinearMap.sum_apply] using (HasFDerivAtFilter.fun_sum h).hasDerivAtFilter
179179

180180
theorem HasStrictDerivAt.sum (h : ∀ i ∈ u, HasStrictDerivAt (A i) (A' i) x) :
181181
HasStrictDerivAt (fun y => ∑ i ∈ u, A i y) (∑ i ∈ u, A' i) x := by
182-
simpa [ContinuousLinearMap.sum_apply] using (HasStrictFDerivAt.sum h).hasStrictDerivAt
182+
simpa [ContinuousLinearMap.sum_apply] using (HasStrictFDerivAt.fun_sum h).hasStrictDerivAt
183183

184184
theorem HasDerivWithinAt.sum (h : ∀ i ∈ u, HasDerivWithinAt (A i) (A' i) s x) :
185185
HasDerivWithinAt (fun y => ∑ i ∈ u, A i y) (∑ i ∈ u, A' i) s x :=
@@ -221,11 +221,11 @@ nonrec theorem HasStrictDerivAt.neg (h : HasStrictDerivAt f f' x) :
221221

222222
theorem derivWithin.neg : derivWithin (fun y => -f y) s x = -derivWithin f s x := by
223223
by_cases hsx : UniqueDiffWithinAt 𝕜 s x
224-
· simp only [derivWithin, fderivWithin_neg hsx, ContinuousLinearMap.neg_apply]
224+
· simp only [derivWithin, fderivWithin_fun_neg hsx, ContinuousLinearMap.neg_apply]
225225
· simp [derivWithin_zero_of_not_uniqueDiffWithinAt hsx]
226226

227227
theorem deriv.neg : deriv (fun y => -f y) x = -deriv f x := by
228-
simp only [deriv, fderiv_neg, ContinuousLinearMap.neg_apply]
228+
simp only [deriv, fderiv_fun_neg, ContinuousLinearMap.neg_apply]
229229

230230
@[simp]
231231
theorem deriv.neg' : (deriv fun y => -f y) = fun x => -deriv f x :=
@@ -310,7 +310,7 @@ theorem HasStrictDerivAt.sub (hf : HasStrictDerivAt f f' x) (hg : HasStrictDeriv
310310
theorem derivWithin_sub (hf : DifferentiableWithinAt 𝕜 f s x)
311311
(hg : DifferentiableWithinAt 𝕜 g s x) :
312312
derivWithin (fun y => f y - g y) s x = derivWithin f s x - derivWithin g s x := by
313-
simp only [sub_eq_add_neg, derivWithin_add hf hg.neg, derivWithin.neg]
313+
simp only [sub_eq_add_neg, derivWithin_add hf hg.fun_neg, derivWithin.neg]
314314

315315
@[simp]
316316
theorem deriv_sub (hf : DifferentiableAt 𝕜 f x) (hg : DifferentiableAt 𝕜 g x) :

0 commit comments

Comments
 (0)