src/HOL/Library/BigO.thy
changeset 19279 48b527d0331b
parent 17199 59c1bfc81d91
child 19736 d8d0f8f51d69
equal deleted inserted replaced
19278:4d762b77d319 19279:48b527d0331b
   580   apply (auto simp add: bigo_def)
   580   apply (auto simp add: bigo_def)
   581   apply (rule_tac x = "abs c" in exI)
   581   apply (rule_tac x = "abs c" in exI)
   582   apply (subst abs_of_nonneg) back back
   582   apply (subst abs_of_nonneg) back back
   583   apply (rule setsum_nonneg)
   583   apply (rule setsum_nonneg)
   584   apply force
   584   apply force
   585   apply (subst setsum_mult)
   585   apply (subst setsum_right_distrib)
   586   apply (rule allI)
   586   apply (rule allI)
   587   apply (rule order_trans)
   587   apply (rule order_trans)
   588   apply (rule setsum_abs)
   588   apply (rule setsum_abs)
   589   apply (rule setsum_mono)
   589   apply (rule setsum_mono)
   590   apply (rule order_trans)
   590   apply (rule order_trans)