src/Doc/Implementation/ML.thy
changeset 78681 38fe769658be
parent 77907 ee9785abbcd6
child 78705 fde0b195cb7d
--- a/src/Doc/Implementation/ML.thy	Thu Sep 21 18:17:26 2023 +0200
+++ b/src/Doc/Implementation/ML.thy	Thu Sep 21 23:45:03 2023 +0200
@@ -1121,7 +1121,8 @@
 text \<open>
   These indicate arbitrary system events: both the ML runtime system and the
   Isabelle/ML infrastructure signal various exceptional situations by raising
-  the special \<^ML>\<open>Exn.Interrupt\<close> exception in user code.
+  special exceptions user code, satisfying the predicate
+  \<^ML>\<open>Exn.is_interrupt\<close>.
 
   This is the one and only way that physical events can intrude an Isabelle/ML
   program. Such an interrupt can mean out-of-memory, stack overflow, timeout,