src/HOL/Library/Landau_Symbols.thy
changeset 75462 7448423e5dba
parent 74543 ee039c11fb6f
child 77200 8f2e6186408f
--- a/src/HOL/Library/Landau_Symbols.thy	Mon May 23 17:21:57 2022 +0100
+++ b/src/HOL/Library/Landau_Symbols.thy	Tue May 24 16:21:49 2022 +0100
@@ -508,6 +508,16 @@
 
 end
 
+lemma summable_comparison_test_bigo:
+  fixes f :: "nat \<Rightarrow> real"
+  assumes "summable (\<lambda>n. norm (g n))" "f \<in> O(g)"
+  shows   "summable f"
+proof -
+  from \<open>f \<in> O(g)\<close> obtain C where C: "eventually (\<lambda>x. norm (f x) \<le> C * norm (g x)) at_top"
+    by (auto elim: landau_o.bigE)
+  thus ?thesis
+    by (rule summable_comparison_test_ev) (insert assms, auto intro: summable_mult)
+qed
 
 lemma bigomega_iff_bigo: "g \<in> \<Omega>[F](f) \<longleftrightarrow> f \<in> O[F](g)"
 proof