aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2017-01-20 13:51:37 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2017-01-20 14:14:24 +0100
commit1d4c34c79624fb81e64dfed8874b2fc9fa66c070 (patch)
tree26532d59e4e304037d5bdee61f2180da4614ae57
parenta9b76df171ceea443885bb4be919ea586a82beee (diff)
Process Next Obligation proofs in parallel (fix #5314)
-rw-r--r--intf/vernacexpr.mli3
-rw-r--r--ltac/g_obligations.ml42
2 files changed, 4 insertions, 1 deletions
diff --git a/intf/vernacexpr.mli b/intf/vernacexpr.mli
index 92e4dd618..c9fb1b598 100644
--- a/intf/vernacexpr.mli
+++ b/intf/vernacexpr.mli
@@ -524,6 +524,9 @@ and vernac_control =
| VtObserve of Stateid.t
| VtBack of Stateid.t
| VtPG
+(* Qed typically generates an opaque proof term. Still, by declaring
+ * a proof terminator one can use such opaque term to generate transparent
+ * ones. In this corner case the STM needs to know... *)
and opacity_guarantee =
| GuaranteesOpacity (** Only generates opaque terms at [Qed] *)
| Doesn'tGuaranteeOpacity (** May generate transparent terms even with [Qed].*)
diff --git a/ltac/g_obligations.ml4 b/ltac/g_obligations.ml4
index 987b9d538..2ae183e6e 100644
--- a/ltac/g_obligations.ml4
+++ b/ltac/g_obligations.ml4
@@ -66,7 +66,7 @@ GEXTEND Gram
open Obligations
-let classify_obbl _ = Vernacexpr.(VtStartProof ("Classic",Doesn'tGuaranteeOpacity,[]), VtLater)
+let classify_obbl _ = Vernacexpr.(VtStartProof ("Classic",GuaranteesOpacity,[]), VtLater)
VERNAC COMMAND EXTEND Obligations CLASSIFIED BY classify_obbl
| [ "Obligation" integer(num) "of" ident(name) ":" lglob(t) withtac(tac) ] ->