src/HOL/Quotient_Examples/Quotient_Rat.thy
changeset 64240 eabf80376aab
parent 61076 bdc1e2f0a86a
child 64290 fb5c74a58796
--- a/src/HOL/Quotient_Examples/Quotient_Rat.thy	Sun Oct 16 09:31:03 2016 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_Rat.thy	Sun Oct 16 09:31:04 2016 +0200
@@ -258,7 +258,7 @@
     fix a b :: int
     assume "b \<noteq> 0"
     then have "a * b \<le> (a div b + 1) * b * b"
-      by (metis mult.commute div_mult_self1_is_id less_int_def linorder_le_cases zdiv_mono1 zdiv_mono1_neg zle_add1_eq_le)
+      by (metis mult.commute nonzero_mult_div_cancel_left less_int_def linorder_le_cases zdiv_mono1 zdiv_mono1_neg zle_add1_eq_le)
     then show "\<exists>z::int. a * b \<le> z * b * b" by auto
   qed
 qed