src/HOL/Analysis/Conformal_Mappings.thy
changeset 65963 ca1e636fa716
parent 65578 e4997c181cce
child 65965 088c79b40156
--- a/src/HOL/Analysis/Conformal_Mappings.thy	Mon May 29 22:49:52 2017 +0200
+++ b/src/HOL/Analysis/Conformal_Mappings.thy	Tue May 30 10:03:35 2017 +0200
@@ -1061,15 +1061,15 @@
     define m where "m = (GREATEST k. k\<le>n \<and> a k \<noteq> 0)"
     have m: "m\<le>n \<and> a m \<noteq> 0"
       unfolding m_def
-      apply (rule GreatestI [where b = "Suc n"])
+      apply (rule GreatestI [where b = n])
       using k apply auto
       done
     have [simp]: "a i = 0" if "m < i" "i \<le> n" for i
-      using Greatest_le [where b = "Suc n" and P = "\<lambda>k. k\<le>n \<and> a k \<noteq> 0"]
+      using Greatest_le [where b = "n" and P = "\<lambda>k. k\<le>n \<and> a k \<noteq> 0"]
       using m_def not_le that by auto
     have "k \<le> m"
       unfolding m_def
-      apply (rule Greatest_le [where b = "Suc n"])
+      apply (rule Greatest_le [where b = "n"])
       using k apply auto
       done
     with k m show ?thesis