src/HOL/ex/BigO.thy
changeset 79566 f783490c6c99
parent 79559 cd9ede8488af
child 80914 d97fdabd9e2b
--- a/src/HOL/ex/BigO.thy	Wed Jan 31 22:36:12 2024 +0100
+++ b/src/HOL/ex/BigO.thy	Fri Feb 02 11:25:11 2024 +0000
@@ -49,7 +49,7 @@
 
 lemma bigo_elt_subset [intro]: "f \<in> O(g) \<Longrightarrow> O(f) \<le> O(g)"
   apply (auto simp add: bigo_alt_def)
-  by (metis (no_types, opaque_lifting) mult.assoc mult_le_cancel_iff2 order.trans
+  by (metis (no_types, opaque_lifting) mult.assoc mult_le_cancel_left_pos order.trans
       zero_less_mult_iff)
 
 lemma bigo_refl [intro]: "f \<in> O(f)"
@@ -77,7 +77,7 @@
   apply (rule conjI)
    apply (rule_tac x = "c + c" in exI)
    apply (clarsimp)
-  apply (smt (verit, ccfv_threshold) mult.commute abs_triangle_ineq add_le_cancel_left dual_order.trans mult.left_commute mult_2 mult_le_cancel_iff2)
+  apply (smt (verit, ccfv_threshold) mult.commute abs_triangle_ineq add_le_cancel_left dual_order.trans mult.left_commute mult_2 mult_le_cancel_left_pos)
   apply (simp add: order_less_le)
   apply (rule_tac x = "\<lambda>n. if \<bar>f n\<bar> < \<bar>g n\<bar> then x n else 0" in exI)
   apply (rule conjI)