src/ZF/ex/Comb.ML
changeset 1732 38776e927da8
parent 1692 5324be24a5fa
child 2469 b50b8c0eec01
--- a/src/ZF/ex/Comb.ML	Wed May 08 16:10:32 1996 +0200
+++ b/src/ZF/ex/Comb.ML	Wed May 08 17:43:23 1996 +0200
@@ -23,9 +23,6 @@
 
 (*** Results about Contraction ***)
 
-bind_thm ("contract_induct",
-    (contract.mutual_induct RS spec RS spec RSN (2,rev_mp)));
-
 (*For type checking: replaces a-1->b by a,b:comb *)
 val contract_combE2 = contract.dom_subset RS subsetD RS SigmaE2;
 val contract_combD1 = contract.dom_subset RS subsetD RS SigmaD1;
@@ -119,9 +116,6 @@
 
 (*** Results about Parallel Contraction ***)
 
-bind_thm ("parcontract_induct",
-    (parcontract.mutual_induct RS spec RS spec RSN (2,rev_mp)));
-
 (*For type checking: replaces a=1=>b by a,b:comb *)
 val parcontract_combE2 = parcontract.dom_subset RS subsetD RS SigmaE2;
 val parcontract_combD1 = parcontract.dom_subset RS subsetD RS SigmaD1;
@@ -163,7 +157,7 @@
 (*Church-Rosser property for parallel contraction*)
 goalw Comb.thy [diamond_def] "diamond(parcontract)";
 by (rtac (impI RS allI RS allI) 1);
-by (etac parcontract_induct 1);
+by (etac parcontract.induct 1);
 by (ALLGOALS 
     (fast_tac (parcontract_cs addSDs [K1_parcontractD,S2_parcontractD])));
 qed "diamond_parcontract";
@@ -192,7 +186,7 @@
 (*** Equivalence of p--->q and p===>q ***)
 
 goal Comb.thy "!!p q. p-1->q ==> p=1=>q";
-by (etac contract_induct 1);
+by (etac contract.induct 1);
 by (ALLGOALS (fast_tac (parcontract_cs)));
 qed "contract_imp_parcontract";
 
@@ -207,7 +201,7 @@
 
 
 goal Comb.thy "!!p q. p=1=>q ==> p--->q";
-by (etac parcontract_induct 1);
+by (etac parcontract.induct 1);
 by (fast_tac (contract_cs addIs reduction_rls) 1);
 by (fast_tac (contract_cs addIs reduction_rls) 1);
 by (fast_tac (contract_cs addIs reduction_rls) 1);