Skip to content

Commit

Permalink
Browse files Browse the repository at this point in the history
  • Loading branch information
Parcly-Taxel committed May 6, 2023
1 parent bc9db78 commit 3cef175
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 7 deletions.
6 changes: 3 additions & 3 deletions Mathlib/MeasureTheory/MeasurableSpace.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Mario Carneiro
! This file was ported from Lean 3 source module measure_theory.measurable_space
! leanprover-community/mathlib commit 9b2b58d6b14b895b2f375108e765cb47de71aebd
! leanprover-community/mathlib commit 3905fa80e62c0898131285baab35559fbc4e5cda
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -1616,7 +1616,7 @@ open Classical

/-- If a measurable space is countably generated, it admits a measurable injection
into the Cantor space `ℕ → Bool` (equipped with the product sigma algebra). -/
theorem measurable_injection_cantor_of_countablyGenerated [MeasurableSpace α]
theorem measurable_injection_nat_bool_of_countablyGenerated [MeasurableSpace α]
[h : CountablyGenerated α] [MeasurableSingletonClass α] :
∃ f : α → ℕ → Bool, Measurable f ∧ Function.Injective f := by
obtain ⟨b, bct, hb⟩ := h.IsCountablyGenerated
Expand Down Expand Up @@ -1647,7 +1647,7 @@ theorem measurable_injection_cantor_of_countablyGenerated [MeasurableSpace α]
specialize this {y} measurableSet_eq
simp only [mem_singleton, iff_true_iff] at this
exact this
#align measurable_space.measurable_injection_cantor_of_countably_generated MeasurableSpace.measurable_injection_cantor_of_countablyGenerated
#align measurable_space.measurable_injection_nat_bool_of_countably_generated MeasurableSpace.measurable_injection_nat_bool_of_countablyGenerated

end MeasurableSpace

Expand Down
6 changes: 2 additions & 4 deletions Mathlib/Topology/Perfect.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Felix Weilacher
! This file was ported from Lean 3 source module topology.perfect
! leanprover-community/mathlib commit 9b2b58d6b14b895b2f375108e765cb47de71aebd
! leanprover-community/mathlib commit 3905fa80e62c0898131285baab35559fbc4e5cda
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand All @@ -21,8 +21,6 @@ including a version of the Cantor-Bendixson Theorem.
* `Perfect C`: A set `C` is perfect, meaning it is closed and every point of it
is an accumulation point of itself.
* `Set.scheme β α`: A `β`-scheme on `α`, a collection of subsets of `α` indexed by `List β`.
Used to construct maps `(β → ℕ) → α` as limiting objects.
## Main Statements
Expand All @@ -32,7 +30,7 @@ including a version of the Cantor-Bendixson Theorem.
* `exists_countable_union_perfect_of_isClosed`: One version of the **Cantor-Bendixson Theorem**:
A closed set in a second countable space can be written as the union of a countable set and a
perfect set.
* `exists_nat_bool_injection`: A perfect nonempty set in a complete metric space
* `Perfect.exists_nat_bool_injection`: A perfect nonempty set in a complete metric space
admits an embedding from the Cantor space.
## Implementation Notes
Expand Down

0 comments on commit 3cef175

Please sign in to comment.