src/HOL/Limits.thy
changeset 45294 3c5d3d286055
parent 45031 9583f2b56f85
child 45892 8dcf6692433f
equal deleted inserted replaced
45293:57def0b39696 45294:3c5d3d286055
   538   "(f ---> l) F \<longleftrightarrow> (\<forall>S. open S \<longrightarrow> l \<in> S \<longrightarrow> eventually (\<lambda>x. f x \<in> S) F)"
   538   "(f ---> l) F \<longleftrightarrow> (\<forall>S. open S \<longrightarrow> l \<in> S \<longrightarrow> eventually (\<lambda>x. f x \<in> S) F)"
   539 
   539 
   540 ML {*
   540 ML {*
   541 structure Tendsto_Intros = Named_Thms
   541 structure Tendsto_Intros = Named_Thms
   542 (
   542 (
   543   val name = "tendsto_intros"
   543   val name = @{binding tendsto_intros}
   544   val description = "introduction rules for tendsto"
   544   val description = "introduction rules for tendsto"
   545 )
   545 )
   546 *}
   546 *}
   547 
   547 
   548 setup Tendsto_Intros.setup
   548 setup Tendsto_Intros.setup