src/HOL/Metis_Examples/Big_O.thy
changeset 59557 ebd8ecacfba6
parent 59554 4044f53326c9
child 59867 58043346ca64
--- a/src/HOL/Metis_Examples/Big_O.thy	Wed Feb 18 22:46:48 2015 +0100
+++ b/src/HOL/Metis_Examples/Big_O.thy	Thu Feb 19 11:53:36 2015 +0100
@@ -457,9 +457,9 @@
   hence F4: "\<exists>(u\<Colon>'a) SKF\<^sub>7\<Colon>'a \<Rightarrow> 'b. \<bar>g (SKF\<^sub>7 (\<bar>inverse c\<bar> * u))\<bar> \<le> u * \<bar>f (SKF\<^sub>7 (\<bar>inverse c\<bar> * u))\<bar> \<and> (0\<Colon>'a) \<le> \<bar>inverse c\<bar>"
     using F3 by metis
   hence "\<exists>(v\<Colon>'a) (u\<Colon>'a) SKF\<^sub>7\<Colon>'a \<Rightarrow> 'b. \<bar>inverse c\<bar> * \<bar>g (SKF\<^sub>7 (u * v))\<bar> \<le> u * (v * \<bar>f (SKF\<^sub>7 (u * v))\<bar>)"
-    by (metis comm_mult_left_mono)
+    by (metis mult_left_mono)
   thus "\<exists>ca\<Colon>'a. \<forall>x\<Colon>'b. \<bar>inverse c\<bar> * \<bar>g x\<bar> \<le> ca * \<bar>f x\<bar>"
-    using A2 F4 by (metis mult.assoc comm_mult_left_mono)
+    using A2 F4 by (metis mult.assoc mult_left_mono)
 qed
 
 lemma bigo_const_mult6 [intro]: "(\<lambda>x. c) *o O(f) <= O(f)"