diff -r a2a7f65f538a -r 51444f205b5b thys/CountSnoc.thy~ --- a/thys/CountSnoc.thy~ Tue Oct 07 18:43:29 2014 +0100 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,29 +0,0 @@ -theory CountSnoc -imports Main -begin - - -datatype 'a myList = Nil | Cons 'a "'a myList" - -fun app_list :: "'a myList \ 'a myList \ 'a myList" where -"app_list Nil ys = ys" | -"app_list (Cons x xs) ys = Cons x (app_list xs ys)" - -fun rev_list :: "'a myList \ 'a myList" where -"rev_list Nil = Nil" | -"rev_list (Cons x xs) = app_list (rev_list xs) (Cons x Nil)" - -fun count_list :: "'a \ 'a list \ nat" where -"count_list x [] = 0" | -"count_list x (y#xs) = ( - if x = y then Suc(count_list x xs) - else count_list x xs)" - -value "count_list (1::nat) [1,1,1]" -value "count_list (1::nat) [2,2,2]" -value "count_list (2::nat) [2,2,1]" - - - - -