aboutsummaryrefslogtreecommitdiffhomepage
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 20:29:58 +0200
commit47b4573a77ef88f8528c8247108eba8b04d81525 (patch)
treeffcc5c98c9f09e7d3e9293536833666ba7ef9758
parent12667b1bb33e05ab473b8ee8c4ef9aede5fa2600 (diff)
Fixing test apply.v (had wrong option name).
-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.