diff -r c8a2755bf220 -r ff784d5a5bfb src/Doc/Tutorial/Misc/Tree2.thy --- a/src/Doc/Tutorial/Misc/Tree2.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/Doc/Tutorial/Misc/Tree2.thy Sat Jan 05 17:24:33 2019 +0100 @@ -3,9 +3,9 @@ (*>*) text\\noindent In Exercise~\ref{ex:Tree} we defined a function -@{term"flatten"} from trees to lists. The straightforward version of -@{term"flatten"} is based on \@\ and is thus, like @{term"rev"}, -quadratic. A linear time version of @{term"flatten"} again reqires an extra +\<^term>\flatten\ from trees to lists. The straightforward version of +\<^term>\flatten\ is based on \@\ and is thus, like \<^term>\rev\, +quadratic. A linear time version of \<^term>\flatten\ again reqires an extra argument, the accumulator. Define\ (*<*)primrec(*>*)flatten2 :: "'a tree \ 'a list \ 'a list"(*<*)where "flatten2 Tip xs = xs" |