src/HOL/Algebra/IntRing.thy
changeset 29242 e190bc2a5399
parent 29237 e90d9d51106b
child 29424 948d616959e4
--- a/src/HOL/Algebra/IntRing.thy	Thu Dec 18 20:19:49 2008 +0100
+++ b/src/HOL/Algebra/IntRing.thy	Fri Dec 19 11:09:09 2008 +0100
@@ -328,7 +328,7 @@
 next
   assume "UNIV = {uu. EX x. uu = x * p}"
   from this obtain x 
-      where "1 = x * p" by fast
+      where "1 = x * p" by best
   from this [symmetric]
       have "p * x = 1" by (subst zmult_commute)
   hence "\<bar>p * x\<bar> = 1" by simp