aboutsummaryrefslogtreecommitdiffstats
path: root/examples/Example.v
diff options
context:
space:
mode:
authorChantal Keller <Chantal.Keller@lri.fr>2022-04-14 18:09:46 +0200
committerChantal Keller <Chantal.Keller@lri.fr>2022-04-14 18:09:46 +0200
commitd2585fac6defa17889a0244556b6822fc0c3cb4e (patch)
treeca0f10fb4be4caadc348670b0fde3ddd49d19cd9 /examples/Example.v
parent7ce6bf4f7740de4c69877ec9179520bcaa0d014c (diff)
parent1f21e1f95d43f5e76e38e1737de9a2a0322fd71c (diff)
downloadsmtcoq-d2585fac6defa17889a0244556b6822fc0c3cb4e.tar.gz
smtcoq-d2585fac6defa17889a0244556b6822fc0c3cb4e.zip
Merge remote-tracking branch 'origin/coq-8.12' into coq-8.13
Diffstat (limited to 'examples/Example.v')
-rw-r--r--examples/Example.v27
1 files changed, 26 insertions, 1 deletions
diff --git a/examples/Example.v b/examples/Example.v
index cd53212..5e12e74 100644
--- a/examples/Example.v
+++ b/examples/Example.v
@@ -14,7 +14,6 @@
If you are using native-coq instead of Coq 8.11, replace it with:
Require Import SMTCoq.
*)
-
Require Import SMTCoq.SMTCoq.
Require Import Bool.
@@ -425,3 +424,29 @@ Section CompCert.
Qed.
End CompCert.
+
+
+(** The verit solver can be called with a timeout (a positive integer,
+ in seconds). If the goal cannot be solved within this given time,
+ then an anomaly is raised.
+ To test, one can uncomment the following examples.
+**)
+
+Section test_timeout.
+
+ Variable P : Z -> bool.
+ Variable H0 : P 0.
+ Variable HInd : forall n, implb (P n) (P (n + 1)).
+
+ Goal P 3.
+ Proof.
+ (* verit_timeout 3. *) verit.
+ Qed.
+
+ Goal true -> P 1000000000.
+ Proof.
+ intro H.
+ (* verit_timeout 5. *)
+ Abort.
+
+End test_timeout.