src/HOL/Analysis/Topology_Euclidean_Space.thy
changeset 66304 cde6ceffcbc7
parent 66286 1c977b13414f
child 66408 46cfd348c373
--- a/src/HOL/Analysis/Topology_Euclidean_Space.thy	Tue Aug 01 17:30:02 2017 +0200
+++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy	Tue Aug 01 17:33:04 2017 +0200
@@ -5300,7 +5300,7 @@
   "compact (s :: 'a::metric_space set) \<longleftrightarrow> seq_compact s"
   using compact_imp_seq_compact seq_compact_imp_heine_borel by blast
 
-lemma compact_def: --\<open>this is the definition of compactness in HOL Light\<close>
+lemma compact_def: \<comment>\<open>this is the definition of compactness in HOL Light\<close>
   "compact (S :: 'a::metric_space set) \<longleftrightarrow>
    (\<forall>f. (\<forall>n. f n \<in> S) \<longrightarrow> (\<exists>l\<in>S. \<exists>r. subseq r \<and> (f \<circ> r) \<longlonglongrightarrow> l))"
   unfolding compact_eq_seq_compact_metric seq_compact_def by auto