src/HOL/Limits.thy
changeset 51360 c4367ed99b5e
parent 51328 d63ec23c9125
child 51471 cad22a3cc09c
--- a/src/HOL/Limits.thy	Wed Mar 06 16:10:56 2013 +0100
+++ b/src/HOL/Limits.thy	Wed Mar 06 16:56:21 2013 +0100
@@ -775,15 +775,24 @@
   tendsto :: "('b \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'b filter \<Rightarrow> bool" (infixr "--->" 55) where
   "(f ---> l) F \<equiv> filterlim f (nhds l) F"
 
+lemma tendsto_eq_rhs: "(f ---> x) F \<Longrightarrow> x = y \<Longrightarrow> (f ---> y) F"
+  by simp
+
 ML {*
+
 structure Tendsto_Intros = Named_Thms
 (
   val name = @{binding tendsto_intros}
   val description = "introduction rules for tendsto"
 )
+
 *}
 
-setup Tendsto_Intros.setup
+setup {*
+  Tendsto_Intros.setup #>
+  Global_Theory.add_thms_dynamic (@{binding tendsto_eq_intros},
+    map (fn thm => @{thm tendsto_eq_rhs} OF [thm]) o Tendsto_Intros.get o Context.proof_of);
+*}
 
 lemma tendsto_def: "(f ---> l) F \<longleftrightarrow> (\<forall>S. open S \<longrightarrow> l \<in> S \<longrightarrow> eventually (\<lambda>x. f x \<in> S) F)"
   unfolding filterlim_def