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

Commit a30c39e

Browse files
committed
feat(measure_theory/borel_space): a compact set has finite measure (#5628)
1 parent 4da8313 commit a30c39e

File tree

1 file changed

+11
-0
lines changed

1 file changed

+11
-0
lines changed

src/measure_theory/borel_space.lean

Lines changed: 11 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1238,3 +1238,14 @@ end regular
12381238

12391239
end measure
12401240
end measure_theory
1241+
1242+
lemma is_compact.measure_lt_top_of_nhds_within [topological_space α]
1243+
{s : set α} {μ : measure α} (h : is_compact s) (hμ : ∀ x ∈ s, μ.finite_at_filter (𝓝[s] x)) :
1244+
μ s < ⊤ :=
1245+
is_compact.induction_on h (by simp) (λ s t hst ht, (measure_mono hst).trans_lt ht)
1246+
(λ s t hs ht, (measure_union_le s t).trans_lt (ennreal.add_lt_top.2 ⟨hs, ht⟩)) hμ
1247+
1248+
lemma is_compact.measure_lt_top [topological_space α] {s : set α} {μ : measure α}
1249+
[locally_finite_measure μ] (h : is_compact s) :
1250+
μ s < ⊤ :=
1251+
h.measure_lt_top_of_nhds_within $ λ x hx, μ.finite_at_nhds_within _ _

0 commit comments

Comments
 (0)