changeset 76216 | 9fc34f76b4e8 |
parent 76215 | a642599ffdea |
child 76217 | 8655344f1cf6 |
--- a/src/ZF/Induct/Rmap.thy Tue Sep 27 17:46:52 2022 +0100 +++ b/src/ZF/Induct/Rmap.thy Tue Sep 27 17:54:20 2022 +0100 @@ -46,7 +46,7 @@ done lemma rmap_functional: "function(r) \<Longrightarrow> function(rmap(r))" - apply (unfold function_def) + unfolding function_def apply (rule impI [THEN allI, THEN allI]) apply (erule rmap.induct) apply blast+