--- a/CookBook/FirstSteps.thy Thu Mar 05 16:46:43 2009 +0000
+++ b/CookBook/FirstSteps.thy Fri Mar 06 16:12:16 2009 +0000
@@ -73,14 +73,14 @@
in your code. This can be done in a ``quick-and-dirty'' fashion using
the function @{ML "warning"}. For example
- @{ML_response [display,gray] "warning \"any string\"" "\"any string\""}
+ @{ML_response_fake [display,gray] "warning \"any string\"" "\"any string\""}
will print out @{text [quotes] "any string"} inside the response buffer
of Isabelle. This function expects a string as argument. If you develop under PolyML,
then there is a convenient, though again ``quick-and-dirty'', method for
converting values into strings, namely the function @{ML makestring}:
- @{ML_response [display,gray] "warning (makestring 1)" "\"1\""}
+ @{ML_response_fake [display,gray] "warning (makestring 1)" "\"1\""}
However @{ML makestring} only works if the type of what is converted is monomorphic
and not a function.
@@ -91,7 +91,7 @@
function @{ML tracing} is more appropriate. This function writes all output into
a separate tracing buffer. For example:
- @{ML_response [display,gray] "tracing \"foo\"" "\"foo\""}
+ @{ML_response_fake [display,gray] "tracing \"foo\"" "\"foo\""}
It is also possible to redirect the ``channel'' where the string @{text "foo"} is
printed to a separate file, e.g.~to prevent ProofGeneral from choking on massive
@@ -708,6 +708,7 @@
| is_nil_or_all (Const (@{const_name "All"}, _) $ _) = true
| is_nil_or_all _ = false *}
+(*
text {*
Occasional you have to calculate what the ``base'' name of a given
constant is. For this you can use the function @{ML Sign.extern_const} or
@@ -725,7 +726,7 @@
FIXME: Find the right files to do with naming.
\end{readmore}
*}
-
+*)
section {* Type-Checking *}