aboutsummaryrefslogtreecommitdiff
path: root/test-suite/ide
diff options
context:
space:
mode:
authorEnrico Tassi2018-12-13 10:56:13 +0100
committerEnrico Tassi2018-12-13 10:59:46 +0100
commita9e87e0b25cf11192d11da4499c3c3122f11a0c4 (patch)
tree350c09ee2dddc1a30b8c350c0263e6ee24bb41b4 /test-suite/ide
parent4838146ee993a3bafb6a359dff529aae815cfff6 (diff)
[test] for join when error resiliency on and async-proofs off
Diffstat (limited to 'test-suite/ide')
-rw-r--r--test-suite/ide/join-sync.fake20
1 files changed, 20 insertions, 0 deletions
diff --git a/test-suite/ide/join-sync.fake b/test-suite/ide/join-sync.fake
new file mode 100644
index 0000000000..236028ce46
--- /dev/null
+++ b/test-suite/ide/join-sync.fake
@@ -0,0 +1,20 @@
+# Script simulating a dialog between coqide and coqtop -ideslave
+# Run it via fake_ide
+#
+# Error resiliency + async proofs off
+# coq-prog-args: ("-async-proofs" "off" "-async-proofs-command-error-resilience" "on")
+#
+
+ADD { Lemma x : True. }
+ADD { Proof using. }
+ADD here { trivial. }
+ADD { fail. }
+ADD { Qed. }
+ADD { Lemma y : True. }
+ADD { Proof using. }
+ADD { trivial. }
+ADD { Qed. }
+WAIT
+FAILJOIN
+ASSERT TIP here
+ABORT