aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman
diff options
context:
space:
mode:
authorGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-30 16:02:22 +0000
committerGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-30 16:02:22 +0000
commit81117e3da0d2a75610c861e466088c311b3727d0 (patch)
tree60199283840a3007f1ee5446af781400de929198 /doc/refman
parent519b9d2f30409f3cfda9dc403a56b1c332bba91f (diff)
add "Print Ring" and "Print Field" vernacular commands
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16751 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/refman')
-rw-r--r--doc/refman/RefMan-tac.tex8
1 files changed, 6 insertions, 2 deletions
diff --git a/doc/refman/RefMan-tac.tex b/doc/refman/RefMan-tac.tex
index 805b2cee0..a1ca53244 100644
--- a/doc/refman/RefMan-tac.tex
+++ b/doc/refman/RefMan-tac.tex
@@ -4505,6 +4505,7 @@ integers. This tactic must be loaded by the command \texttt{Require Import
\tacindex{ring}
\tacindex{ring\_simplify}
\comindex{Add Ring}
+\comindex{Print Rings}
The {\tt ring} tactic solves equations upon polynomial expressions of
a ring (or semi-ring) structure. It proceeds by normalizing both hand
@@ -4519,7 +4520,8 @@ forms. If no term is given, then the conclusion should be an equation
and both hand sides are normalized.
See Chapter~\ref{ring} for more information on the tactic and how to
-declare new ring structures.
+declare new ring structures. All declared field structures can be
+printed with the {\tt Print Rings} command.
\subsection{{\tt field}, {\tt field\_simplify \term$_1$ \mbox{\dots}
\term$_n$}, and \tt field\_simplify\_eq}
@@ -4527,6 +4529,7 @@ declare new ring structures.
\tacindex{field\_simplify}
\tacindex{field\_simplify\_eq}
\comindex{Add Field}
+\comindex{Print Fields}
The {\tt field} tactic is built on the same ideas as {\tt ring}: this
is a reflexive tactic that solves or simplifies equations in a field
@@ -4545,7 +4548,8 @@ All of these 3 tactics may generate a subgoal in order to prove that
denominators are different from zero.
See Chapter~\ref{ring} for more information on the tactic and how to
-declare new field structures.
+declare new field structures. All declared field structures can be
+printed with the {\tt Print Fields} command.
\Example
\begin{coq_example*}