Skip to content

Commit 468b507

Browse files
committed
feat: drop an assumption in mfderivWithin_const (#19936)
Followup to #19694
1 parent b09464f commit 468b507

File tree

2 files changed

+10
-3
lines changed

2 files changed

+10
-3
lines changed

Mathlib/Geometry/Manifold/MFDeriv/Basic.lean

Lines changed: 8 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -693,11 +693,18 @@ protected theorem MDifferentiableAt.mfderiv (h : MDifferentiableAt I I' f x) :
693693
protected theorem HasMFDerivAt.mfderiv (h : HasMFDerivAt I I' f x f') : mfderiv I I' f x = f' :=
694694
(hasMFDerivAt_unique h h.mdifferentiableAt.hasMFDerivAt).symm
695695

696-
theorem HasMFDerivWithinAt.mfderivWithin (h : HasMFDerivWithinAt I I' f s x f')
696+
protected theorem HasMFDerivWithinAt.mfderivWithin (h : HasMFDerivWithinAt I I' f s x f')
697697
(hxs : UniqueMDiffWithinAt I s x) : mfderivWithin I I' f s x = f' := by
698698
ext
699699
rw [hxs.eq h h.mdifferentiableWithinAt.hasMFDerivWithinAt]
700700

701+
theorem HasMFDerivWithinAt.mfderivWithin_eq_zero (h : HasMFDerivWithinAt I I' f s x 0) :
702+
mfderivWithin I I' f s x = 0 := by
703+
simp only [mfld_simps, mfderivWithin, h.mdifferentiableWithinAt, ↓reduceIte]
704+
simp only [HasMFDerivWithinAt, mfld_simps] at h
705+
rw [fderivWithin, if_pos]
706+
exact h.2
707+
701708
theorem MDifferentiable.mfderivWithin (h : MDifferentiableAt I I' f x)
702709
(hxs : UniqueMDiffWithinAt I s x) : mfderivWithin I I' f s x = mfderiv I I' f x := by
703710
apply HasMFDerivWithinAt.mfderivWithin _ hxs

Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -198,9 +198,9 @@ theorem mfderiv_const :
198198
mfderiv I I' (fun _ : M => c) x = (0 : TangentSpace I x →L[𝕜] TangentSpace I' c) :=
199199
HasMFDerivAt.mfderiv (hasMFDerivAt_const c x)
200200

201-
theorem mfderivWithin_const (hxs : UniqueMDiffWithinAt I s x) :
201+
theorem mfderivWithin_const :
202202
mfderivWithin I I' (fun _ : M => c) s x = (0 : TangentSpace I x →L[𝕜] TangentSpace I' c) :=
203-
(hasMFDerivWithinAt_const _ _ _).mfderivWithin hxs
203+
(hasMFDerivWithinAt_const _ _ _).mfderivWithin_eq_zero
204204

205205
end Const
206206

0 commit comments

Comments
 (0)