src/ZF/ex/ListN.ML
changeset 1732 38776e927da8
parent 1461 6bcb44e4d6e5
child 2469 b50b8c0eec01
--- a/src/ZF/ex/ListN.ML	Wed May 08 16:10:32 1996 +0200
+++ b/src/ZF/ex/ListN.ML	Wed May 08 17:43:23 1996 +0200
@@ -11,9 +11,6 @@
 
 open ListN;
 
-val listn_induct = standard 
-    (listn.mutual_induct RS spec RS spec RSN (2,rev_mp));
-
 goal ListN.thy "!!l. l:list(A) ==> <length(l),l> : listn(A)";
 by (etac list.induct 1);
 by (ALLGOALS (asm_simp_tac list_ss));
@@ -22,7 +19,7 @@
 
 goal ListN.thy "<n,l> : listn(A) <-> l:list(A) & length(l)=n";
 by (rtac iffI 1);
-by (etac listn_induct 1);
+by (etac listn.induct 1);
 by (safe_tac (ZF_cs addSIs (list_typechecks @
                             [length_Nil, length_Cons, list_into_listn])));
 qed "listn_iff";
@@ -41,7 +38,7 @@
 goal ListN.thy
     "!!n l. [| <n,l> : listn(A);  <n',l'> : listn(A) |] ==> \
 \           <n#+n', l@l'> : listn(A)";
-by (etac listn_induct 1);
+by (etac listn.induct 1);
 by (ALLGOALS (asm_simp_tac (list_ss addsimps listn.intrs)));
 qed "listn_append";