src/HOL/Library/Fraction_Field.thy
changeset 53374 a14d2a854c02
parent 53196 942a1b48bb31
child 54230 b1d955791529
--- a/src/HOL/Library/Fraction_Field.thy	Tue Sep 03 00:51:08 2013 +0200
+++ b/src/HOL/Library/Fraction_Field.thy	Tue Sep 03 01:12:40 2013 +0200
@@ -209,7 +209,7 @@
 next
   case False
   then obtain a b where "q = Fract a b" and "b \<noteq> 0" by (cases q) auto
-  moreover with False have "0 \<noteq> Fract a b" by simp
+  with False have "0 \<noteq> Fract a b" by simp
   with `b \<noteq> 0` have "a \<noteq> 0" by (simp add: Zero_fract_def eq_fract)
   with Fract `q = Fract a b` `b \<noteq> 0` show thesis by auto
 qed