diff -r a642599ffdea -r 9fc34f76b4e8 src/ZF/Induct/Term.thy --- 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]: "\t \ term(A); \x. x \ A \ f(x): B\ \ term_map(f,t) \ term(B)" - apply (unfold term_map_def) + unfolding term_map_def apply (erule term_rec_simple_type) apply fast done