Skip to content

Commit fe1548c

Browse files
committed
chore(Normed/Operator): add smulRightL_apply_apply (#31642)
1 parent dbaa152 commit fe1548c

File tree

2 files changed

+6
-8
lines changed

2 files changed

+6
-8
lines changed

Mathlib/Analysis/Calculus/ParametricIntegral.lean

Lines changed: 1 addition & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -268,10 +268,7 @@ theorem hasDerivAt_integral_of_dominated_loc_of_lip {F' : α → E} (ε_pos : 0
268268
ε_pos hF_meas hF_int hm h_lipsch bound_integrable h_diff
269269
replace hF'_int : Integrable F' μ := by
270270
rw [← integrable_norm_iff hm] at hF'_int
271-
simpa only [L, (· ∘ ·), integrable_norm_iff, hF'_meas, one_mul, norm_one,
272-
ContinuousLinearMap.comp_apply, ContinuousLinearMap.coe_restrict_scalarsL',
273-
ContinuousLinearMap.norm_restrictScalars, ContinuousLinearMap.norm_smulRightL_apply] using
274-
hF'_int
271+
simpa [L, (· ∘ ·), integrable_norm_iff hF'_meas] using hF'_int
275272
refine ⟨hF'_int, ?_⟩
276273
by_cases hE : CompleteSpace E; swap
277274
· simpa [integral, hE] using hasDerivAt_const x₀ 0

Mathlib/Analysis/Normed/Operator/Bilinear.lean

Lines changed: 5 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -402,6 +402,7 @@ theorem nnnorm_smulRight_apply (c : StrongDual 𝕜 E) (f : Fₗ) : ‖smulRight
402402
variable (𝕜 E Fₗ) in
403403
/-- `ContinuousLinearMap.smulRight` as a continuous trilinear map:
404404
`smulRightL (c : StrongDual 𝕜 E) (f : F) (x : E) = c x • f`. -/
405+
@[simps! apply_apply]
405406
def smulRightL : StrongDual 𝕜 E →L[𝕜] Fₗ →L[𝕜] E →L[𝕜] Fₗ :=
406407
LinearMap.mkContinuous₂
407408
{ toFun := smulRightₗ
@@ -416,10 +417,10 @@ def smulRightL : StrongDual 𝕜 E →L[𝕜] Fₗ →L[𝕜] E →L[𝕜] Fₗ
416417
simp only [coe_smulRightₗ, one_mul, norm_smulRight_apply, LinearMap.coe_mk, AddHom.coe_mk,
417418
le_refl]
418419

419-
420-
@[simp]
421-
theorem norm_smulRightL_apply (c : StrongDual 𝕜 E) (f : Fₗ) : ‖smulRightL 𝕜 E Fₗ c f‖ = ‖c‖ * ‖f‖ :=
422-
norm_smulRight_apply c f
420+
@[deprecated norm_smulRight_apply (since := "2025-11-12")]
421+
theorem norm_smulRightL_apply (c : StrongDual 𝕜 E) (f : Fₗ) :
422+
‖smulRightL 𝕜 E Fₗ c f‖ = ‖c‖ * ‖f‖ := by
423+
simp
423424

424425
end ContinuousLinearMap
425426

0 commit comments

Comments
 (0)