Zulip Chat Archive
Stream: Is there code for X?
Topic: limits of measures on reals
Floris van Doorn (Jun 27 2024 at 10:23):
We have docs#MeasureTheory.tendsto_measure_iInter which shows that measures converge along countable limits in certain cases. Often you take a limit indexed by the real numbers which has a countable dense subset, which should be just as good. Do we have results in this direction in Mathlib? Here is an example that shows what I roughly want (though I'm not interested in this particular theorem) :
import Mathlib
open MeasureTheory Metric Topology
theorem tendsto_measure_ball_zero {α : Type*} [MeasurableSpace α] [MetricSpace α]
[BorelSpace α] [ProperSpace α]
{μ : Measure α} [IsFiniteMeasureOnCompacts μ] {x : α} :
Filter.Tendsto (fun r ↦ μ (ball x r)) (𝓝[>] 0) (𝓝 (μ {x})) := by sorry
Floris van Doorn (Jun 27 2024 at 10:33):
Ah, I found docs#MeasureTheory.tendsto_measure_biInter_gt . Perfect! @Leo Diedering: this will be useful for you.
Last updated: May 02 2025 at 03:31 UTC