Skip to content

Commit 188562f

Browse files
committed
chore: make MDifferentiableAt.mfderiv_prod an alias. (#31048)
It duplicates a lemma above, but having this name is nice for discoverability.
1 parent 150a1e4 commit 188562f

File tree

1 file changed

+2
-8
lines changed

1 file changed

+2
-8
lines changed

Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean

Lines changed: 2 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -633,14 +633,8 @@ theorem tangentMapWithin_prodSnd {s : Set (M × M')} {p : TangentBundle (I.prod
633633
@[deprecated (since := "2025-04-18")]
634634
alias tangentMapWithin_prod_snd := tangentMapWithin_prodSnd
635635

636-
theorem MDifferentiableAt.mfderiv_prod {f : M → M'} {g : M → M''} {x : M}
637-
(hf : MDifferentiableAt I I' f x) (hg : MDifferentiableAt I I'' g x) :
638-
mfderiv I (I'.prod I'') (fun x => (f x, g x)) x =
639-
(mfderiv I I' f x).prod (mfderiv I I'' g x) := by
640-
classical
641-
simp_rw [mfderiv, if_pos (hf.prodMk hg), if_pos hf, if_pos hg]
642-
exact hf.differentiableWithinAt_writtenInExtChartAt.fderivWithin_prodMk
643-
hg.differentiableWithinAt_writtenInExtChartAt (I.uniqueDiffOn _ (mem_range_self _))
636+
-- Kept as an alias for discoverability.
637+
alias MDifferentiableAt.mfderiv_prod := mfderiv_prodMk
644638

645639
theorem mfderiv_prod_left {x₀ : M} {y₀ : M'} :
646640
mfderiv I (I.prod I') (fun x => (x, y₀)) x₀ =

0 commit comments

Comments
 (0)