src/HOL/Topological_Spaces.thy
changeset 62381 a6479cb85944
parent 62369 acfc4ad7b76a
child 62397 5ae24f33d343
equal deleted inserted replaced
62379:340738057c8c 62381:a6479cb85944
   191 
   191 
   192 text \<open>A perfect space is a topological space with no isolated points.\<close>
   192 text \<open>A perfect space is a topological space with no isolated points.\<close>
   193 
   193 
   194 class perfect_space = topological_space +
   194 class perfect_space = topological_space +
   195   assumes not_open_singleton: "\<not> open {x}"
   195   assumes not_open_singleton: "\<not> open {x}"
       
   196 
       
   197 lemma UNIV_not_singleton: "UNIV \<noteq> {x::'a::perfect_space}"
       
   198   by (metis open_UNIV not_open_singleton)
   196 
   199 
   197 
   200 
   198 subsection \<open>Generators for toplogies\<close>
   201 subsection \<open>Generators for toplogies\<close>
   199 
   202 
   200 inductive generate_topology for S where
   203 inductive generate_topology for S where