adapted proof of less_succ: problem because of non-confluent SimpSet removed
authoroheimb
Thu, 18 Apr 1996 14:11:02 +0200
changeset 1662 a6b55b9d2f22
parent 1661 1e2462c3fece
child 1663 7e84d8712a0b
adapted proof of less_succ: problem because of non-confluent SimpSet removed
src/FOL/ex/Nat2.ML
--- a/src/FOL/ex/Nat2.ML	Thu Apr 18 12:33:05 1996 +0200
+++ b/src/FOL/ex/Nat2.ML	Thu Apr 18 14:11:02 1996 +0200
@@ -158,9 +158,7 @@
 by (IND_TAC nat_ind (simp_tac nat_ss) "j" 1);
 by (ALL_IND_TAC nat_exh (simp_tac nat_ss) 1);
 by (resolve_tac [impI RS allI] 1);
-by (rtac nat_exh 1);
-by (simp_tac nat_ss 1);
-by (simp_tac nat_ss 1);
+by (ALL_IND_TAC nat_exh (simp_tac nat_ss) 1);
 by (asm_simp_tac nat_ss 1);
 qed "less_succ";