added done to the proof.
authorChristian Urban <christian dot urban at kcl dot ac dot uk>
Wed, 08 Oct 2014 10:30:14 +0100
changeset 27 378077bab5d2
parent 26 51444f205b5b
child 28 d3831bf423f2
added done to the proof.
thys/CountSnoc.thy
--- 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