src/HOL/ex/Sqrt.thy
changeset 62348 9a5f43dac883
parent 61762 d50b993b4fb9
child 63534 523b488b15c9
--- a/src/HOL/ex/Sqrt.thy	Wed Feb 17 21:51:57 2016 +0100
+++ b/src/HOL/ex/Sqrt.thy	Wed Feb 17 21:51:57 2016 +0100
@@ -77,7 +77,7 @@
   with p have "n\<^sup>2 = p * k\<^sup>2" by (simp add: power2_eq_square)
   then have "p dvd n\<^sup>2" ..
   with \<open>prime p\<close> have "p dvd n" by (rule prime_dvd_power_nat)
-  with dvd_m have "p dvd gcd m n" by (rule gcd_greatest_nat)
+  with dvd_m have "p dvd gcd m n" by (rule gcd_greatest)
   with \<open>coprime m n\<close> have "p = 1" by simp
   with p show False by simp
 qed