aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-07-31 21:31:37 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-08-02 15:06:53 +0200
commit2418cf8d5ff6f479a5b43a87c861141bf9067507 (patch)
treec9c9f026f3f5f2c2951a668bcf05f909ecfaa80c /doc/refman
parentcb0dea2a0c2993d4ca7747afc61fecdbb1c525b1 (diff)
Granting Jason's request for an ad hoc compatibility option on
considering trivial unifications "?x = t" in tactics working under conjunctions (see #3545). Also updating and fixing wrong comments in test apply.v.
Diffstat (limited to 'doc/refman')
-rw-r--r--doc/refman/RefMan-tac.tex17
1 files changed, 17 insertions, 0 deletions
diff --git a/doc/refman/RefMan-tac.tex b/doc/refman/RefMan-tac.tex
index cc262708a..fa6f78393 100644
--- a/doc/refman/RefMan-tac.tex
+++ b/doc/refman/RefMan-tac.tex
@@ -485,7 +485,24 @@ apply Rmp.
Reset R.
\end{coq_eval}
+\noindent {\bf Remark: } When the conclusion of the type of the term
+to apply is an inductive type isomorphic to a tuple type and {\em apply}
+looks recursively whether a component of the tuple matches the goal,
+it excludes components whose statement would result in applying an
+universal lemma of the form {\tt forall A, ... -> A}. Excluding this
+kind of lemma can be avoided by setting the following option:
+
+\begin{quote}
+\optindex{Universal Lemma Under Conjunction}
+{\tt Set Universal Lemma Under Conjunction}
+\end{quote}
+
+This option, which preserves compatibility with versions of {\Coq}
+prior to 8.4 is also available for {\tt apply {\term} in {\ident}}
+(see Section~\ref{apply-in}).
+
\subsection{\tt apply {\term} in {\ident}}
+\label{apply-in}
\tacindex{apply \dots\ in}
This tactic applies to any goal. The argument {\term} is a term