thys/CountSnoc.thy
changeset 27 378077bab5d2
parent 25 a2a7f65f538a
child 34 33065bde3bbd
--- a/thys/CountSnoc.thy	Wed Oct 08 10:28:19 2014 +0100
+++ b/thys/CountSnoc.thy	Wed Oct 08 10:30:14 2014 +0100
@@ -26,6 +26,7 @@
 lemma count1: "count_list n(xs @ ys) = count_list n xs + count_list n ys"
 apply(induct xs)
 apply(auto)
+done