Eliminated mutual_induct_tac.
authorberghofe
Wed, 13 Oct 1999 15:41:24 +0200
changeset 7848 6ddcc24038e1
parent 7847 5a3fa0c4b215
child 7849 29a2a1d71128
Eliminated mutual_induct_tac.
doc-src/Tutorial/Datatype/abgoalfind.ML
doc-src/Tutorial/Datatype/abgoalind.ML
doc-src/Tutorial/Datatype/tidproof.ML
doc-src/Tutorial/fp.tex
--- a/doc-src/Tutorial/Datatype/abgoalfind.ML	Wed Oct 13 15:18:15 1999 +0200
+++ b/doc-src/Tutorial/Datatype/abgoalfind.ML	Wed Oct 13 15:41:24 1999 +0200
@@ -1,4 +1,4 @@
 Goal
  "evala env (substa s a) = evala (%x. evala env (s x)) a & \
 \ evalb env (substb s b) = evalb (%x. evala env (s x)) b";
-by(mutual_induct_tac ["a","b"] 1);
+by(induct_tac "a b" 1);
--- a/doc-src/Tutorial/Datatype/abgoalind.ML	Wed Oct 13 15:18:15 1999 +0200
+++ b/doc-src/Tutorial/Datatype/abgoalind.ML	Wed Oct 13 15:41:24 1999 +0200
@@ -1,4 +1,4 @@
 Goal
  "evala env (substa s a) = evala (%x. evala env (s x)) a & \
 \ evalb env (substb s b) = evalb (%x. evala env (s x)) b";
-by(mutual_induct_tac ["a","b"] 1);
+by(induct_tac "a b" 1);
--- a/doc-src/Tutorial/Datatype/tidproof.ML	Wed Oct 13 15:18:15 1999 +0200
+++ b/doc-src/Tutorial/Datatype/tidproof.ML	Wed Oct 13 15:41:24 1999 +0200
@@ -1,4 +1,4 @@
 Goal "subst  Var t  = (t ::('a,'b)term)  & \
 \     substs Var ts = (ts::('a,'b)term list)";
-by(mutual_induct_tac ["t", "ts"] 1);
+by(induct_tac "t ts" 1);
 by(Auto_tac);
--- a/doc-src/Tutorial/fp.tex	Wed Oct 13 15:18:15 1999 +0200
+++ b/doc-src/Tutorial/fp.tex	Wed Oct 13 15:41:24 1999 +0200
@@ -1356,7 +1356,7 @@
 theorems simultaneously:
 \begin{quote}\small
 \verbatiminput{Datatype/abgoalind.ML}
-\end{quote}\indexbold{*mutual_induct_tac}
+\end{quote}
 The resulting 8 goals (one for each constructor) are proved in one fell swoop
 \texttt{by Auto_tac;}.
 
@@ -1365,7 +1365,7 @@
 \[ P@1(x@1)\ \texttt{\&}\ \dots\ \texttt{\&}\ P@n(x@n) \]
 where each variable $x@i$ is of type $\tau@i$. Induction is started by
 \begin{ttbox}
-by(mutual_induct_tac ["\(x@1\)",\(\dots\),"\(x@n\)"] \(k\));
+by(induct_tac "\(x@1\) \(\dots\) \(x@n\)" \(k\));
 \end{ttbox}
 
 \begin{exercise}