diff -r 880f31a62784 -r 281d44905cab src/HOL/UNITY/SubstAx.ML --- a/src/HOL/UNITY/SubstAx.ML Wed Apr 28 13:36:31 1999 +0200 +++ b/src/HOL/UNITY/SubstAx.ML Thu Apr 29 10:51:58 1999 +0200 @@ -6,21 +6,21 @@ LeadsTo relation, restricted to the set of reachable states. *) -overload_1st_set "SubstAx.LeadsTo"; +overload_1st_set "SubstAx.op LeadsTo"; (*** Specialized laws for handling invariants ***) (** Conjoining a safety property **) -Goal "[| reachable F <= C; F : LeadsTo (C Int A) A' |] \ -\ ==> F : LeadsTo A A'"; +Goal "[| reachable F <= C; F : (C Int A) LeadsTo A' |] \ +\ ==> F : A LeadsTo A'"; by (asm_full_simp_tac (simpset() addsimps [LeadsTo_def, Int_absorb2, Int_assoc RS sym]) 1); qed "reachable_LeadsToI"; -Goal "[| reachable F <= C; F : LeadsTo A A' |] \ -\ ==> F : LeadsTo A (C Int A')"; +Goal "[| reachable F <= C; F : A LeadsTo A' |] \ +\ ==> F : A LeadsTo (C Int A')"; by (asm_full_simp_tac (simpset() addsimps [LeadsTo_def, Int_absorb2, Int_assoc RS sym]) 1); @@ -29,11 +29,11 @@ (** Conjoining an invariant **) -(* [| Invariant F C; F : LeadsTo (C Int A) A' |] ==> F : LeadsTo A A' *) +(* [| Invariant F C; F : (C Int A) LeadsTo A' |] ==> F : A LeadsTo A' *) bind_thm ("Invariant_LeadsToI", Invariant_includes_reachable RS reachable_LeadsToI); -(* [| Invariant F C; F : LeadsTo A A' |] ==> F : LeadsTo A (C Int A') *) +(* [| Invariant F C; F : A LeadsTo A' |] ==> F : A LeadsTo (C Int A') *) bind_thm ("Invariant_LeadsToD", Invariant_includes_reachable RS reachable_LeadsToD); @@ -42,18 +42,18 @@ (*** Introduction rules: Basis, Trans, Union ***) -Goal "F : leadsTo A B ==> F : LeadsTo A B"; +Goal "F : A leadsTo B ==> F : A LeadsTo B"; by (simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (blast_tac (claset() addIs [psp_stable2, stable_reachable]) 1); qed "leadsTo_imp_LeadsTo"; -Goal "[| F : LeadsTo A B; F : LeadsTo B C |] ==> F : LeadsTo A C"; +Goal "[| F : A LeadsTo B; F : B LeadsTo C |] ==> F : A LeadsTo C"; by (full_simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (blast_tac (claset() addIs [leadsTo_Trans]) 1); qed "LeadsTo_Trans"; val prems = Goalw [LeadsTo_def] - "(!!A. A : S ==> F : LeadsTo A B) ==> F : LeadsTo (Union S) B"; + "(!!A. A : S ==> F : A LeadsTo B) ==> F : (Union S) LeadsTo B"; by (Simp_tac 1); by (stac Int_Union 1); by (blast_tac (claset() addIs [leadsTo_UN] addDs prems) 1); @@ -62,34 +62,34 @@ (*** Derived rules ***) -Goal "F : LeadsTo A UNIV"; +Goal "F : A LeadsTo UNIV"; by (asm_simp_tac (simpset() addsimps [LeadsTo_def, Int_lower1 RS subset_imp_leadsTo]) 1); qed "LeadsTo_UNIV"; Addsimps [LeadsTo_UNIV]; (*Useful with cancellation, disjunction*) -Goal "F : LeadsTo A (A' Un A') ==> F : LeadsTo A A'"; +Goal "F : A LeadsTo (A' Un A') ==> F : A LeadsTo A'"; by (asm_full_simp_tac (simpset() addsimps Un_ac) 1); qed "LeadsTo_Un_duplicate"; -Goal "F : LeadsTo A (A' Un C Un C) ==> F : LeadsTo A (A' Un C)"; +Goal "F : A LeadsTo (A' Un C Un C) ==> F : A LeadsTo (A' Un C)"; by (asm_full_simp_tac (simpset() addsimps Un_ac) 1); qed "LeadsTo_Un_duplicate2"; val prems = -Goal "(!!i. i : I ==> F : LeadsTo (A i) B) ==> F : LeadsTo (UN i:I. A i) B"; +Goal "(!!i. i : I ==> F : (A i) LeadsTo B) ==> F : (UN i:I. A i) LeadsTo B"; by (simp_tac (HOL_ss addsimps [Union_image_eq RS sym]) 1); by (blast_tac (claset() addIs (LeadsTo_Union::prems)) 1); qed "LeadsTo_UN"; (*Binary union introduction rule*) -Goal "[| F : LeadsTo A C; F : LeadsTo B C |] ==> F : LeadsTo (A Un B) C"; +Goal "[| F : A LeadsTo C; F : B LeadsTo C |] ==> F : (A Un B) LeadsTo C"; by (stac Un_eq_Union 1); by (blast_tac (claset() addIs [LeadsTo_Union]) 1); qed "LeadsTo_Un"; -Goal "A <= B ==> F : LeadsTo A B"; +Goal "A <= B ==> F : A LeadsTo B"; by (simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (blast_tac (claset() addIs [subset_imp_leadsTo]) 1); qed "subset_imp_LeadsTo"; @@ -97,39 +97,39 @@ bind_thm ("empty_LeadsTo", empty_subsetI RS subset_imp_LeadsTo); Addsimps [empty_LeadsTo]; -Goal "[| F : LeadsTo A A'; A' <= B' |] ==> F : LeadsTo A B'"; +Goal "[| F : A LeadsTo A'; A' <= B' |] ==> F : A LeadsTo B'"; by (full_simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (blast_tac (claset() addIs [leadsTo_weaken_R]) 1); qed_spec_mp "LeadsTo_weaken_R"; -Goal "[| F : LeadsTo A A'; B <= A |] \ -\ ==> F : LeadsTo B A'"; +Goal "[| F : A LeadsTo A'; B <= A |] \ +\ ==> F : B LeadsTo A'"; by (full_simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (blast_tac (claset() addIs [leadsTo_weaken_L]) 1); qed_spec_mp "LeadsTo_weaken_L"; -Goal "[| F : LeadsTo A A'; \ +Goal "[| F : A LeadsTo A'; \ \ B <= A; A' <= B' |] \ -\ ==> F : LeadsTo B B'"; +\ ==> F : B LeadsTo B'"; by (blast_tac (claset() addIs [LeadsTo_weaken_R, LeadsTo_weaken_L, LeadsTo_Trans]) 1); qed "LeadsTo_weaken"; -Goal "[| reachable F <= C; F : LeadsTo A A'; \ +Goal "[| reachable F <= C; F : A LeadsTo A'; \ \ C Int B <= A; C Int A' <= B' |] \ -\ ==> F : LeadsTo B B'"; +\ ==> F : B LeadsTo B'"; by (blast_tac (claset() addDs [reachable_LeadsToI] addIs[LeadsTo_weaken] addIs [reachable_LeadsToD]) 1); qed "reachable_LeadsTo_weaken"; (** Two theorems for "proof lattices" **) -Goal "[| F : LeadsTo A B |] ==> F : LeadsTo (A Un B) B"; +Goal "[| F : A LeadsTo B |] ==> F : (A Un B) LeadsTo B"; by (blast_tac (claset() addIs [LeadsTo_Un, subset_imp_LeadsTo]) 1); qed "LeadsTo_Un_post"; -Goal "[| F : LeadsTo A B; F : LeadsTo B C |] \ -\ ==> F : LeadsTo (A Un B) C"; +Goal "[| F : A LeadsTo B; F : B LeadsTo C |] \ +\ ==> F : (A Un B) LeadsTo C"; by (blast_tac (claset() addIs [LeadsTo_Un, subset_imp_LeadsTo, LeadsTo_weaken_L, LeadsTo_Trans]) 1); qed "LeadsTo_Trans_Un"; @@ -137,23 +137,23 @@ (** Distributive laws **) -Goal "(F : LeadsTo (A Un B) C) = (F : LeadsTo A C & F : LeadsTo B C)"; +Goal "(F : (A Un B) LeadsTo C) = (F : A LeadsTo C & F : B LeadsTo C)"; by (blast_tac (claset() addIs [LeadsTo_Un, LeadsTo_weaken_L]) 1); qed "LeadsTo_Un_distrib"; -Goal "(F : LeadsTo (UN i:I. A i) B) = (ALL i : I. F : LeadsTo (A i) B)"; +Goal "(F : (UN i:I. A i) LeadsTo B) = (ALL i : I. F : (A i) LeadsTo B)"; by (blast_tac (claset() addIs [LeadsTo_UN, LeadsTo_weaken_L]) 1); qed "LeadsTo_UN_distrib"; -Goal "(F : LeadsTo (Union S) B) = (ALL A : S. F : LeadsTo A B)"; +Goal "(F : (Union S) LeadsTo B) = (ALL A : S. F : A LeadsTo B)"; by (blast_tac (claset() addIs [LeadsTo_Union, LeadsTo_weaken_L]) 1); qed "LeadsTo_Union_distrib"; (** More rules using the premise "Invariant F" **) -Goal "[| F : Constrains (A-A') (A Un A'); F : transient (A-A') |] \ -\ ==> F : LeadsTo A A'"; +Goal "[| F : (A-A') Co (A Un A'); F : transient (A-A') |] \ +\ ==> F : A LeadsTo A'"; by (asm_full_simp_tac (simpset() addsimps [LeadsTo_def, Constrains_def]) 1); by (rtac (ensuresI RS leadsTo_Basis) 1); by (blast_tac (claset() addIs [transient_strengthen]) 2); @@ -161,9 +161,9 @@ qed "LeadsTo_Basis"; Goal "[| F : Invariant INV; \ -\ F : Constrains (INV Int (A-A')) (A Un A'); \ +\ F : (INV Int (A-A')) Co (A Un A'); \ \ F : transient (INV Int (A-A')) |] \ -\ ==> F : LeadsTo A A'"; +\ ==> F : A LeadsTo A'"; by (rtac Invariant_LeadsToI 1); by (assume_tac 1); by (rtac LeadsTo_Basis 1); @@ -172,8 +172,8 @@ qed "Invariant_LeadsTo_Basis"; Goal "[| F : Invariant INV; \ -\ F : LeadsTo A A'; INV Int B <= A; INV Int A' <= B' |] \ -\ ==> F : LeadsTo B B'"; +\ F : A LeadsTo A'; INV Int B <= A; INV Int A' <= B' |] \ +\ ==> F : B LeadsTo B'"; by (REPEAT (ares_tac [Invariant_includes_reachable, reachable_LeadsTo_weaken] 1)); qed "Invariant_LeadsTo_weaken"; @@ -181,15 +181,15 @@ (*Set difference: maybe combine with leadsTo_weaken_L?? This is the most useful form of the "disjunction" rule*) -Goal "[| F : LeadsTo (A-B) C; F : LeadsTo (A Int B) C |] \ -\ ==> F : LeadsTo A C"; +Goal "[| F : (A-B) LeadsTo C; F : (A Int B) LeadsTo C |] \ +\ ==> F : A LeadsTo C"; by (blast_tac (claset() addIs [LeadsTo_Un, LeadsTo_weaken]) 1); qed "LeadsTo_Diff"; val prems = -Goal "(!! i. i:I ==> F : LeadsTo (A i) (A' i)) \ -\ ==> F : LeadsTo (UN i:I. A i) (UN i:I. A' i)"; +Goal "(!! i. i:I ==> F : (A i) LeadsTo (A' i)) \ +\ ==> F : (UN i:I. A i) LeadsTo (UN i:I. A' i)"; by (simp_tac (HOL_ss addsimps [Union_image_eq RS sym]) 1); by (blast_tac (claset() addIs [LeadsTo_Union, LeadsTo_weaken_R] addIs prems) 1); @@ -198,22 +198,22 @@ (*Version with no index set*) val prems = -Goal "(!! i. F : LeadsTo (A i) (A' i)) \ -\ ==> F : LeadsTo (UN i. A i) (UN i. A' i)"; +Goal "(!! i. F : (A i) LeadsTo (A' i)) \ +\ ==> F : (UN i. A i) LeadsTo (UN i. A' i)"; by (blast_tac (claset() addIs [LeadsTo_UN_UN] addIs prems) 1); qed "LeadsTo_UN_UN_noindex"; (*Version with no index set*) -Goal "ALL i. F : LeadsTo (A i) (A' i) \ -\ ==> F : LeadsTo (UN i. A i) (UN i. A' i)"; +Goal "ALL i. F : (A i) LeadsTo (A' i) \ +\ ==> F : (UN i. A i) LeadsTo (UN i. A' i)"; by (blast_tac (claset() addIs [LeadsTo_UN_UN]) 1); qed "all_LeadsTo_UN_UN"; (*Binary union version*) -Goal "[| F : LeadsTo A A'; F : LeadsTo B B' |] \ -\ ==> F : LeadsTo (A Un B) (A' Un B')"; +Goal "[| F : A LeadsTo A'; F : B LeadsTo B' |] \ +\ ==> F : (A Un B) LeadsTo (A' Un B')"; by (blast_tac (claset() addIs [LeadsTo_Un, LeadsTo_weaken_R]) 1); qed "LeadsTo_Un_Un"; @@ -221,27 +221,27 @@ (** The cancellation law **) -Goal "[| F : LeadsTo A (A' Un B); F : LeadsTo B B' |] \ -\ ==> F : LeadsTo A (A' Un B')"; +Goal "[| F : A LeadsTo (A' Un B); F : B LeadsTo B' |] \ +\ ==> F : A LeadsTo (A' Un B')"; by (blast_tac (claset() addIs [LeadsTo_Un_Un, subset_imp_LeadsTo, LeadsTo_Trans]) 1); qed "LeadsTo_cancel2"; -Goal "[| F : LeadsTo A (A' Un B); F : LeadsTo (B-A') B' |] \ -\ ==> F : LeadsTo A (A' Un B')"; +Goal "[| F : A LeadsTo (A' Un B); F : (B-A') LeadsTo B' |] \ +\ ==> F : A LeadsTo (A' Un B')"; by (rtac LeadsTo_cancel2 1); by (assume_tac 2); by (ALLGOALS Asm_simp_tac); qed "LeadsTo_cancel_Diff2"; -Goal "[| F : LeadsTo A (B Un A'); F : LeadsTo B B' |] \ -\ ==> F : LeadsTo A (B' Un A')"; +Goal "[| F : A LeadsTo (B Un A'); F : B LeadsTo B' |] \ +\ ==> F : A LeadsTo (B' Un A')"; by (asm_full_simp_tac (simpset() addsimps [Un_commute]) 1); by (blast_tac (claset() addSIs [LeadsTo_cancel2]) 1); qed "LeadsTo_cancel1"; -Goal "[| F : LeadsTo A (B Un A'); F : LeadsTo (B-A') B' |] \ -\ ==> F : LeadsTo A (B' Un A')"; +Goal "[| F : A LeadsTo (B Un A'); F : (B-A') LeadsTo B' |] \ +\ ==> F : A LeadsTo (B' Un A')"; by (rtac LeadsTo_cancel1 1); by (assume_tac 2); by (ALLGOALS Asm_simp_tac); @@ -251,7 +251,7 @@ (** The impossibility law **) (*The set "A" may be non-empty, but it contains no reachable states*) -Goal "F : LeadsTo A {} ==> reachable F Int A = {}"; +Goal "F : A LeadsTo {} ==> reachable F Int A = {}"; by (full_simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (etac leadsTo_empty 1); qed "LeadsTo_empty"; @@ -260,33 +260,33 @@ (** PSP: Progress-Safety-Progress **) (*Special case of PSP: Misra's "stable conjunction"*) -Goal "[| F : LeadsTo A A'; F : Stable B |] \ -\ ==> F : LeadsTo (A Int B) (A' Int B)"; +Goal "[| F : A LeadsTo A'; F : Stable B |] \ +\ ==> F : (A Int B) LeadsTo (A' Int B)"; by (full_simp_tac (simpset() addsimps [LeadsTo_def, Stable_eq_stable]) 1); by (dtac psp_stable 1); by (assume_tac 1); by (asm_full_simp_tac (simpset() addsimps Int_ac) 1); qed "PSP_stable"; -Goal "[| F : LeadsTo A A'; F : Stable B |] \ -\ ==> F : LeadsTo (B Int A) (B Int A')"; +Goal "[| F : A LeadsTo A'; F : Stable B |] \ +\ ==> F : (B Int A) LeadsTo (B Int A')"; by (asm_simp_tac (simpset() addsimps PSP_stable::Int_ac) 1); qed "PSP_stable2"; Goalw [LeadsTo_def, Constrains_def] - "[| F : LeadsTo A A'; F : Constrains B B' |] \ -\ ==> F : LeadsTo (A Int B) ((A' Int B) Un (B' - B))"; + "[| F : A LeadsTo A'; F : B Co B' |] \ +\ ==> F : (A Int B) LeadsTo ((A' Int B) Un (B' - B))"; by (blast_tac (claset() addDs [psp] addIs [leadsTo_weaken]) 1); qed "PSP"; -Goal "[| F : LeadsTo A A'; F : Constrains B B' |] \ -\ ==> F : LeadsTo (B Int A) ((B Int A') Un (B' - B))"; +Goal "[| F : A LeadsTo A'; F : B Co B' |] \ +\ ==> F : (B Int A) LeadsTo ((B Int A') Un (B' - B))"; by (asm_simp_tac (simpset() addsimps PSP::Int_ac) 1); qed "PSP2"; Goalw [Unless_def] - "[| F : LeadsTo A A'; F : Unless B B' |] \ -\ ==> F : LeadsTo (A Int B) ((A' Int B) Un B')"; + "[| F : A LeadsTo A'; F : B Unless B' |] \ +\ ==> F : (A Int B) LeadsTo ((A' Int B) Un B')"; by (dtac PSP 1); by (assume_tac 1); by (blast_tac (claset() addIs [LeadsTo_Diff, LeadsTo_weaken, @@ -295,7 +295,7 @@ Goal "[| F : Stable A; F : transient C; \ -\ reachable F <= (-A Un B Un C) |] ==> F : LeadsTo A B"; +\ reachable F <= (-A Un B Un C) |] ==> F : A LeadsTo B"; by (etac reachable_LeadsTo_weaken 1); by (rtac LeadsTo_Diff 1); by (etac (transient_imp_leadsTo RS leadsTo_imp_LeadsTo RS PSP_stable2) 2); @@ -307,9 +307,9 @@ (** Meta or object quantifier ????? **) Goal "[| wf r; \ -\ ALL m. F : LeadsTo (A Int f-``{m}) \ +\ ALL m. F : (A Int f-``{m}) LeadsTo \ \ ((A Int f-``(r^-1 ^^ {m})) Un B) |] \ -\ ==> F : LeadsTo A B"; +\ ==> F : A LeadsTo B"; by (full_simp_tac (simpset() addsimps [LeadsTo_def]) 1); by (etac leadsTo_wf_induct 1); by (blast_tac (claset() addIs [leadsTo_weaken]) 1); @@ -317,9 +317,9 @@ Goal "[| wf r; \ -\ ALL m:I. F : LeadsTo (A Int f-``{m}) \ +\ ALL m:I. F : (A Int f-``{m}) LeadsTo \ \ ((A Int f-``(r^-1 ^^ {m})) Un B) |] \ -\ ==> F : LeadsTo A ((A - (f-``I)) Un B)"; +\ ==> F : A LeadsTo ((A - (f-``I)) Un B)"; by (etac LeadsTo_wf_induct 1); by Safe_tac; by (case_tac "m:I" 1); @@ -328,9 +328,9 @@ qed "Bounded_induct"; -Goal "[| ALL m. F : LeadsTo (A Int f-``{m}) \ +Goal "[| ALL m. F : (A Int f-``{m}) LeadsTo \ \ ((A Int f-``(lessThan m)) Un B) |] \ -\ ==> F : LeadsTo A B"; +\ ==> F : A LeadsTo B"; by (rtac (wf_less_than RS LeadsTo_wf_induct) 1); by (Asm_simp_tac 1); qed "LessThan_induct"; @@ -338,26 +338,26 @@ (*Integer version. Could generalize from #0 to any lower bound*) val [reach, prem] = Goal "[| reachable F <= {s. #0 <= f s}; \ -\ !! z. F : LeadsTo (A Int {s. f s = z}) \ +\ !! z. F : (A Int {s. f s = z}) LeadsTo \ \ ((A Int {s. f s < z}) Un B) |] \ -\ ==> F : LeadsTo A B"; +\ ==> F : A LeadsTo B"; by (res_inst_tac [("f", "nat o f")] (allI RS LessThan_induct) 1); by (simp_tac (simpset() addsimps [vimage_def]) 1); by (rtac ([reach, prem] MRS reachable_LeadsTo_weaken) 1); by (auto_tac (claset(), simpset() addsimps [nat_eq_iff, nat_less_iff])); qed "integ_0_le_induct"; -Goal "[| ALL m:(greaterThan l). F : LeadsTo (A Int f-``{m}) \ +Goal "[| ALL m:(greaterThan l). F : (A Int f-``{m}) LeadsTo \ \ ((A Int f-``(lessThan m)) Un B) |] \ -\ ==> F : LeadsTo A ((A Int (f-``(atMost l))) Un B)"; +\ ==> F : A LeadsTo ((A Int (f-``(atMost l))) Un B)"; by (simp_tac (HOL_ss addsimps [Diff_eq RS sym, vimage_Compl, Compl_greaterThan RS sym]) 1); by (rtac (wf_less_than RS Bounded_induct) 1); by (Asm_simp_tac 1); qed "LessThan_bounded_induct"; -Goal "[| ALL m:(lessThan l). F : LeadsTo (A Int f-``{m}) \ +Goal "[| ALL m:(lessThan l). F : (A Int f-``{m}) LeadsTo \ \ ((A Int f-``(greaterThan m)) Un B) |] \ -\ ==> F : LeadsTo A ((A Int (f-``(atLeast l))) Un B)"; +\ ==> F : A LeadsTo ((A Int (f-``(atLeast l))) Un B)"; by (res_inst_tac [("f","f"),("f1", "%k. l - k")] (wf_less_than RS wf_inv_image RS LeadsTo_wf_induct) 1); by (simp_tac (simpset() addsimps [inv_image_def, Image_singleton]) 1); @@ -370,27 +370,27 @@ (*** Completion: Binary and General Finite versions ***) -Goal "[| F : LeadsTo A A'; F : Stable A'; \ -\ F : LeadsTo B B'; F : Stable B' |] \ -\ ==> F : LeadsTo (A Int B) (A' Int B')"; +Goal "[| F : A LeadsTo A'; F : Stable A'; \ +\ F : B LeadsTo B'; F : Stable B' |] \ +\ ==> F : (A Int B) LeadsTo (A' Int B')"; by (full_simp_tac (simpset() addsimps [LeadsTo_def, Stable_eq_stable]) 1); by (blast_tac (claset() addIs [stable_completion, leadsTo_weaken]) 1); qed "Stable_completion"; Goal "finite I \ -\ ==> (ALL i:I. F : LeadsTo (A i) (A' i)) --> \ +\ ==> (ALL i:I. F : (A i) LeadsTo (A' i)) --> \ \ (ALL i:I. F : Stable (A' i)) --> \ -\ F : LeadsTo (INT i:I. A i) (INT i:I. A' i)"; +\ F : (INT i:I. A i) LeadsTo (INT i:I. A' i)"; by (etac finite_induct 1); by (Asm_simp_tac 1); by (asm_simp_tac (simpset() addsimps [Stable_completion, ball_Stable_INT]) 1); qed_spec_mp "Finite_stable_completion"; -Goal "[| F : LeadsTo A (A' Un C); F : Constrains A' (A' Un C); \ -\ F : LeadsTo B (B' Un C); F : Constrains B' (B' Un C) |] \ -\ ==> F : LeadsTo (A Int B) ((A' Int B') Un C)"; +Goal "[| F : A LeadsTo (A' Un C); F : A' Co (A' Un C); \ +\ F : B LeadsTo (B' Un C); F : B' Co (B' Un C) |] \ +\ ==> F : (A Int B) LeadsTo ((A' Int B') Un C)"; by (full_simp_tac (simpset() addsimps [LeadsTo_def, Constrains_def, Int_Un_distrib]) 1); by (blast_tac (claset() addIs [completion, leadsTo_weaken]) 1); @@ -398,9 +398,9 @@ Goal "[| finite I |] \ -\ ==> (ALL i:I. F : LeadsTo (A i) (A' i Un C)) --> \ -\ (ALL i:I. F : Constrains (A' i) (A' i Un C)) --> \ -\ F : LeadsTo (INT i:I. A i) ((INT i:I. A' i) Un C)"; +\ ==> (ALL i:I. F : (A i) LeadsTo (A' i Un C)) --> \ +\ (ALL i:I. F : (A' i) Co (A' i Un C)) --> \ +\ F : (INT i:I. A i) LeadsTo ((INT i:I. A' i) Un C)"; by (etac finite_induct 1); by (ALLGOALS Asm_simp_tac); by (Clarify_tac 1); @@ -416,7 +416,7 @@ etac Invariant_LeadsTo_Basis 1 ORELSE (*subgoal may involve LeadsTo, leadsTo or ensures*) REPEAT (ares_tac [LeadsTo_Basis, ensuresI] 1), - (*now there are two subgoals: constrains & transient*) + (*now there are two subgoals: co & transient*) simp_tac (simpset() addsimps !program_defs_ref) 2, res_inst_tac [("act", sact)] transient_mem 2, (*simplify the command's domain*)