src/HOL/Analysis/Great_Picard.thy
changeset 67719 bffb7482faaa
parent 67399 eab6ce8368fa
child 68255 009f783d1bac
--- a/src/HOL/Analysis/Great_Picard.thy	Sat Feb 24 17:21:35 2018 +0100
+++ b/src/HOL/Analysis/Great_Picard.thy	Sun Feb 25 12:54:55 2018 +0000
@@ -46,7 +46,7 @@
   have "(n-1)^2 \<le> n^2 - 1"
     using assms by (simp add: algebra_simps power2_eq_square)
   then have "real (n - 1) \<le> sqrt (real (n\<^sup>2 - 1))"
-    by (metis Extended_Nonnegative_Real.of_nat_le_iff of_nat_power real_le_rsqrt)
+    by (metis of_nat_le_iff of_nat_power real_le_rsqrt)
   then have "n-1 \<le> sqrt(real n ^ 2 - 1)"
     by (simp add: Suc_leI assms of_nat_diff)
   then show ?thesis