aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Tactics.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-23 09:48:18 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-23 09:48:18 +0000
commit6e02a35b241c29d257c8bb90f29161892f69153b (patch)
treeeb47aa53ae2d6b1a46492a1a752d695043f5af3c /test-suite/output/Tactics.v
parent6eeef3e6e1a0f8fe9183101db86349a5de33754d (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
Diffstat (limited to 'test-suite/output/Tactics.v')
-rw-r--r--test-suite/output/Tactics.v9
1 files changed, 9 insertions, 0 deletions
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.