# HG changeset patch # User paulson # Date 979121798 -3600 # Node ID 49868b703e4d3e2f3b36e5adb5131f826af4b891 # Parent 31ac62e3a0ed6710419a65bb5593aa952292044b deleted the obsolete nat_neqE (and reformatting) diff -r 31ac62e3a0ed -r 49868b703e4d src/HOL/UNITY/Counter.ML --- a/src/HOL/UNITY/Counter.ML Wed Jan 10 11:15:24 2001 +0100 +++ b/src/HOL/UNITY/Counter.ML Wed Jan 10 11:16:38 2001 +0100 @@ -61,9 +61,7 @@ Goal "ALL i. i(sum I s = s (c i) + sumj I i s)"; by (induct_tac "I" 1); -by Auto_tac; -by (etac nat_neqE 1); -by (ALLGOALS(asm_simp_tac (simpset() addsimps [sumj_sum_eq]))); +by (auto_tac (claset(), simpset() addsimps [linorder_neq_iff, sumj_sum_eq])); qed_spec_mp "sum_sumj"; (* Correctness proofs for Components *) diff -r 31ac62e3a0ed -r 49868b703e4d src/HOL/UNITY/Counterc.ML --- a/src/HOL/UNITY/Counterc.ML Wed Jan 10 11:15:24 2001 +0100 +++ b/src/HOL/UNITY/Counterc.ML Wed Jan 10 11:16:38 2001 +0100 @@ -24,17 +24,14 @@ Goal "i sum I s = c s i + sumj I i s"; by (induct_tac "I" 1); -by (auto_tac (claset() addSEs [nat_neqE], - simpset() addsimps [sum_sumj_eq1])); +by (auto_tac (claset(), simpset() addsimps [linorder_neq_iff, sum_sumj_eq1])); qed_spec_mp "sum_sumj_eq2"; -Goal -"(ALL i. i c s' i = c s i) --> (sum I s' = sum I s)"; +Goal "(ALL i. i c s' i = c s i) --> (sum I s' = sum I s)"; by (induct_tac "I" 1 THEN Auto_tac); qed_spec_mp "sum_ext"; -Goal -"(ALL j. j c s' j = c s j) --> (sumj I i s' = sumj I i s)"; +Goal "(ALL j. j c s' j = c s j) --> (sumj I i s' = sumj I i s)"; by (induct_tac "I" 1); by Safe_tac; by (auto_tac (claset() addSIs [sum_ext], simpset())); @@ -52,7 +49,7 @@ Goal "(Component i ok G) = \ \ (G: preserves (%s. c s i) & Component i:Allowed G)"; by (auto_tac (claset(), - simpset() addsimps [ok_iff_Allowed, Component_def RS def_prg_Allowed])); + simpset() addsimps [ok_iff_Allowed, Component_def RS def_prg_Allowed])); qed "Component_ok_iff"; AddIffs [Component_ok_iff]; AddIffs [OK_iff_ok]; @@ -63,9 +60,8 @@ by (constrains_tac 1); qed "p2"; -Goal -"[| OK I Component; i:I |] ==> \ -\ Component i: stable {s. ALL j:I. j~=i --> c s j = c k j}"; +Goal "[| OK I Component; i:I |] \ +\ ==> Component i: stable {s. ALL j:I. j~=i --> c s j = c k j}"; by (full_simp_tac (simpset() addsimps [stable_def, constrains_def]) 1); by (Blast_tac 1); qed "p3"; @@ -79,26 +75,24 @@ qed "p2_p3_lemma1"; -Goal -"(ALL k. F:stable ({s. C s = (c s) i + sumj I i k} Int \ -\ {s. ALL j:{i. i c s j = c k j})) ==> \ -\ (F:stable {s. C s = c s i + sumj I i s})"; +Goal "(ALL k. F:stable ({s. C s = (c s) i + sumj I i k} Int \ +\ {s. ALL j:{i. i c s j = c k j})) \ +\ ==> (F:stable {s. C s = c s i + sumj I i s})"; by (full_simp_tac (simpset() addsimps [constrains_def, stable_def]) 1); by (force_tac (claset() addSIs [sumj_ext], simpset()) 1); qed "p2_p3_lemma2"; -Goal -"[| OK {i. i \ -\ Component i: stable {s. C s = c s i + sumj I i s}"; +Goal "[| OK {i. i Component i: stable {s. C s = c s i + sumj I i s}"; by (blast_tac (claset() addIs [p2_p3_lemma1 RS p2_p3_lemma2]) 1); qed "p2_p3"; (* Compositional correctness *) Goalw [invariant_def] - "[| 0 \ -\ (JN i:{i. i (JN i:{i. i