Skip to content

Commit

Permalink
chore: fix docstring (#21027)
Browse files Browse the repository at this point in the history
  • Loading branch information
sgouezel committed Jan 24, 2025
1 parent 725eddc commit 59eed68
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean
Original file line number Diff line number Diff line change
Expand Up @@ -198,8 +198,8 @@ theorem ae_eq_of_integral_contDiff_smul_eq
(fun g g_diff g_supp ↦ h g g_diff.contDiff g_supp)

/-- If a function `f` locally integrable on an open subset `U` of a finite-dimensional real
manifold has zero integral when multiplied by any smooth function compactly supported
in an open set `U`, then `f` vanishes almost everywhere in `U`. -/
vector space has zero integral when multiplied by any smooth function compactly supported
in `U`, then `f` vanishes almost everywhere in `U`. -/
theorem IsOpen.ae_eq_zero_of_integral_contDiff_smul_eq_zero {U : Set E} (hU : IsOpen U)
(hf : LocallyIntegrableOn f U μ)
(h : ∀ (g : E → ℝ), ContDiff ℝ ∞ g → HasCompactSupport g → tsupport g ⊆ U →
Expand Down

0 comments on commit 59eed68

Please sign in to comment.