aboutsummaryrefslogtreecommitdiff
path: root/lib
diff options
context:
space:
mode:
authorMaxime Dénès2019-04-01 17:41:22 +0200
committerMaxime Dénès2019-04-03 12:01:25 +0200
commitf374b79e08e135de11def93005110a833686c5f7 (patch)
tree5b48870361b12c53f254381cbf809e2697e5e5ef /lib
parentb45d4425b760b4e6346df4ea19f24d5c1e84b911 (diff)
Protect some I/O routines from SIGALRM
This is necessary to prevent Coq from sending ill-formed output in some scenarios involving `Timeout`. Co-authored-by: Enrico Tassi <Enrico.Tassi@inria.fr>
Diffstat (limited to 'lib')
-rw-r--r--lib/control.ml18
-rw-r--r--lib/control.mli11
2 files changed, 29 insertions, 0 deletions
diff --git a/lib/control.ml b/lib/control.ml
index ffb3584f1e..9054507e46 100644
--- a/lib/control.ml
+++ b/lib/control.ml
@@ -89,3 +89,21 @@ let timeout_fun_ref = ref timeout_fun
let set_timeout f = timeout_fun_ref := f
let timeout n f e = !timeout_fun_ref.timeout n f e
+
+let protect_sigalrm f x =
+ let timed_out = ref false in
+ let timeout_handler _ = timed_out := true in
+ try
+ let old_handler = Sys.signal Sys.sigalrm (Sys.Signal_handle timeout_handler) in
+ try
+ let res = f x in
+ Sys.set_signal Sys.sigalrm old_handler;
+ match !timed_out, old_handler with
+ | true, Sys.Signal_handle f -> f Sys.sigalrm; res
+ | _, _ -> res
+ with e ->
+ let e = Backtrace.add_backtrace e in
+ Sys.set_signal Sys.sigalrm old_handler;
+ Exninfo.iraise e
+ with Invalid_argument _ -> (* This happens on Windows, as handling SIGALRM does not seem supported *)
+ f x
diff --git a/lib/control.mli b/lib/control.mli
index 59e2a15158..640d41a4f7 100644
--- a/lib/control.mli
+++ b/lib/control.mli
@@ -29,3 +29,14 @@ val timeout : int -> ('a -> 'b) -> 'a -> exn -> 'b
API and it is scheduled to go away. *)
type timeout = { timeout : 'a 'b. int -> ('a -> 'b) -> 'a -> exn -> 'b }
val set_timeout : timeout -> unit
+
+(** [protect_sigalrm f x] computes [f x], but if SIGALRM is received during that
+ computation, the signal handler is executed only once the computation is
+ terminated. Otherwise said, it makes the execution of [f] atomic w.r.t.
+ handling of SIGALRM.
+
+ This is useful for example to prevent the implementation of `Timeout` to
+ interrupt I/O routines, generating ill-formed output.
+
+*)
+val protect_sigalrm : ('a -> 'b) -> 'a -> 'b