src/HOL/Library/Float.thy
changeset 30034 60f64f112174
parent 29988 747f0c519090
child 30122 1c912a9d8200
--- a/src/HOL/Library/Float.thy	Fri Feb 20 23:46:03 2009 +0100
+++ b/src/HOL/Library/Float.thy	Sat Feb 21 09:58:26 2009 +0100
@@ -795,7 +795,7 @@
     have "x \<noteq> y"
     proof (rule ccontr)
       assume "\<not> x \<noteq> y" hence "x = y" by auto
-      have "?X mod y = 0" unfolding `x = y` using zmod_zmult_self2 by auto
+      have "?X mod y = 0" unfolding `x = y` using mod_mult_self1_is_0 by auto
       thus False using False by auto
     qed
     hence "x < y" using `x \<le> y` by auto