Zulip Chat Archive
Stream: new members
Topic: How do I show that Affine maps preserve measureable sets?
Toby Cathcart Burn (Apr 10 2025 at 15:00):
How should I prove that affine maps send measurable sets to measurable sets? Is this in mathlib, and should it be? I'm specifically interested in functions ℝ × ℝ → ℝ × ℝ .
measurableEmbedding_addRight
reduces this problem to showing that linear maps preserve measurable sets, but I can't find that in mathlib either.
Aaron Liu (Apr 10 2025 at 15:02):
Maybe docs#Continuous.measurable
Aaron Liu (Apr 10 2025 at 15:05):
We have docs#AffineMap.continuous_iff
Toby Cathcart Burn (Apr 10 2025 at 15:06):
Thanks, that looks great.
Aaron Liu (Apr 10 2025 at 15:15):
Maybe docs#AffineMap.continuous_linear_iff would be better
Toby Cathcart Burn (Apr 10 2025 at 15:31):
docs#Measurable talks about inverse images. Does this mean I need to get hold the inverse map (the cases I care about are invertible)?
Aaron Liu (Apr 10 2025 at 15:42):
Why would you need the inverse map?
Aaron Liu (Apr 10 2025 at 15:42):
Can you post the statement you want, written out in Lean?
Toby Cathcart Burn (Apr 10 2025 at 15:43):
theorem affine_Measurable (f : (ℝ × ℝ) →ᵃ[ℝ] (ℝ × ℝ)) {s : Set (ℝ×ℝ)} (h : MeasurableSet s ) : MeasurableSet (f '' s) := by
sorry
Aaron Liu (Apr 10 2025 at 15:46):
hmmm
Sébastien Gouëzel (Apr 10 2025 at 15:47):
This one is not true. There are measurable subsets of R^2 whose projection on R is not measurable. So taking f (x, y) = (x, 0)
, you get a counterexample to your statement. Preimages are much better behaved than direct images in many respects.
Toby Cathcart Burn (Apr 10 2025 at 15:52):
I hadn't realized the theorem wasn't true in general, thanks for pointing it out.
In this particular case, wouldn't the image of f always have measure 0 (as a subset of R^2)?
Sébastien Gouëzel (Apr 10 2025 at 15:57):
Sure. Here by measurable I mean Borel-measurable, which is the standard meaning in mathlib. It's true that the image is always Lebesgue measurable, but that's a deep theorem.
Toby Cathcart Burn (Apr 10 2025 at 16:05):
Thanks for explaining that. I guess I'll show that my affine maps have inverses. How would I find which kind of measure is the default? docs#Real.measureSpace doesn't have the most informative definition.
Toby Cathcart Burn (Apr 10 2025 at 16:14):
I've found docs#Real.measurableSpace. So MeasurableSet
(on R) means Borel measurable, but since volume
is defined on all subsets of R, it makes sense to extend it usefully by using the Lebesgue measure.
Etienne Marion (Apr 10 2025 at 16:17):
In Mathlib measures are always defined for any set as the biggest outer measure which coincides with the measure on measurable sets.
Last updated: May 02 2025 at 03:31 UTC