aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/RefMan-tac.tex
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-10 03:05:59 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-10 03:05:59 +0000
commite23ce63217dea3dcd1a760b44d774ad81f01a202 (patch)
tree932042f855ab7419b43734f939dad0bd49b8aa78 /doc/RefMan-tac.tex
parent28025ba8daddfb093ba3feafebb56290fd924fa6 (diff)
MAJ decompose
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8182 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/RefMan-tac.tex')
-rw-r--r--doc/RefMan-tac.tex2
1 files changed, 2 insertions, 0 deletions
diff --git a/doc/RefMan-tac.tex b/doc/RefMan-tac.tex
index 5f82ef8f6..eb1d65d81 100644
--- a/doc/RefMan-tac.tex
+++ b/doc/RefMan-tac.tex
@@ -955,6 +955,8 @@ Intros A B C H; Decompose [and or] H; Assumption.
Qed.
\end{coq_example*}
+{\tt Decompose} does not work on right-hand sides of implications or products.
+
\begin{Variants}
\item {\tt Decompose Sum \term}\tacindex{Decompose Sum}