changeset 18415 | eb68dc98bda2 |
parent 16417 | 9bc16273c2d4 |
child 35762 | af3ff2ba4c54 |
--- a/src/ZF/Induct/ListN.thy Thu Dec 15 19:42:02 2005 +0100 +++ b/src/ZF/Induct/ListN.thy Thu Dec 15 19:42:03 2005 +0100 @@ -23,7 +23,7 @@ lemma list_into_listn: "l \<in> list(A) ==> <length(l),l> \<in> listn(A)" - by (erule list.induct) (simp_all add: listn.intros) + by (induct set: list) (simp_all add: listn.intros) lemma listn_iff: "<n,l> \<in> listn(A) <-> l \<in> list(A) & length(l)=n" apply (rule iffI)