src/HOL/GCD.thy
changeset 66936 cf8d8fc23891
parent 66836 4eb431c3f974
child 67051 e7e54a0b9197
--- a/src/HOL/GCD.thy	Sun Oct 29 19:39:03 2017 +0100
+++ b/src/HOL/GCD.thy	Mon Oct 30 13:18:41 2017 +0000
@@ -1600,13 +1600,10 @@
     by simp
 next
   case False
-  then have "inj (times b)"
-    by (rule inj_times)
   show ?thesis proof (cases "finite A")
     case False
-    moreover from \<open>inj (times b)\<close>
-    have "inj_on (times b) A"
-      by (rule inj_on_subset) simp
+    moreover have "inj_on (times b) A"
+      using \<open>b \<noteq> 0\<close> by (rule inj_on_mult)
     ultimately have "infinite (times b ` A)"
       by (simp add: finite_image_iff)
     with False show ?thesis