aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-08-02 18:47:08 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-08-02 19:13:52 +0200
commit164637cc3a4e8895ed4ec420e300bd692d3e7812 (patch)
tree06bda2595e309a4d0739630ef522c238e1c179b8 /test-suite
parentb9c96c601a8366b75ee8b76d3184ee57379e2620 (diff)
Fixing test apply.v (had wrong option name).
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/success/apply.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v
index 24d5cf8a9..074004fa1 100644
--- a/test-suite/success/apply.v
+++ b/test-suite/success/apply.v
@@ -371,7 +371,7 @@ Qed.
Goal True.
Fail eapply existT.
-Set Trivial Tactic Unification Under Conjunction.
+Set Universal Lemma Under Conjunction.
eapply existT.
Abort.