Skip to content

Commit

Permalink
feat(Analysis/Distribution/SchwartzMap): pderiv equals lineDeriv (#9954)
Browse files Browse the repository at this point in the history
  • Loading branch information
mcdoll committed Feb 14, 2024
1 parent 088de1d commit 84a99a9
Showing 1 changed file with 5 additions and 2 deletions.
7 changes: 5 additions & 2 deletions Mathlib/Analysis/Distribution/SchwartzSpace.lean
Expand Up @@ -3,10 +3,9 @@ Copyright (c) 2022 Moritz Doll. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Moritz Doll
-/
import Mathlib.Analysis.Calculus.Deriv.Add
import Mathlib.Analysis.Calculus.Deriv.Mul
import Mathlib.Analysis.Calculus.ContDiff.Bounds
import Mathlib.Analysis.Calculus.IteratedDeriv.Defs
import Mathlib.Analysis.Calculus.LineDeriv.Basic
import Mathlib.Analysis.LocallyConvex.WithSeminorms
import Mathlib.Topology.Algebra.UniformFilterBasis
import Mathlib.Analysis.Normed.Group.ZeroAtInfty
Expand Down Expand Up @@ -946,6 +945,10 @@ theorem pderivCLM_apply (m : E) (f : 𝓒(E, F)) (x : E) : pderivCLM π•œ m f x
rfl
#align schwartz_map.pderiv_clm_apply SchwartzMap.pderivCLM_apply

theorem pderivCLM_eq_lineDeriv (m : E) (f : 𝓒(E, F)) (x : E) :
pderivCLM π•œ m f x = lineDeriv ℝ f x m := by
simp only [pderivCLM_apply, f.differentiableAt.lineDeriv_eq_fderiv]

/-- The iterated partial derivative (or directional derivative) as a continuous linear map on
Schwartz space. -/
def iteratedPDeriv {n : β„•} : (Fin n β†’ E) β†’ 𝓒(E, F) β†’L[π•œ] 𝓒(E, F) :=
Expand Down

0 comments on commit 84a99a9

Please sign in to comment.