src/HOL/Limits.thy
changeset 68721 53ad5c01be3f
parent 68615 3ed4ff0b7ac4
child 68860 f443ec10447d
equal deleted inserted replaced
68720:1e1818612124 68721:53ad5c01be3f
  1314 lemma filterlim_uminus_at_top: "(LIM x F. f x :> at_top) \<longleftrightarrow> (LIM x F. - (f x) :: real :> at_bot)"
  1314 lemma filterlim_uminus_at_top: "(LIM x F. f x :> at_top) \<longleftrightarrow> (LIM x F. - (f x) :: real :> at_bot)"
  1315   using filterlim_compose[OF filterlim_uminus_at_bot_at_top, of f F]
  1315   using filterlim_compose[OF filterlim_uminus_at_bot_at_top, of f F]
  1316     and filterlim_compose[OF filterlim_uminus_at_top_at_bot, of "\<lambda>x. - f x" F]
  1316     and filterlim_compose[OF filterlim_uminus_at_top_at_bot, of "\<lambda>x. - f x" F]
  1317   by auto
  1317   by auto
  1318 
  1318 
       
  1319 lemma tendsto_at_botI_sequentially:
       
  1320   fixes f :: "real \<Rightarrow> 'b::first_countable_topology"
       
  1321   assumes *: "\<And>X. filterlim X at_bot sequentially \<Longrightarrow> (\<lambda>n. f (X n)) \<longlonglongrightarrow> y"
       
  1322   shows "(f \<longlongrightarrow> y) at_bot"
       
  1323   unfolding filterlim_at_bot_mirror
       
  1324 proof (rule tendsto_at_topI_sequentially)
       
  1325   fix X :: "nat \<Rightarrow> real" assume "filterlim X at_top sequentially"
       
  1326   thus "(\<lambda>n. f (-X n)) \<longlonglongrightarrow> y" by (intro *) (auto simp: filterlim_uminus_at_top)
       
  1327 qed
       
  1328 
  1319 lemma filterlim_at_infinity_imp_filterlim_at_top:
  1329 lemma filterlim_at_infinity_imp_filterlim_at_top:
  1320   assumes "filterlim (f :: 'a \<Rightarrow> real) at_infinity F"
  1330   assumes "filterlim (f :: 'a \<Rightarrow> real) at_infinity F"
  1321   assumes "eventually (\<lambda>x. f x > 0) F"
  1331   assumes "eventually (\<lambda>x. f x > 0) F"
  1322   shows   "filterlim f at_top F"
  1332   shows   "filterlim f at_top F"
  1323 proof -
  1333 proof -