src/HOL/Topological_Spaces.thy
changeset 63092 a949b2a5f51d
parent 63040 eb4ddd18d635
child 63170 eae6549dbea2
equal deleted inserted replaced
63091:54f16a0a3069 63092:a949b2a5f51d
  1365   unfolding at_within_def
  1365   unfolding at_within_def
  1366   by (intro sequentially_imp_eventually_nhds_within) auto
  1366   by (intro sequentially_imp_eventually_nhds_within) auto
  1367 
  1367 
  1368 lemma (in first_countable_topology) sequentially_imp_eventually_at:
  1368 lemma (in first_countable_topology) sequentially_imp_eventually_at:
  1369   "(\<forall>f. (\<forall>n. f n \<noteq> a) \<and> f \<longlonglongrightarrow> a \<longrightarrow> eventually (\<lambda>n. P (f n)) sequentially) \<Longrightarrow> eventually P (at a)"
  1369   "(\<forall>f. (\<forall>n. f n \<noteq> a) \<and> f \<longlonglongrightarrow> a \<longrightarrow> eventually (\<lambda>n. P (f n)) sequentially) \<Longrightarrow> eventually P (at a)"
  1370   using assms sequentially_imp_eventually_within [where s=UNIV] by simp
  1370   using sequentially_imp_eventually_within [where s=UNIV] by simp
  1371 
  1371 
  1372 lemma LIMSEQ_SEQ_conv1:
  1372 lemma LIMSEQ_SEQ_conv1:
  1373   fixes f :: "'a::topological_space \<Rightarrow> 'b::topological_space"
  1373   fixes f :: "'a::topological_space \<Rightarrow> 'b::topological_space"
  1374   assumes f: "f \<midarrow>a\<rightarrow> l"
  1374   assumes f: "f \<midarrow>a\<rightarrow> l"
  1375   shows "\<forall>S. (\<forall>n. S n \<noteq> a) \<and> S \<longlonglongrightarrow> a \<longrightarrow> (\<lambda>n. f (S n)) \<longlonglongrightarrow> l"
  1375   shows "\<forall>S. (\<forall>n. S n \<noteq> a) \<and> S \<longlonglongrightarrow> a \<longrightarrow> (\<lambda>n. f (S n)) \<longlonglongrightarrow> l"