aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-09-15 19:17:34 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-09-15 19:17:34 +0200
commit1c113305039857ca219f252f5e80f4b179a39082 (patch)
treec807f1c6cd1b0840f9fbc1abd33ca14b89914f2d /test-suite/success
parentc3e23086ea7fe78d6ae75ed0f162975d76ddd3bf (diff)
Adapting ltac output test to new interpretation of binders.
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/ltac.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/ltac.v b/test-suite/success/ltac.v
index c4a45b031..badce063e 100644
--- a/test-suite/success/ltac.v
+++ b/test-suite/success/ltac.v
@@ -143,7 +143,7 @@ Qed.
Ltac check_binding y := cut ((fun y => y) = S).
Goal True.
-check_binding true.
+check_binding ipattern:H.
Abort.
(* Check that variables explicitly parsed as ltac variables are not