diff options
author | gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2013-10-10 11:22:52 +0000 |
---|---|---|
committer | gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2013-10-10 11:22:52 +0000 |
commit | 2449426bef2e8cfecf46c9ee55a326633064fe4f (patch) | |
tree | 20a40bcff55947e8a5dbfed0ff1d35256e43b530 /test-suite | |
parent | e0f8d741b933361fc33a4ccd683b0137c869c468 (diff) |
fake_ide: ported to Document + 2 tests for editing a proof (locally)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16871 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/Makefile | 2 | ||||
-rw-r--r-- | test-suite/ide/undo007.fake | 5 | ||||
-rw-r--r-- | test-suite/ide/undo020.fake | 27 | ||||
-rw-r--r-- | test-suite/ide/undo021.fake | 29 |
4 files changed, 59 insertions, 4 deletions
diff --git a/test-suite/Makefile b/test-suite/Makefile index f47b0aa0c..cc39e8ac2 100644 --- a/test-suite/Makefile +++ b/test-suite/Makefile @@ -434,7 +434,7 @@ ide : $(patsubst %.fake,%.fake.log,$(wildcard ide/*.fake)) @echo "TEST $<" $(HIDE){ \ echo $(call log_intro,$<); \ - $(BIN)fake_ide "$(BIN)coqtop -boot" < $< 2>&1; \ + $(BIN)fake_ide $< "$(BIN)coqtop -boot -coq-slaves on -coq-slaves-opts min-proof-length-to-delegate=0" 2>&1; \ if [ $$? = 0 ]; then \ echo $(log_success); \ echo " $<...Ok"; \ diff --git a/test-suite/ide/undo007.fake b/test-suite/ide/undo007.fake index 770350fbd..7a1dc81e0 100644 --- a/test-suite/ide/undo007.fake +++ b/test-suite/ide/undo007.fake @@ -11,11 +11,10 @@ ADD { Definition f := O. } # This is a bug in Stm undo, e is lost from master EDIT_AT here ADD { Definition f := O. } - ADD { assert True by trivial. } ADD { exact (eq_refl e). } ADD { Qed. } -ADD { Stm PrintDag. } -ADD { Stm Finish. } +# QUERY { Stm PrintDag. } +# QUERY { Stm Finish. } QUERY { Print d. } QUERY { Check e. } diff --git a/test-suite/ide/undo020.fake b/test-suite/ide/undo020.fake new file mode 100644 index 000000000..2adde908d --- /dev/null +++ b/test-suite/ide/undo020.fake @@ -0,0 +1,27 @@ +# Script simulating a dialog between coqide and coqtop -ideslave +# Run it via fake_ide +# +# focusing a broken proof and fixing it + +# first proof +ADD { Lemma a : True. } +ADD { Proof using. } +ADD here { idtac. } +ADD { exact Ix. } +ADD { Qed. } +# second proof +ADD { Lemma b : False. } +ADD { Proof using. } +ADD { admit. } +ADD last { Qed. } +# We join and expect some proof to fail +WAIT +# Going back to the error +EDIT_AT here +# Fixing the proof +ADD { exact I. } +ADD { Qed. } +# we are back at the end +ASSERT TIP last +QUERY { Check a. } +QUERY { Check b. } diff --git a/test-suite/ide/undo021.fake b/test-suite/ide/undo021.fake new file mode 100644 index 000000000..0d83ad25a --- /dev/null +++ b/test-suite/ide/undo021.fake @@ -0,0 +1,29 @@ +# Script simulating a dialog between coqide and coqtop -ideslave +# Run it via fake_ide +# +# jumping between broken proofs + +# first proof +ADD { Lemma a : True. } +ADD { Proof using. } +ADD here { idtac. } +ADD { exact Ix. } +ADD { Qed. } +# second proof +ADD { Lemma b : True. } +ADD here2 { Proof using. } +ADD { exact Ix. } +ADD { Qed. } +# We wait all slaves and expect both proofs to fail +WAIT +# Going back to the error +EDIT_AT here2 +# this is not implemented yet, all after here is erased +EDIT_AT here +# Fixing the proof +ADD { exact I. } +ADD last { Qed. } +ASSERT TIP last +# we are back at the end +QUERY { Check a. } +QUERY { Fail Check b. } |