src/ZF/List_ZF.thy
changeset 58860 fee7cfa69c50
parent 46953 2b6e55924af3
child 58871 c399ae4b836f
--- a/src/ZF/List_ZF.thy	Sat Nov 01 11:40:55 2014 +0100
+++ b/src/ZF/List_ZF.thy	Sat Nov 01 14:20:38 2014 +0100
@@ -1216,7 +1216,7 @@
 lemma sublist_upt_eq_take [rule_format, simp]:
     "xs:list(A) ==> \<forall>n\<in>nat. sublist(xs,n) = take(n,xs)"
 apply (erule list.induct, simp)
-apply (clarify );
+apply (clarify )
 apply (erule natE)
 apply (simp_all add: nat_eq_Collect_lt Ord_mem_iff_lt sublist_Cons)
 done