src/HOL/List.thy
changeset 19585 70a1ce3b23ae
parent 19487 d5e79a41bce0
child 19607 07eeb832f28d
--- a/src/HOL/List.thy	Sun May 07 00:21:13 2006 +0200
+++ b/src/HOL/List.thy	Sun May 07 00:22:05 2006 +0200
@@ -818,7 +818,7 @@
 lemma Cons_eq_filterD:
  "x#xs = filter P ys \<Longrightarrow>
   \<exists>us vs. ys = us @ x # vs \<and> (\<forall>u\<in>set us. \<not> P u) \<and> P x \<and> xs = filter P vs"
-  (concl is "\<exists>us vs. ?P ys us vs")
+  (is "_ \<Longrightarrow> \<exists>us vs. ?P ys us vs")
 proof(induct ys)
   case Nil thus ?case by simp
 next