Skip to content

Commit

Permalink
feat: on a countable type, if singletons are measurable the discrete …
Browse files Browse the repository at this point in the history
…topology is Borel (#8591)

Extracted from the PFR Project: teorth/pfr#67
  • Loading branch information
ocfnash committed Nov 24, 2023
1 parent 7efcade commit afce553
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean
Expand Up @@ -283,6 +283,12 @@ instance Subtype.borelSpace {α : Type*} [TopologicalSpace α] [MeasurableSpace
by borelize α; symm; apply borel_comap⟩
#align subtype.borel_space Subtype.borelSpace

instance Countable.instBorelSpace [Countable α] [MeasurableSpace α] [MeasurableSingletonClass α]
[TopologicalSpace α] [DiscreteTopology α] : BorelSpace α := by
have : ∀ s, @MeasurableSet α inferInstance s := fun s ↦ s.to_countable.measurableSet
have : ∀ s, @MeasurableSet α (borel α) s := fun s ↦ measurableSet_generateFrom (isOpen_discrete s)
exact ⟨by aesop⟩

instance Subtype.opensMeasurableSpace {α : Type*} [TopologicalSpace α] [MeasurableSpace α]
[h : OpensMeasurableSpace α] (s : Set α) : OpensMeasurableSpace s :=
by
Expand Down

0 comments on commit afce553

Please sign in to comment.