Skip to content

Commit 69e7283

Browse files
committed
feat: add more lemmas about derivatives and tsupport (#6228)
1 parent 358bd33 commit 69e7283

File tree

1 file changed

+19
-4
lines changed

1 file changed

+19
-4
lines changed

β€ŽMathlib/Analysis/Calculus/FDeriv/Basic.leanβ€Ž

Lines changed: 19 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1151,17 +1151,32 @@ end
11511151

11521152
/-! ### Support of derivatives -/
11531153

1154-
11551154
section Support
11561155

11571156
open Function
11581157

11591158
variable (π•œ : Type _) {E F : Type _} [NontriviallyNormedField π•œ] [NormedAddCommGroup E]
1160-
[NormedSpace π•œ E] [NormedAddCommGroup F] [NormedSpace π•œ F] {f : E β†’ F}
1159+
[NormedSpace π•œ E] [NormedAddCommGroup F] [NormedSpace π•œ F] {f : E β†’ F} {x : E}
1160+
1161+
theorem HasStrictFDerivAt.of_not_mem_tsupport (h : x βˆ‰ tsupport f) :
1162+
HasStrictFDerivAt f (0 : E β†’L[π•œ] F) x := by
1163+
rw [not_mem_tsupport_iff_eventuallyEq] at h
1164+
exact (hasStrictFDerivAt_const (0 : F) x).congr_of_eventuallyEq h.symm
1165+
1166+
theorem HasFDerivAt.of_not_mem_tsupport (h : x βˆ‰ tsupport f) :
1167+
HasFDerivAt f (0 : E β†’L[π•œ] F) x :=
1168+
(HasStrictFDerivAt.of_not_mem_tsupport π•œ h).hasFDerivAt
1169+
1170+
theorem HasFDerivWithinAt.of_not_mem_tsupport (h : x βˆ‰ tsupport f) :
1171+
HasFDerivWithinAt f (0 : E β†’L[π•œ] F) s x :=
1172+
(HasFDerivAt.of_not_mem_tsupport π•œ h).hasFDerivWithinAt
1173+
1174+
theorem fderiv_of_not_mem_tsupport (h : x βˆ‰ tsupport f) : fderiv π•œ f x = 0 :=
1175+
(HasFDerivAt.of_not_mem_tsupport π•œ h).fderiv
11611176

11621177
theorem support_fderiv_subset : support (fderiv π•œ f) βŠ† tsupport f := fun x ↦ by
1163-
rw [← not_imp_not, not_mem_tsupport_iff_eventuallyEq, nmem_support]
1164-
exact fun hx => hx.fderiv_eq.trans <| fderiv_const_apply 0
1178+
rw [← not_imp_not, nmem_support]
1179+
exact fderiv_of_not_mem_tsupport _
11651180
#align support_fderiv_subset support_fderiv_subset
11661181

11671182
theorem tsupport_fderiv_subset : tsupport (fderiv π•œ f) βŠ† tsupport f :=

0 commit comments

Comments
Β (0)