Skip to content

Commit

Permalink
feat: T2Space is Antitone (#18188)
Browse files Browse the repository at this point in the history
  • Loading branch information
scholzhannah committed Oct 24, 2024
1 parent 779f4ef commit 9d8ba93
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Topology/Separation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1892,6 +1892,10 @@ theorem not_preirreducible_nontrivial_t2 (X) [TopologicalSpace X] [Preirreducibl
[Nontrivial X] [T2Space X] : False :=
(PreirreducibleSpace.isPreirreducible_univ (X := X)).subsingleton.not_nontrivial nontrivial_univ

theorem t2Space_antitone {X : Type*} : Antitone (@T2Space X) :=
fun inst₁ inst₂ h_top h_t2 ↦ @T2Space.of_injective_continuous _ _ inst₁ inst₂
h_t2 _ Function.injective_id <| continuous_id_of_le h_top

end Separation

section RegularSpace
Expand Down

0 comments on commit 9d8ba93

Please sign in to comment.