Zulip Chat Archive

Stream: Is there code for X?

Topic: Outer regularity of Hausdorff measure


Bhavik Mehta (Mar 17 2025 at 11:43):

Do we have a proof that the Hausdorff measure is outer regular (docs#MeasureTheory.Measure.OuterRegular)?

Aaron Liu (Mar 17 2025 at 12:00):

For docs#MeasureTheory.Measure.hausdorffMeasure, I don't think it is in general. Are you maybe thinking of a special case?

Bhavik Mehta (Mar 17 2025 at 12:10):

It's a pretty standard result as far as I can tell: https://math.stackexchange.com/questions/3632955/is-hausdorff-measure-regular, https://math.stackexchange.com/questions/128085/is-the-hausdorff-outer-measure-regular

Bhavik Mehta (Mar 17 2025 at 12:14):

It's also in standard textbooks on this, eg Falconer Geometry of Fractal Sets

Aaron Liu (Mar 17 2025 at 12:15):

I took a look at the stackexchange posts, these seem to be proving slightly different things.

Kalle Kytölä (Mar 17 2025 at 12:23):

I'm not aware of it exactly in that form, but I think results around docs#instHasOuterApproxClosedOfPseudoMetrizableSpace should hopefully be of some use. I see that the type classes don't match exactly, though: the above requires docs#PseudoMetrizableSpace whereas docs#MeasureTheory.Measure.hausdorffMeasure has docs#EMetricSpace. And local finiteness presumably needs to be used, too (I used this so far only for finite measures). [UPDATE: And maybe there are a few further steps, so after all these may not shorten a direct proof by a lot.]

Bhavik Mehta (Mar 17 2025 at 12:41):

Unfortunately I don't have local finiteness here either...

Aaron Liu (Mar 17 2025 at 14:30):

Bhavik Mehta said:

It's a pretty standard result as far as I can tell: https://math.stackexchange.com/questions/3632955/is-hausdorff-measure-regular, https://math.stackexchange.com/questions/128085/is-the-hausdorff-outer-measure-regular

I seem to have disproved it here?

import Mathlib

open MeasureTheory Measure

example : ¬(μH[0] : Measure ).OuterRegular := by
  intro h
  apply OuterRegular.outerRegular at h
  specialize h (measurableSet_singleton 0) 2
  rw [hausdorffMeasure_zero_singleton] at h
  specialize h (by norm_num)
  obtain U, hU, ho, h2 := h
  obtain h0 | hinf := hausdorffMeasure_zero_or_top zero_lt_one U
  · rw [hausdorffMeasure_real, ho.measure_zero_iff_eq_empty] at h0
    simp [h0] at hU
  · simp [hinf] at h2

Yaël Dillies (Mar 17 2025 at 14:39):

Yes, it won't be outer-regular according to the usual topology. You will need to take a topology where lower-dimensional sets are open

Bhavik Mehta (Mar 17 2025 at 15:46):

Aaron Liu said:

Bhavik Mehta said:

It's a pretty standard result as far as I can tell: https://math.stackexchange.com/questions/3632955/is-hausdorff-measure-regular, https://math.stackexchange.com/questions/128085/is-the-hausdorff-outer-measure-regular

I seem to have disproved it here?

import Mathlib

open MeasureTheory Measure

example : ¬(μH[0] : Measure ).OuterRegular := by
  intro h
  apply OuterRegular.outerRegular at h
  specialize h (measurableSet_singleton 0) 2
  rw [hausdorffMeasure_zero_singleton] at h
  specialize h (by norm_num)
  obtain U, hU, ho, h2 := h
  obtain h0 | hinf := hausdorffMeasure_zero_or_top zero_lt_one U
  · rw [hausdorffMeasure_real, ho.measure_zero_iff_eq_empty] at h0
    simp [h0] at hU
  · simp [hinf] at h2

Ah, I should have said that I can assume s > 0 :)

Bhavik Mehta (Mar 17 2025 at 16:18):

Ah, I instead need to weaken to Gdelta (in the usual topology) rather than open, that's what was missing

Bhavik Mehta (Mar 19 2025 at 06:23):

And now this result is sorry-free (it turned out I can allow s = 0 too!)

example {s : } (hs : 0  s) (E : Set X) :
     G : Set X, IsGδ G  E  G  μH[s] G = μH[s] E := by

Last updated: May 02 2025 at 03:31 UTC