diff -r a642599ffdea -r 9fc34f76b4e8 src/ZF/Trancl.thy --- a/src/ZF/Trancl.thy Tue Sep 27 17:46:52 2022 +0100 +++ b/src/ZF/Trancl.thy Tue Sep 27 17:54:20 2022 +0100 @@ -101,7 +101,7 @@ by (rule bnd_monoI, blast+) lemma rtrancl_mono: "r<=s \ r^* \ s^*" -apply (unfold rtrancl_def) + unfolding rtrancl_def apply (rule lfp_mono) apply (rule rtrancl_bnd_mono)+ apply blast @@ -172,7 +172,7 @@ (*transitivity of transitive closure\-- by induction.*) lemma trans_rtrancl: "trans(r^*)" -apply (unfold trans_def) + unfolding trans_def apply (intro allI impI) apply (erule_tac b = z in rtrancl_induct, assumption) apply (blast intro: rtrancl_into_rtrancl) @@ -208,13 +208,13 @@ (** Conversions between trancl and rtrancl **) lemma trancl_into_rtrancl: "\a,b\ \ r^+ \ \a,b\ \ r^*" -apply (unfold trancl_def) + unfolding trancl_def apply (blast intro: rtrancl_into_rtrancl) done (*r^+ contains all pairs in r *) lemma r_into_trancl: "\a,b\ \ r \ \a,b\ \ r^+" -apply (unfold trancl_def) + unfolding trancl_def apply (blast intro!: rtrancl_refl) done @@ -266,7 +266,7 @@ done lemma trancl_type: "r^+ \ field(r)*field(r)" -apply (unfold trancl_def) + unfolding trancl_def apply (blast elim: rtrancl_type [THEN subsetD, THEN SigmaE2]) done