diff -r a642599ffdea -r 9fc34f76b4e8 src/ZF/Ordinal.thy --- a/src/ZF/Ordinal.thy Tue Sep 27 17:46:52 2022 +0100 +++ b/src/ZF/Ordinal.thy Tue Sep 27 17:54:20 2022 +0100 @@ -40,7 +40,7 @@ by (unfold Transset_def, blast) lemma Transset_iff_Union_succ: "Transset(A) <-> \(succ(A)) = A" -apply (unfold Transset_def) + unfolding Transset_def apply (blast elim!: equalityE) done @@ -157,12 +157,12 @@ by (blast intro: Ord_succ dest!: Ord_succD) lemma Ord_Un [intro,simp,TC]: "\Ord(i); Ord(j)\ \ Ord(i \ j)" -apply (unfold Ord_def) + unfolding Ord_def apply (blast intro!: Transset_Un) done lemma Ord_Int [TC]: "\Ord(i); Ord(j)\ \ Ord(i \ j)" -apply (unfold Ord_def) + unfolding Ord_def apply (blast intro!: Transset_Int) done @@ -188,7 +188,7 @@ lemma ltE: "\ii\j; Ord(i); Ord(j)\ \ P\ \ P" -apply (unfold lt_def) + unfolding lt_def apply (blast intro: Ord_in_Ord) done @@ -214,7 +214,7 @@ by (blast intro!: ltI elim!: ltE intro: Ord_trans) lemma lt_not_sym: "i \ (jLimit Ordinals -- General Properties\ lemma Limit_Union_eq: "Limit(i) \ \(i) = i" -apply (unfold Limit_def) + unfolding Limit_def apply (fast intro!: ltI elim!: ltE elim: Ord_trans) done lemma Limit_is_Ord: "Limit(i) \ Ord(i)" -apply (unfold Limit_def) + unfolding Limit_def apply (erule conjunct1) done lemma Limit_has_0: "Limit(i) \ 0 < i" -apply (unfold Limit_def) + unfolding Limit_def apply (erule conjunct2 [THEN conjunct1]) done