--- a/CookBook/Solutions.thy Mon Jan 26 12:29:01 2009 +0000
+++ b/CookBook/Solutions.thy Mon Jan 26 12:29:43 2009 +0000
@@ -41,11 +41,14 @@
@{ML scan_all} retruns a string, instead of the pair a parser would
normally return. For example:
- @{ML_response [display,gray] "scan_all (explode \"foo bar\")" "\"foo bar\""}
-
- @{ML_response [display,gray] "scan_all (explode \"foo (*test*) bar (*test*)\")"
- "\"foo (**test**) bar (**test**)\""}
-
+ @{ML_response [display,gray]
+"let
+ val input1 = (explode \"foo bar\")
+ val input2 = (explode \"foo (*test*) bar (*test*)\")
+ in
+ (scan_all input1, scan_all input2)
+ end"
+"(\"foo bar\",\"foo (**test**) bar (**test**)\")"}
*}
end
\ No newline at end of file