@@ -414,78 +414,117 @@ open scoped RealInnerProductSpace
414414
415415variable [FiniteDimensional β V]
416416
417- instance FourierTransform : FourierTransform (V β E) (V β E) where
418- fourierTransform f := VectorFourier.fourierIntegral π volume (innerβ V) f
417+ instance instFourierTransform : FourierTransform (V β E) (V β E) where
418+ fourier f := VectorFourier.fourierIntegral π volume (innerβ V) f
419419
420- instance FourierTransformInv : FourierTransformInv (V β E) (V β E) where
421- fourierTransformInv f w := VectorFourier.fourierIntegral π volume (-innerβ V) f w
420+ instance instFourierTransformInv : FourierTransformInv (V β E) (V β E) where
421+ fourierInv f w := VectorFourier.fourierIntegral π volume (-innerβ V) f w
422422
423423@[deprecated (since := "2025-11-12")]
424- alias fourierIntegral := FourierTransform.fourierTransform
424+ alias fourierIntegral := FourierTransform.fourier
425425
426426@[deprecated (since := "2025-11-12")]
427- alias fourierIntegralInv := FourierTransform.fourierTransformInv
427+ alias fourierIntegralInv := FourierTransform.fourierInv
428428
429- lemma fourierIntegral_eq (f : V β E) (w : V) :
429+ lemma fourier_eq (f : V β E) (w : V) :
430430 π f w = β« v, π (-βͺv, wβ«) β’ f v := rfl
431431
432- lemma fourierIntegral_eq' (f : V β E) (w : V) :
432+ @[deprecated (since := "2025-11-16")]
433+ alias fourierIntegral_eq := fourier_eq
434+
435+ lemma fourier_eq' (f : V β E) (w : V) :
433436 π f w = β« v, Complex.exp ((β(-2 * Ο * βͺv, wβ«) * Complex.I)) β’ f v := by
434- simp_rw [fourierIntegral_eq, Circle.smul_def, Real.fourierChar_apply, mul_neg, neg_mul]
437+ simp_rw [fourier_eq, Circle.smul_def, Real.fourierChar_apply, mul_neg, neg_mul]
438+
439+ @[deprecated (since := "2025-11-16")]
440+ alias fourierIntegral_eq' := fourier_eq'
435441
436- lemma fourierIntegralInv_eq (f : V β E) (w : V) :
442+ lemma fourierInv_eq (f : V β E) (w : V) :
437443 πβ» f w = β« v, π βͺv, wβ« β’ f v := by
438- simp [FourierTransformInv.fourierTransformInv , VectorFourier.fourierIntegral]
444+ simp [FourierTransformInv.fourierInv , VectorFourier.fourierIntegral]
439445
440- lemma fourierIntegralInv_eq' (f : V β E) (w : V) :
446+ @[deprecated (since := "2025-11-16")]
447+ alias fourierIntegralInv_eq := fourierInv_eq
448+
449+ lemma fourierInv_eq' (f : V β E) (w : V) :
441450 πβ» f w = β« v, Complex.exp ((β(2 * Ο * βͺv, wβ«) * Complex.I)) β’ f v := by
442- simp_rw [fourierIntegralInv_eq, Circle.smul_def, Real.fourierChar_apply]
451+ simp_rw [fourierInv_eq, Circle.smul_def, Real.fourierChar_apply]
452+
453+ @[deprecated (since := "2025-11-16")]
454+ alias fourierIntegralInv_eq' := fourierInv_eq'
443455
444- lemma fourierIntegral_comp_linearIsometry (A : W ββα΅’[β] V) (f : V β E) (w : W) :
456+ lemma fourier_comp_linearIsometry (A : W ββα΅’[β] V) (f : V β E) (w : W) :
445457 π (f β A) w = (π f) (A w) := by
446- simp only [fourierIntegral_eq , β A.inner_map_map, Function.comp_apply,
458+ simp only [fourier_eq , β A.inner_map_map, Function.comp_apply,
447459 β MeasurePreserving.integral_comp A.measurePreserving A.toHomeomorph.measurableEmbedding]
448460
449- lemma fourierIntegralInv_eq_fourierIntegral_neg (f : V β E) (w : V) :
461+ @[deprecated (since := "2025-11-16")]
462+ alias fourierIntegral_comp_linearIsometry := fourier_comp_linearIsometry
463+
464+ lemma fourierInv_eq_fourier_neg (f : V β E) (w : V) :
450465 πβ» f w = π f (-w) := by
451- simp [fourierIntegral_eq, fourierIntegralInv_eq]
466+ simp [fourier_eq, fourierInv_eq]
467+
468+ @[deprecated (since := "2025-11-16")]
469+ alias fourierIntegralInv_eq_fourierIntegral_neg := fourierInv_eq_fourier_neg
452470
453- lemma fourierIntegralInv_eq_fourierIntegral_comp_neg (f : V β E) :
471+ lemma fourierInv_eq_fourier_comp_neg (f : V β E) :
454472 πβ» f = π (fun x β¦ f (-x)) := by
455473 ext y
456- rw [fourierIntegralInv_eq_fourierIntegral_neg ]
474+ rw [fourierInv_eq_fourier_neg ]
457475 change π f (LinearIsometryEquiv.neg β y) = π (f β LinearIsometryEquiv.neg β) y
458- exact (fourierIntegral_comp_linearIsometry _ _ _).symm
476+ exact (fourier_comp_linearIsometry _ _ _).symm
477+
478+ @[deprecated (since := "2025-11-16")]
479+ alias fourierIntegralInv_eq_fourierIntegral_comp_neg := fourierInv_eq_fourier_comp_neg
459480
460- lemma fourierIntegralInv_comm (f : V β E) :
481+ lemma fourierInv_comm (f : V β E) :
461482 π (πβ» f) = πβ» (π f) := by
462- conv_rhs => rw [fourierIntegralInv_eq_fourierIntegral_comp_neg ]
463- simp_rw [β fourierIntegralInv_eq_fourierIntegral_neg ]
483+ conv_rhs => rw [fourierInv_eq_fourier_comp_neg ]
484+ simp_rw [β fourierInv_eq_fourier_neg ]
464485
465- lemma fourierIntegralInv_comp_linearIsometry (A : W ββα΅’[β] V) (f : V β E) (w : W) :
486+ @[deprecated (since := "2025-11-16")]
487+ alias fourierIntegralInv_comm := fourierInv_comm
488+
489+ lemma fourierInv_comp_linearIsometry (A : W ββα΅’[β] V) (f : V β E) (w : W) :
466490 πβ» (f β A) w = (πβ» f) (A w) := by
467- simp [fourierIntegralInv_eq_fourierIntegral_neg, fourierIntegral_comp_linearIsometry]
491+ simp [fourierInv_eq_fourier_neg, fourier_comp_linearIsometry]
492+
493+ @[deprecated (since := "2025-11-16")]
494+ alias fourierIntegralInv_comp_linearIsometry := fourierInv_comp_linearIsometry
468495
469- theorem fourierIntegral_real_eq (f : β β E) (w : β) :
496+ theorem fourier_real_eq (f : β β E) (w : β) :
470497 π f w = β« v : β, π (-(v * w)) β’ f v := by
471498 simp_rw [mul_comm _ w]
472499 rfl
473500
474- theorem fourierIntegral_real_eq_integral_exp_smul (f : β β E) (w : β) :
501+ @[deprecated (since := "2025-11-16")]
502+ alias fourierIntegral_real_eq := fourier_real_eq
503+
504+ theorem fourier_real_eq_integral_exp_smul (f : β β E) (w : β) :
475505 π f w = β« v : β, Complex.exp (β(-2 * Ο * v * w) * Complex.I) β’ f v := by
476- simp_rw [fourierIntegral_real_eq , Circle.smul_def, Real.fourierChar_apply, mul_neg, neg_mul,
506+ simp_rw [fourier_real_eq , Circle.smul_def, Real.fourierChar_apply, mul_neg, neg_mul,
477507 mul_assoc]
478508
479- theorem fourierIntegral_continuousLinearMap_apply
509+ @[deprecated (since := "2025-11-16")]
510+ alias fourierIntegral_real_eq_integral_exp_smul := fourier_real_eq_integral_exp_smul
511+
512+ theorem fourier_continuousLinearMap_apply
480513 {F : Type *} [NormedAddCommGroup F] [NormedSpace β F]
481514 {f : V β (F βL[β] E)} {a : F} {v : V} (hf : Integrable f) :
482515 π f v a = π (fun x β¦ f x a) v :=
483516 fourierIntegral_continuousLinearMap_apply' (L := innerSL β) hf
484517
485- theorem fourierIntegral_continuousMultilinearMap_apply {ΞΉ : Type *} [Fintype ΞΉ]
518+ @[deprecated (since := "2025-11-16")]
519+ alias fourierIntegral_continuousLinearMap_apply := fourier_continuousLinearMap_apply
520+
521+ theorem fourier_continuousMultilinearMap_apply {ΞΉ : Type *} [Fintype ΞΉ]
486522 {M : ΞΉ β Type *} [β i, NormedAddCommGroup (M i)] [β i, NormedSpace β (M i)]
487523 {f : V β ContinuousMultilinearMap β M E} {m : (i : ΞΉ) β M i} {v : V} (hf : Integrable f) :
488524 π f v m = π (fun x β¦ f x m) v :=
489525 fourierIntegral_continuousMultilinearMap_apply' (L := innerSL β) hf
490526
527+ @[deprecated (since := "2025-11-16")]
528+ alias fourierIntegral_continuousMultilinearMap_apply := fourier_continuousMultilinearMap_apply
529+
491530end Real
0 commit comments