aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorcoqbot-app[bot]2021-03-31 15:48:13 +0000
committerGitHub2021-03-31 15:48:13 +0000
commit1a64b1560ce88855a76e2faa14cec2864de2f37c (patch)
tree4b63e2bf8d4c29ce789bd84d511a62608d59fe2c /test-suite
parent3442bfa0e7c7e5ba3ce7d62f16d221c2e6da03cf (diff)
parentf77d6a239ff70a8aaa10d256f545fc21b2c7ecc0 (diff)
Merge PR #14035: Fix printing of ssr do intros and seq tactics
Reviewed-by: gares Reviewed-by: ppedrot
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/output/bug_13240.out3
-rw-r--r--test-suite/output/bug_13240.v10
2 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/output/bug_13240.out b/test-suite/output/bug_13240.out
new file mode 100644
index 0000000000..5fccef5cfe
--- /dev/null
+++ b/test-suite/output/bug_13240.out
@@ -0,0 +1,3 @@
+Ltac t1 a b := a ; last b
+Ltac t2 := do !idtac
+Ltac t3 := idtac => True
diff --git a/test-suite/output/bug_13240.v b/test-suite/output/bug_13240.v
new file mode 100644
index 0000000000..a999450cd2
--- /dev/null
+++ b/test-suite/output/bug_13240.v
@@ -0,0 +1,10 @@
+Require Import ssreflect.
+
+Ltac t1 a b := a; last b.
+Print t1.
+
+Ltac t2 := do !idtac.
+Print t2.
+
+Ltac t3 := idtac => True.
+Print t3.