src/HOL/Limits.thy
changeset 36655 88f0125c3bd2
parent 36654 7c8eb32724ce
child 36656 fec55067ae9b
equal deleted inserted replaced
36654:7c8eb32724ce 36655:88f0125c3bd2
   583 
   583 
   584 lemma tendsto_ident_at [tendsto_intros]: "((\<lambda>x. x) ---> a) (at a)"
   584 lemma tendsto_ident_at [tendsto_intros]: "((\<lambda>x. x) ---> a) (at a)"
   585 unfolding tendsto_def eventually_at_topological by auto
   585 unfolding tendsto_def eventually_at_topological by auto
   586 
   586 
   587 lemma tendsto_ident_at_within [tendsto_intros]:
   587 lemma tendsto_ident_at_within [tendsto_intros]:
   588   "a \<in> S \<Longrightarrow> ((\<lambda>x. x) ---> a) (at a within S)"
   588   "((\<lambda>x. x) ---> a) (at a within S)"
   589 unfolding tendsto_def eventually_within eventually_at_topological by auto
   589 unfolding tendsto_def eventually_within eventually_at_topological by auto
   590 
   590 
   591 lemma tendsto_const [tendsto_intros]: "((\<lambda>x. k) ---> k) net"
   591 lemma tendsto_const [tendsto_intros]: "((\<lambda>x. k) ---> k) net"
   592 by (simp add: tendsto_def)
   592 by (simp add: tendsto_def)
   593 
   593