src/HOL/Library/GCD.thy
changeset 25112 98824cc791c0
parent 23994 3ddc90d1eda1
child 25594 43c718438f9f
--- a/src/HOL/Library/GCD.thy	Sat Oct 20 12:09:30 2007 +0200
+++ b/src/HOL/Library/GCD.thy	Sat Oct 20 12:09:33 2007 +0200
@@ -396,7 +396,7 @@
   assumes nz: "a \<noteq> 0 \<or> b \<noteq> 0"
   shows "igcd (a div (igcd a b)) (b div (igcd a b)) = 1"
 proof -
-  from nz have nz': "nat \<bar>a\<bar> \<noteq> 0 \<or> nat \<bar>b\<bar> \<noteq> 0" by simp
+  from nz have nz': "nat \<bar>a\<bar> \<noteq> 0 \<or> nat \<bar>b\<bar> \<noteq> 0" by arith 
   let ?g = "igcd a b"
   let ?a' = "a div ?g"
   let ?b' = "b div ?g"