src/HOL/Analysis/Topology_Euclidean_Space.thy
changeset 68617 75129a73aca3
parent 68607 67bb59e49834
child 69000 7cb3ddd60fd6
--- a/src/HOL/Analysis/Topology_Euclidean_Space.thy	Wed Jul 11 23:24:25 2018 +0100
+++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy	Thu Jul 12 11:23:46 2018 +0200
@@ -603,7 +603,7 @@
 text \<open>Textbooks define Polish spaces as completely metrizable.
   We assume the topology to be complete for a given metric.\<close>
 
-class%important polish_space = complete_space + second_countable_topology
+class polish_space = complete_space + second_countable_topology
 
 subsection \<open>General notion of a topology as a value\<close>
 
@@ -4573,7 +4573,7 @@
   Heine-Borel property if every closed and bounded subset is compact.
 \<close>
 
-class%important heine_borel = metric_space +
+class heine_borel = metric_space +
   assumes bounded_imp_convergent_subsequence:
     "bounded (range f) \<Longrightarrow> \<exists>l r. strict_mono (r::nat\<Rightarrow>nat) \<and> ((f \<circ> r) \<longlongrightarrow> l) sequentially"