aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proofview.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-08-28 15:14:29 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-08-28 22:45:24 +0200
commit58543b45425b85233c068f9da859996270d1fdcf (patch)
tree6981dca5a3bf4468d2533bb239dcf44aca190ebf /proofs/proofview.mli
parent32c83676c96ae4a218de0bec75d2f3353381dfb3 (diff)
Simplification of the tclCHECKINTERRUPT tactic.
Diffstat (limited to 'proofs/proofview.mli')
-rw-r--r--proofs/proofview.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/proofs/proofview.mli b/proofs/proofview.mli
index b10cc1843..b1466fcfb 100644
--- a/proofs/proofview.mli
+++ b/proofs/proofview.mli
@@ -140,9 +140,6 @@ val apply : Environ.env -> 'a tactic -> proofview -> 'a
(* Unit of the tactic monad *)
val tclUNIT : 'a -> 'a tactic
-(* Unit but checks for interrupts *)
-val tclCHECKINTERRUPT : 'a -> 'a tactic
-
(* Bind operation of the tactic monad *)
val tclBIND : 'a tactic -> ('a -> 'b tactic) -> 'b tactic
@@ -259,6 +256,9 @@ val tclIN_ENV : Environ.env -> 'a tactic -> 'a tactic
(* [tclEFFECTS eff] add the effects [eff] to the current state. *)
val tclEFFECTS : Declareops.side_effects -> unit tactic
+(* Checks for interrupts *)
+val tclCHECKINTERRUPT : unit tactic
+
(* Shelves all the goals under focus. The goals are placed on the
shelf for later use (or being solved by side-effects). *)
val shelve : unit tactic