Commit 2024-12-18 10:57 2375546c

View on Github →

chore(Topology/Separation): split large file (#20031) This splits up the behemoth Mathlib.Topology.Separation.Basic (2700 lines) into 5 smaller files:

  • Mathlib.Topology.Separation.SeparatedNhds: auxiliary definitions of SeparatedNhds and HasSeparatingCover
  • Mathlib.Topology.Separation.Basic: T0, R0, T1 and R1 spaces
  • Mathlib.Topology.Separation.Hausdorff: T2 and T2.5 spaces
  • Mathlib.Topology.Separation.Regular: regular, normal, completely normal, T3-T5
  • Mathlib.Topology.Separation.Profinite: totally disconnected compact Hausdorff spaces are totally separated. It also moves Mathlib.Topology.CompletelyRegular and Mathlib.Topology.CountableSeparatingOn into the Separation directory. The only changes outside the files listed above are updating import lines. The only change to actual code is in Mathlib.Topology.Separation.Profinite, where I realised that we had two theorems asserting exactly the same thing, one under strictly more general typeclass hypotheses than the other (locally compact rather than compact spaces). So I made the less general theorem into a deprecated alias for the more general one.

Estimated changes

deleted theorem Continuous.ext_on
deleted theorem Continuous.limUnder_eq
deleted theorem Filter.limUnder_eq_iff
deleted theorem HasSeparatingCover.mono
deleted def HasSeparatingCover
deleted theorem IsCompact.inter
deleted theorem IsCompact.isClosed
deleted theorem Pi.isCompact_closure_iff
deleted theorem Pi.isCompact_iff
deleted theorem RegularSpace.inf
deleted theorem RegularSpace.of_hasBasis
deleted theorem SeparatedNhds.comm
deleted theorem SeparatedNhds.empty_left
deleted theorem SeparatedNhds.empty_right
deleted theorem SeparatedNhds.mono
deleted theorem SeparatedNhds.preimage
deleted theorem SeparatedNhds.symm
deleted theorem SeparatedNhds.union_left
deleted theorem SeparatedNhds.union_right
deleted def SeparatedNhds
deleted theorem Set.Finite.t2_separation
deleted theorem closed_nhds_basis
deleted theorem disjoint_nested_nhds
deleted theorem disjoint_nhdsSet_nhds
deleted theorem disjoint_nhdsSet_nhdsSet
deleted theorem disjoint_nhds_nhds
deleted theorem disjoint_nhds_nhdsSet
deleted theorem eqOn_closure₂'
deleted theorem eqOn_closure₂
deleted theorem eq_of_nhds_neBot
deleted theorem hasBasis_nhds_closure
deleted theorem hasBasis_opens_closure
deleted theorem isClosed_diagonal
deleted theorem isClosed_eq
deleted theorem isOpen_iff_ultrafilter'
deleted theorem isOpen_ne_fun
deleted theorem lift'_nhds_closure
deleted theorem limUnder_nhdsWithin_id
deleted theorem limUnder_nhds_id
deleted theorem lim_eq
deleted theorem lim_eq_iff
deleted theorem lim_nhds
deleted theorem lim_nhdsWithin
deleted theorem nhds_basis_clopen
deleted theorem normal_separation
deleted theorem pairwise_disjoint_nhds
deleted theorem regularSpace_TFAE
deleted theorem regularSpace_iInf
deleted theorem regularSpace_induced
deleted theorem regularSpace_sInf
deleted theorem separated_by_continuous
deleted theorem t2Quotient.compatible
deleted theorem t2Quotient.continuous_mk
deleted def t2Quotient.lift
deleted theorem t2Quotient.lift_mk
deleted def t2Quotient.mk
deleted theorem t2Quotient.mk_eq
deleted theorem t2Quotient.surjective_mk
deleted theorem t2Quotient.unique_lift
deleted def t2Quotient
deleted def t2Setoid
deleted theorem t2Space_antitone
deleted theorem t2Space_iff_disjoint_nhds
deleted theorem t2Space_iff_nhds
deleted theorem t2_iff_isClosed_diagonal
deleted theorem t2_iff_nhds
deleted theorem t2_iff_ultrafilter
deleted theorem t2_separation
deleted theorem t2_separation_nhds
deleted theorem tendsto_nhds_unique'
deleted theorem tendsto_nhds_unique
added theorem Continuous.ext_on
added theorem Continuous.limUnder_eq
added theorem Filter.limUnder_eq_iff
added theorem IsCompact.inter
added theorem IsCompact.isClosed
added theorem Pi.isCompact_iff
added theorem disjoint_nhds_nhds
added theorem eqOn_closure₂'
added theorem eqOn_closure₂
added theorem eq_of_nhds_neBot
added theorem isClosed_diagonal
added theorem isClosed_eq
added theorem isOpen_ne_fun
added theorem limUnder_nhdsWithin_id
added theorem limUnder_nhds_id
added theorem lim_eq
added theorem lim_eq_iff
added theorem lim_nhds
added theorem lim_nhdsWithin
added theorem pairwise_disjoint_nhds
added theorem t2Quotient.compatible
added def t2Quotient.lift
added theorem t2Quotient.lift_mk
added def t2Quotient.mk
added theorem t2Quotient.mk_eq
added theorem t2Quotient.unique_lift
added def t2Quotient
added def t2Setoid
added theorem t2Space_antitone
added theorem t2Space_iff_nhds
added theorem t2_iff_nhds
added theorem t2_iff_ultrafilter
added theorem t2_separation
added theorem t2_separation_nhds
added theorem tendsto_nhds_unique'
added theorem tendsto_nhds_unique
added theorem RegularSpace.inf
added theorem closed_nhds_basis
added theorem disjoint_nested_nhds
added theorem disjoint_nhdsSet_nhds
added theorem disjoint_nhds_nhdsSet
added theorem hasBasis_nhds_closure
added theorem hasBasis_opens_closure
added theorem lift'_nhds_closure
added theorem normal_separation
added theorem regularSpace_TFAE
added theorem regularSpace_iInf
added theorem regularSpace_induced
added theorem regularSpace_sInf