diff -r a642599ffdea -r 9fc34f76b4e8 src/ZF/AC/Cardinal_aux.thy --- a/src/ZF/AC/Cardinal_aux.thy Tue Sep 27 17:46:52 2022 +0100 +++ b/src/ZF/AC/Cardinal_aux.thy Tue Sep 27 17:54:20 2022 +0100 @@ -99,7 +99,7 @@ by blast lemma UN_sing_lepoll: "Ord(a) \ (\x \ a. {P(x)}) \ a" -apply (unfold lepoll_def) + unfolding lepoll_def apply (rule_tac x = "\z \ (\x \ a. {P (x) }) . (\ i. P (i) =z) " in exI) apply (rule_tac d = "\z. P (z) " in lam_injective) apply (fast intro!: Least_in_Ord)