equal
deleted
inserted
replaced
182 "rev (Cons x xs) = app (rev xs) (Cons x Nil)" |
182 "rev (Cons x xs) = app (rev xs) (Cons x Nil)" |
183 |
183 |
184 text{* By default, variables @{text xs}, @{text ys} and @{text zs} are of |
184 text{* By default, variables @{text xs}, @{text ys} and @{text zs} are of |
185 @{text list} type. |
185 @{text list} type. |
186 |
186 |
187 Command \isacom{value}\indexed{{\sf\textbf{value}}}{value} evaluates a term. For example, *} |
187 Command \indexed{\isacommand{value}}{value} evaluates a term. For example, *} |
188 |
188 |
189 value "rev(Cons True (Cons False Nil))" |
189 value "rev(Cons True (Cons False Nil))" |
190 |
190 |
191 text{* yields the result @{value "rev(Cons True (Cons False Nil))"}. This works symbolically, too: *} |
191 text{* yields the result @{value "rev(Cons True (Cons False Nil))"}. This works symbolically, too: *} |
192 |
192 |