src/Doc/IsarImplementation/ML.thy
changeset 51058 98c48d023136
parent 48985 5386df44a037
child 51295 71fc3776c453
equal deleted inserted replaced
51057:a22b134f862e 51058:98c48d023136
  1048   perfectly legal alternative: it means that the error is absorbed
  1048   perfectly legal alternative: it means that the error is absorbed
  1049   without any message output.
  1049   without any message output.
  1050 
  1050 
  1051   \begin{warn}
  1051   \begin{warn}
  1052   The actual error channel is accessed via @{ML Output.error_msg}, but
  1052   The actual error channel is accessed via @{ML Output.error_msg}, but
  1053   the interaction protocol of Proof~General \emph{crashes} if that
  1053   the old interaction protocol of Proof~General \emph{crashes} if that
  1054   function is used in regular ML code: error output and toplevel
  1054   function is used in regular ML code: error output and toplevel
  1055   command failure always need to coincide.
  1055   command failure always need to coincide.
  1056   \end{warn}
  1056   \end{warn}
  1057 
  1057 
  1058   \end{description}
  1058   \end{description}