src/HOL/Library/Landau_Symbols.thy
changeset 75462 7448423e5dba
parent 74543 ee039c11fb6f
child 77200 8f2e6186408f
equal deleted inserted replaced
75461:4c3bc0d2568f 75462:7448423e5dba
   506   qed simp_all
   506   qed simp_all
   507 qed
   507 qed
   508 
   508 
   509 end
   509 end
   510 
   510 
       
   511 lemma summable_comparison_test_bigo:
       
   512   fixes f :: "nat \<Rightarrow> real"
       
   513   assumes "summable (\<lambda>n. norm (g n))" "f \<in> O(g)"
       
   514   shows   "summable f"
       
   515 proof -
       
   516   from \<open>f \<in> O(g)\<close> obtain C where C: "eventually (\<lambda>x. norm (f x) \<le> C * norm (g x)) at_top"
       
   517     by (auto elim: landau_o.bigE)
       
   518   thus ?thesis
       
   519     by (rule summable_comparison_test_ev) (insert assms, auto intro: summable_mult)
       
   520 qed
   511 
   521 
   512 lemma bigomega_iff_bigo: "g \<in> \<Omega>[F](f) \<longleftrightarrow> f \<in> O[F](g)"
   522 lemma bigomega_iff_bigo: "g \<in> \<Omega>[F](f) \<longleftrightarrow> f \<in> O[F](g)"
   513 proof
   523 proof
   514   assume "f \<in> O[F](g)"
   524   assume "f \<in> O[F](g)"
   515   then obtain c where "0 < c" "\<forall>\<^sub>F x in F. norm (f x) \<le> c * norm (g x)"
   525   then obtain c where "0 < c" "\<forall>\<^sub>F x in F. norm (f x) \<le> c * norm (g x)"