equal
deleted
inserted
replaced
720 @@{ML_antiquotation print} @{syntax name}? |
720 @@{ML_antiquotation print} @{syntax name}? |
721 \<close>} |
721 \<close>} |
722 |
722 |
723 \begin{description} |
723 \begin{description} |
724 |
724 |
725 \item @{text "@{make_string}"} inlines a function to print arbitrary |
725 \item @{text "@{make_string}"} inlines a function to print arbitrary values |
726 values similar to the ML toplevel. The result is compiler dependent |
726 similar to the ML toplevel. The result is compiler dependent and may fall |
727 and may fall back on "?" in certain situations. |
727 back on "?" in certain situations. The value of configuration option |
|
728 @{attribute_ref ML_print_depth} is used implicitly at compile-time. |
728 |
729 |
729 \item @{text "@{print f}"} uses the ML function @{text "f: string -> |
730 \item @{text "@{print f}"} uses the ML function @{text "f: string -> |
730 unit"} to output the result of @{text "@{make_string}"} above, |
731 unit"} to output the result of @{text "@{make_string}"} above, |
731 together with the source position of the antiquotation. The default |
732 together with the source position of the antiquotation. The default |
732 output function is @{ML writeln}. |
733 output function is @{ML writeln}. |