src/HOL/List.thy
changeset 25157 8b80535cd017
parent 25134 3d4953e88449
child 25162 ad4d5365d9d8
--- a/src/HOL/List.thy	Tue Oct 23 12:47:21 2007 +0200
+++ b/src/HOL/List.thy	Tue Oct 23 13:10:19 2007 +0200
@@ -961,9 +961,7 @@
   next
     assume "\<not> p x"
     hence eq: "?S' = Suc ` ?S"
-      apply(auto simp add: nth_Cons image_def split:nat.split elim:lessE)
-      apply (rule_tac x="xa - 1" in exI, auto)
-      done
+      by(auto simp add: image_def neq0_conv split:nat.split elim:lessE)
     have "length (filter p (x # xs)) = card ?S"
       using Cons `\<not> p x` by simp
     also have "\<dots> = card(Suc ` ?S)" using fin