aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/ltac.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-22 11:38:51 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-22 11:46:42 +0200
commit56744aadd413dd9417d245951083117b05170e14 (patch)
tree70557ce730b3c15b3fab584c162cd3da1da0d73f /test-suite/output/ltac.v
parent5609da1e08f950fab85b87b257ed343b491f1ef5 (diff)
Fixing printing of generic arguments of tag "var".
Diffstat (limited to 'test-suite/output/ltac.v')
-rw-r--r--test-suite/output/ltac.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/output/ltac.v b/test-suite/output/ltac.v
index 7e2610c7d..e5bcff8dd 100644
--- a/test-suite/output/ltac.v
+++ b/test-suite/output/ltac.v
@@ -15,3 +15,8 @@ lazymatch goal with
| H1 : HT |- _ => idtac
end.
Abort.
+
+(* Check printing of the "var" argument "Hx" *)
+Ltac m H := idtac H; exact H.
+Goal True.
+let a:=constr:(let Hx := 0 in ltac:(m Hx)) in idtac.