src/ZF/Induct/Term.thy
changeset 76216 9fc34f76b4e8
parent 76215 a642599ffdea
child 76217 8655344f1cf6
--- a/src/ZF/Induct/Term.thy	Tue Sep 27 17:46:52 2022 +0100
+++ b/src/ZF/Induct/Term.thy	Tue Sep 27 17:54:20 2022 +0100
@@ -169,7 +169,7 @@
 
 lemma term_map_type [TC]:
     "\<lbrakk>t \<in> term(A);  \<And>x. x \<in> A \<Longrightarrow> f(x): B\<rbrakk> \<Longrightarrow> term_map(f,t) \<in> term(B)"
-  apply (unfold term_map_def)
+    unfolding term_map_def
   apply (erule term_rec_simple_type)
   apply fast
   done