diff -r 33147ecac5f9 -r a1ba833d6b61 src/ZF/UNITY/Follows.thy --- a/src/ZF/UNITY/Follows.thy Wed Jul 09 12:41:47 2003 +0200 +++ b/src/ZF/UNITY/Follows.thy Thu Jul 10 17:14:41 2003 +0200 @@ -274,26 +274,33 @@ \x \ state. g(x):A |] ==> F \ Follows(A, r, g, h)" apply (unfold Follows_def Increasing_def Stable_def) apply (simp add: INT_iff, auto) -apply (rule_tac [3] C = "{s \ state. f (s) =g (s) }" and A = "{s \ state. \ r}" and A' = "{s \ state. \ r}" in Always_LeadsTo_weaken) -apply (erule_tac A = "{s \ state. \ r}" and A' = "{s \ state. \ r}" in Always_Constrains_weaken) +apply (rule_tac [3] C = "{s \ state. f(s)=g(s)}" + and A = "{s \ state. \ r}" + and A' = "{s \ state. \ r}" in Always_LeadsTo_weaken) +apply (erule_tac A = "{s \ state. \ r}" + and A' = "{s \ state. \ r}" in Always_Constrains_weaken) apply auto apply (drule Always_Int_I, assumption) -apply (erule_tac A = "{s \ state . f (s) = g (s) } \ {s \ state . \f (s), h (s) \ \ r}" in Always_weaken) +apply (erule_tac A = "{s \ state. f(s)=g(s)} \ {s \ state. \ r}" + in Always_weaken) apply auto done + lemma Always_Follows2: "[| F \ Always({s \ state. g(s) = h(s)}); F \ Follows(A, r, f, g); \x \ state. h(x):A |] ==> F \ Follows(A, r, f, h)" apply (unfold Follows_def Increasing_def Stable_def) -apply (simp (no_asm_use) add: INT_iff) -apply auto -apply (erule_tac [3] V = "k \ A" in thin_rl) -apply (rule_tac [3] C = "{s \ state. g (s) =h (s) }" and A = "{s \ state. \ r}" and A' = "{s \ state. \ r}" in Always_LeadsTo_weaken) -apply (erule_tac A = "{s \ state. \ r}" and A' = "{s \ state. \ r}" in Always_Constrains_weaken) +apply (simp add: INT_iff, auto) +apply (rule_tac [3] C = "{s \ state. g (s) =h (s) }" + and A = "{s \ state. \ r}" + and A' = "{s \ state. \ r}" in Always_LeadsTo_weaken) +apply (erule_tac A = "{s \ state. \ r}" + and A' = "{s \ state. \ r}" in Always_Constrains_weaken) apply auto apply (drule Always_Int_I, assumption) -apply (erule_tac A = "{s \ state . g (s) = h (s) } \ {s \ state . \f (s), g (s) \ \ r}" in Always_weaken) +apply (erule_tac A = "{s \ state. g(s)=h(s)} \ {s \ state. \ r}" + in Always_weaken) apply auto done