src/ZF/Induct/Rmap.thy
changeset 76217 8655344f1cf6
parent 76216 9fc34f76b4e8
--- a/src/ZF/Induct/Rmap.thy	Tue Sep 27 17:54:20 2022 +0100
+++ b/src/ZF/Induct/Rmap.thy	Tue Sep 27 18:02:34 2022 +0100
@@ -21,7 +21,7 @@
   type_intros domainI rangeI list.intros
 
 lemma rmap_mono: "r \<subseteq> s \<Longrightarrow> rmap(r) \<subseteq> rmap(s)"
-  apply (unfold rmap.defs)
+    unfolding rmap.defs
   apply (rule lfp_mono)
     apply (rule rmap.bnd_mono)+
   apply (assumption | rule Sigma_mono list_mono domain_mono range_mono basic_monos)+