| author | blanchet | 
| Tue, 20 May 2014 09:57:10 +0200 | |
| changeset 57014 | b7999893ffcc | 
| parent 56451 | 856492b0f755 | 
| child 57804 | fcf966675478 | 
| permissions | -rw-r--r-- | 
theory MyList imports Main begin datatype 'a list = Nil | Cons 'a "'a list" fun app :: "'a list => 'a list => 'a list" where "app Nil ys = ys" | "app (Cons x xs) ys = Cons x (app xs ys)" fun rev :: "'a list => 'a list" where "rev Nil = Nil" | "rev (Cons x xs) = app (rev xs) (Cons x Nil)" value "rev(Cons True (Cons False Nil))" end