changeset 76217 | 8655344f1cf6 |
parent 76215 | a642599ffdea |
child 76987 | 4c275405faae |
--- a/src/ZF/Induct/ListN.thy Tue Sep 27 17:54:20 2022 +0100 +++ b/src/ZF/Induct/ListN.thy Tue Sep 27 18:02:34 2022 +0100 @@ -37,7 +37,7 @@ done lemma listn_mono: "A \<subseteq> B \<Longrightarrow> listn(A) \<subseteq> listn(B)" - apply (unfold listn.defs) + unfolding listn.defs apply (rule lfp_mono) apply (rule listn.bnd_mono)+ apply (assumption | rule univ_mono Sigma_mono list_mono basic_monos)+