src/Doc/Implementation/ML.thy
changeset 57834 0d295e339f52
parent 57832 5b48f2047c24
child 58555 7975676c08c0
--- a/src/Doc/Implementation/ML.thy	Thu Jul 31 21:29:31 2014 +0200
+++ b/src/Doc/Implementation/ML.thy	Thu Jul 31 22:02:21 2014 +0200
@@ -725,7 +725,7 @@
   \item @{text "@{make_string}"} inlines a function to print arbitrary values
   similar to the ML toplevel. The result is compiler dependent and may fall
   back on "?" in certain situations. The value of configuration option
-  @{attribute_ref ML_print_depth} is used implicitly at compile-time.
+  @{attribute_ref ML_print_depth} determines further details of output.
 
   \item @{text "@{print f}"} uses the ML function @{text "f: string ->
   unit"} to output the result of @{text "@{make_string}"} above,