diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2005-12-23 09:48:18 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2005-12-23 09:48:18 +0000 |
commit | 6e02a35b241c29d257c8bb90f29161892f69153b (patch) | |
tree | eb47aa53ae2d6b1a46492a1a752d695043f5af3c | |
parent | 6eeef3e6e1a0f8fe9183101db86349a5de33754d (diff) |
Test printing of Tactic Notation which was broken until dec 2005
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7707 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r-- | test-suite/output/Tactics.out | 1 | ||||
-rw-r--r-- | test-suite/output/Tactics.v | 9 |
2 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/output/Tactics.out b/test-suite/output/Tactics.out new file mode 100644 index 000000000..71c59e432 --- /dev/null +++ b/test-suite/output/Tactics.out @@ -0,0 +1 @@ +intro H; split; [ a H | e H ]. diff --git a/test-suite/output/Tactics.v b/test-suite/output/Tactics.v new file mode 100644 index 000000000..24a33651c --- /dev/null +++ b/test-suite/output/Tactics.v @@ -0,0 +1,9 @@ +(* Test printing of Tactic Notation *) + +Tactic Notation "a" constr(x) := apply x. +Tactic Notation "e" constr(x) := exact x. + +Lemma test : True -> True /\ True. +intro H; split; [a H|e H]. +Show Script. +Qed. |