src/Doc/IsarImplementation/ML.thy
changeset 56303 4cc3f4db3447
parent 56199 8e8d28ed7529
child 56399 386e4cb7ad68
--- a/src/Doc/IsarImplementation/ML.thy	Thu Mar 27 13:00:40 2014 +0100
+++ b/src/Doc/IsarImplementation/ML.thy	Thu Mar 27 17:12:40 2014 +0100
@@ -1163,7 +1163,7 @@
   @{index_ML_exception Fail: string} \\
   @{index_ML Exn.is_interrupt: "exn -> bool"} \\
   @{index_ML reraise: "exn -> 'a"} \\
-  @{index_ML ML_Compiler.exn_trace: "(unit -> 'a) -> 'a"} \\
+  @{index_ML Runtime.exn_trace: "(unit -> 'a) -> 'a"} \\
   \end{mldecls}
 
   \begin{description}
@@ -1191,12 +1191,12 @@
   while preserving its implicit position information (if possible,
   depending on the ML platform).
 
-  \item @{ML ML_Compiler.exn_trace}~@{ML_text "(fn () =>"}~@{text
+  \item @{ML Runtime.exn_trace}~@{ML_text "(fn () =>"}~@{text
   "e"}@{ML_text ")"} evaluates expression @{text "e"} while printing
   a full trace of its stack of nested exceptions (if possible,
   depending on the ML platform).
 
-  Inserting @{ML ML_Compiler.exn_trace} into ML code temporarily is
+  Inserting @{ML Runtime.exn_trace} into ML code temporarily is
   useful for debugging, but not suitable for production code.
 
   \end{description}