aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/ide
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-05-27 11:50:11 +0200
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-05-28 13:50:43 +0200
commit5c437ab917bd24de66986e95dcf58c3f31e17a34 (patch)
tree500f703631f042df930e688b61247054269a5db3 /test-suite/ide
parentc6714db203f60413523ebeaac86242a6e4cc05e3 (diff)
STM: preserve branch name on edit (Close: #4245, #4246)
Diffstat (limited to 'test-suite/ide')
-rw-r--r--test-suite/ide/reopen.fake21
1 files changed, 21 insertions, 0 deletions
diff --git a/test-suite/ide/reopen.fake b/test-suite/ide/reopen.fake
new file mode 100644
index 000000000..8166d0137
--- /dev/null
+++ b/test-suite/ide/reopen.fake
@@ -0,0 +1,21 @@
+# Script simulating a dialog between coqide and coqtop -ideslave
+# Run it via fake_ide
+#
+# jumping between broken proofs + interp error while fixing.
+# the error should note make the GUI unfocus the currently focused proof.
+
+# first proof
+ADD { Lemma a : True. }
+ADD here { Proof using. }
+ADD { fail. }
+ADD { trivial. } # first error
+ADD { Qed. }
+WAIT
+EDIT_AT here
+# Fixing the proof
+ADD fix { trivial. }
+ADD { Qed. }
+WAIT
+EDIT_AT fix
+ADD { Qed. }
+JOIN