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

Commit c7a1319

Browse files
committed
feat(measure_theory/measure/measure_space): add interval_oc_ae_eq_interval (#14566)
1 parent 2c89306 commit c7a1319

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

src/measure_theory/measure/measure_space.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -2360,6 +2360,8 @@ lemma insert_ae_eq_self (a : α) (s : set α) :
23602360
(insert a s : set α) =ᵐ[μ] s :=
23612361
union_ae_eq_right.2 $ measure_mono_null (diff_subset _ _) (measure_singleton _)
23622362

2363+
section
2364+
23632365
variables [partial_order α] {a b : α}
23642366

23652367
lemma Iio_ae_eq_Iic : Iio a =ᵐ[μ] Iic a :=
@@ -2386,6 +2388,12 @@ Ico_ae_eq_Icc' (measure_singleton b)
23862388
lemma Ico_ae_eq_Ioc : Ico a b =ᵐ[μ] Ioc a b :=
23872389
Ico_ae_eq_Ioc' (measure_singleton a) (measure_singleton b)
23882390

2391+
end
2392+
2393+
open_locale interval
2394+
2395+
lemma interval_oc_ae_eq_interval [linear_order α] {a b : α} : Ι a b =ᵐ[μ] [a, b] := Ioc_ae_eq_Icc
2396+
23892397
end no_atoms
23902398

23912399
lemma ite_ae_eq_of_measure_zero {γ} (f : α → γ) (g : α → γ) (s : set α) (hs_zero : μ s = 0) :

0 commit comments

Comments
 (0)