Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a8c97ed

Browse files
loefflerdsgouezel
andcommitted
feat(measure_theory/function/continuous_map_dense): compactly supported functions are dense in L^p (#18710)
We have already the fact that bounded continuous functions are dense in L^p. We refactor the proof to extract an approach that is common to bounded continuous functions and to compactly supported functions, to avoid code duplication as much as possible. We also give elementary versions of the statements (in the form: for all epsilon > 0, there exists g such that...) as they may be easier to use, and specialized versions for integrable functions. Co-authored-by: sgouezel <sebastien.gouezel@univ-rennes1.fr>
1 parent df5e993 commit a8c97ed

File tree

4 files changed

+415
-111
lines changed

4 files changed

+415
-111
lines changed

src/analysis/fourier/add_circle.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -263,7 +263,7 @@ lemma coe_fn_fourier_Lp (p : ℝ≥0∞) [fact (1 ≤ p)] (n : ℤ) :
263263
lemma span_fourier_Lp_closure_eq_top {p : ℝ≥0∞} [fact (1 ≤ p)] (hp : p ≠ ∞) :
264264
(span ℂ (range (@fourier_Lp T _ p _))).topological_closure = ⊤ :=
265265
begin
266-
convert (continuous_map.to_Lp_dense_range ℂ hp (@haar_add_circle T hT) ℂ
266+
convert (continuous_map.to_Lp_dense_range ℂ (@haar_add_circle T hT) hp
267267
).topological_closure_map_submodule (span_fourier_closure_eq_top),
268268
rw [map_span, range_comp],
269269
simp only [continuous_linear_map.coe_coe],

0 commit comments

Comments
 (0)