| author | paulson | 
| Wed, 11 Jul 2001 10:50:18 +0200 | |
| changeset 11401 | 26cbf43d76af | 
| parent 9166 | 74d403974c8d | 
| child 12886 | 75ca1bf5ae12 | 
| permissions | -rw-r--r-- | 
| 4530 | 1 | (* Title: HOL/IOA/IOA.ML | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 2 | ID: $Id$ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 3 | Author: Tobias Nipkow & Konrad Slind | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 4 | Copyright 1994 TU Muenchen | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 5 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 6 | The I/O automata of Lynch and Tuttle. | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 7 | *) | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 8 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 9 | Addsimps [Let_def]; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 10 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 11 | val ioa_projections = [asig_of_def, starts_of_def, trans_of_def]; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 12 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 13 | val exec_rws = [executions_def,is_execution_fragment_def]; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 14 | |
| 5069 | 15 | Goal | 
| 8114 | 16 | "asig_of(x,y,z) = x & starts_of(x,y,z) = y & trans_of(x,y,z) = z"; | 
| 4089 | 17 | by (simp_tac (simpset() addsimps ioa_projections) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 18 | qed "ioa_triple_proj"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 19 | |
| 5069 | 20 | Goalw [ioa_def,state_trans_def,actions_def, is_asig_def] | 
| 5148 
74919e8f221c
More tidying and removal of "\!\!... from Goal commands
 paulson parents: 
5143diff
changeset | 21 | "[| IOA(A); (s1,a,s2):trans_of(A) |] ==> a:actions(asig_of(A))"; | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 22 | by (REPEAT(etac conjE 1)); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 23 | by (EVERY1[etac allE, etac impE, atac]); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 24 | by (Asm_full_simp_tac 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 25 | qed "trans_in_actions"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 26 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 27 | |
| 5069 | 28 | Goal "filter_oseq p (filter_oseq p s) = filter_oseq p s"; | 
| 4089 | 29 | by (simp_tac (simpset() addsimps [filter_oseq_def]) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 30 | by (rtac ext 1); | 
| 8442 
96023903c2df
case_tac now subsumes both boolean and datatype cases;
 wenzelm parents: 
8423diff
changeset | 31 | by (case_tac "s(i)" 1); | 
| 3346 | 32 | by (Asm_simp_tac 1); | 
| 4831 | 33 | by (Asm_simp_tac 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 34 | qed "filter_oseq_idemp"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 35 | |
| 5069 | 36 | Goalw [mk_trace_def,filter_oseq_def] | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 37 | "(mk_trace A s n = None) = \ | 
| 3346 | 38 | \ (s(n)=None | (? a. s(n)=Some(a) & a ~: externals(asig_of(A)))) \ | 
| 39 | \ & \ | |
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 40 | \ (mk_trace A s n = Some(a)) = \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 41 | \ (s(n)=Some(a) & a : externals(asig_of(A)))"; | 
| 8442 
96023903c2df
case_tac now subsumes both boolean and datatype cases;
 wenzelm parents: 
8423diff
changeset | 42 | by (case_tac "s(n)" 1); | 
| 4831 | 43 | by (ALLGOALS Asm_simp_tac); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 44 | by (Fast_tac 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 45 | qed "mk_trace_thm"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 46 | |
| 5143 
b94cd208f073
Removal of leading "\!\!..." from most Goal commands
 paulson parents: 
5132diff
changeset | 47 | Goalw [reachable_def] "s:starts_of(A) ==> reachable A s"; | 
| 3842 | 48 |   by (res_inst_tac [("x","(%i. None,%i. s)")] bexI 1);
 | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 49 | by (Simp_tac 1); | 
| 4089 | 50 | by (asm_simp_tac (simpset() addsimps exec_rws) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 51 | qed "reachable_0"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 52 | |
| 5069 | 53 | Goalw (reachable_def::exec_rws) | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 54 | "!!A. [| reachable A s; (s,a,t) : trans_of(A) |] ==> reachable A t"; | 
| 4089 | 55 | by (asm_full_simp_tac (simpset() delsimps bex_simps) 1); | 
| 4828 | 56 | by (split_all_tac 1); | 
| 5132 | 57 | by Safe_tac; | 
| 4828 | 58 | by (rename_tac "ex1 ex2 n" 1); | 
| 4772 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 59 |   by (res_inst_tac [("x","(%i. if i<n then ex1 i                    \
 | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 60 | \ else (if i=n then Some a else None), \ | 
| 4772 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 61 | \ %i. if i<Suc n then ex2 i else t)")] bexI 1); | 
| 4828 | 62 |    by (res_inst_tac [("x","Suc n")] exI 1);
 | 
| 4772 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 63 | by (Simp_tac 1); | 
| 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 64 | by (Asm_full_simp_tac 1); | 
| 4828 | 65 | by (rtac allI 1); | 
| 9166 | 66 |   by (cut_inst_tac [("m","na"),("n","n")] less_linear 1);
 | 
| 67 | by Auto_tac; | |
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 68 | qed "reachable_n"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 69 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 70 | val [p1,p2] = goalw IOA.thy [invariant_def] | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 71 | "[| !!s. s:starts_of(A) ==> P(s); \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 72 | \ !!s t a. [|reachable A s; P(s)|] ==> (s,a,t): trans_of(A) --> P(t) |] \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 73 | \ ==> invariant A P"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 74 | by (rewrite_goals_tac(reachable_def::Let_def::exec_rws)); | 
| 5132 | 75 | by Safe_tac; | 
| 4828 | 76 | by (rename_tac "ex1 ex2 n" 1); | 
| 4772 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 77 |   by (res_inst_tac [("Q","reachable A (ex2 n)")] conjunct1 1);
 | 
| 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 78 | by (Asm_full_simp_tac 1); | 
| 5184 | 79 | by (induct_tac "n" 1); | 
| 4772 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 80 | by (fast_tac (claset() addIs [p1,reachable_0]) 1); | 
| 5184 | 81 |   by (eres_inst_tac[("x","na")] allE 1);
 | 
| 8442 
96023903c2df
case_tac now subsumes both boolean and datatype cases;
 wenzelm parents: 
8423diff
changeset | 82 | by (case_tac "ex1 na" 1 THEN ALLGOALS Asm_full_simp_tac); | 
| 4153 | 83 | by Safe_tac; | 
| 4772 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 84 | by (etac (p2 RS mp) 1); | 
| 
8c7e7eaffbdf
split_all_tac now fails if there is nothing to split
 oheimb parents: 
4530diff
changeset | 85 | by (ALLGOALS(fast_tac(claset() addDs [reachable_n]))); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 86 | qed "invariantI"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 87 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 88 | val [p1,p2] = goal IOA.thy | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 89 | "[| !!s. s : starts_of(A) ==> P(s); \ | 
| 9166 | 90 | \ !!s t a. reachable A s ==> P(s) --> (s,a,t):trans_of(A) --> P(t) \ | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 91 | \ |] ==> invariant A P"; | 
| 4089 | 92 | by (fast_tac (claset() addSIs [invariantI] addSDs [p1,p2]) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 93 | qed "invariantI1"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 94 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 95 | val [p1,p2] = goalw IOA.thy [invariant_def] | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 96 | "[| invariant A P; reachable A s |] ==> P(s)"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 97 | by (rtac (p2 RS (p1 RS spec RS mp)) 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 98 | qed "invariantE"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 99 | |
| 5069 | 100 | Goal | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 101 | "actions(asig_comp a b) = actions(a) Un actions(b)"; | 
| 4089 | 102 | by (simp_tac (simpset() addsimps | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 103 | ([actions_def,asig_comp_def]@asig_projections)) 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 104 | by (Fast_tac 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 105 | qed "actions_asig_comp"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 106 | |
| 5069 | 107 | Goal | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 108 | "starts_of(A || B) = {p. fst(p):starts_of(A) & snd(p):starts_of(B)}";
 | 
| 4089 | 109 | by (simp_tac (simpset() addsimps (par_def::ioa_projections)) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 110 | qed "starts_of_par"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 111 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 112 | (* Every state in an execution is reachable *) | 
| 5069 | 113 | Goalw [reachable_def] | 
| 5148 
74919e8f221c
More tidying and removal of "\!\!... from Goal commands
 paulson parents: 
5143diff
changeset | 114 | "ex:executions(A) ==> !n. reachable A (snd ex n)"; | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 115 | by (Fast_tac 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 116 | qed "states_of_exec_reachable"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 117 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 118 | |
| 5069 | 119 | Goal | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 120 | "(s,a,t) : trans_of(A || B || C || D) = \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 121 | \ ((a:actions(asig_of(A)) | a:actions(asig_of(B)) | a:actions(asig_of(C)) | \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 122 | \ a:actions(asig_of(D))) & \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 123 | \ (if a:actions(asig_of(A)) then (fst(s),a,fst(t)):trans_of(A) \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 124 | \ else fst t=fst s) & \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 125 | \ (if a:actions(asig_of(B)) then (fst(snd(s)),a,fst(snd(t))):trans_of(B) \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 126 | \ else fst(snd(t))=fst(snd(s))) & \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 127 | \ (if a:actions(asig_of(C)) then \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 128 | \ (fst(snd(snd(s))),a,fst(snd(snd(t)))):trans_of(C) \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 129 | \ else fst(snd(snd(t)))=fst(snd(snd(s)))) & \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 130 | \ (if a:actions(asig_of(D)) then \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 131 | \ (snd(snd(snd(s))),a,snd(snd(snd(t)))):trans_of(D) \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 132 | \ else snd(snd(snd(t)))=snd(snd(snd(s)))))"; | 
| 9166 | 133 | (*SLOW*) | 
| 134 | by (simp_tac (simpset() addsimps ([par_def,actions_asig_comp,Pair_fst_snd_eq] | |
| 135 | @ ioa_projections)) 1); | |
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 136 | qed "trans_of_par4"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 137 | |
| 5069 | 138 | Goal "starts_of(restrict ioa acts) = starts_of(ioa) & \ | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 139 | \ trans_of(restrict ioa acts) = trans_of(ioa) & \ | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 140 | \ reachable (restrict ioa acts) s = reachable ioa s"; | 
| 4089 | 141 | by (simp_tac (simpset() addsimps ([is_execution_fragment_def,executions_def, | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 142 | reachable_def,restrict_def]@ioa_projections)) 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 143 | qed "cancel_restrict"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 144 | |
| 5069 | 145 | Goal "asig_of(A || B) = asig_comp (asig_of A) (asig_of B)"; | 
| 4089 | 146 | by (simp_tac (simpset() addsimps (par_def::ioa_projections)) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 147 | qed "asig_of_par"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 148 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 149 | |
| 5069 | 150 | Goal "externals(asig_of(A1||A2)) = \ | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 151 | \ (externals(asig_of(A1)) Un externals(asig_of(A2)))"; | 
| 4089 | 152 | by (asm_full_simp_tac (simpset() addsimps [externals_def,asig_of_par,asig_comp_def,asig_inputs_def,asig_outputs_def,Un_def,set_diff_def]) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 153 | by (rtac set_ext 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 154 | by (Fast_tac 1); | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 155 | qed"externals_of_par"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 156 | |
| 5069 | 157 | Goalw [externals_def,actions_def,compat_ioas_def,compat_asigs_def] | 
| 5148 
74919e8f221c
More tidying and removal of "\!\!... from Goal commands
 paulson parents: 
5143diff
changeset | 158 | "[| compat_ioas A1 A2; a:externals(asig_of(A1))|] ==> a~:internals(asig_of(A2))"; | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 159 | by (Asm_full_simp_tac 1); | 
| 4089 | 160 | by (best_tac (claset() addEs [equalityCE]) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 161 | qed"ext1_is_not_int2"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 162 | |
| 5069 | 163 | Goalw [externals_def,actions_def,compat_ioas_def,compat_asigs_def] | 
| 5148 
74919e8f221c
More tidying and removal of "\!\!... from Goal commands
 paulson parents: 
5143diff
changeset | 164 | "[| compat_ioas A2 A1 ; a:externals(asig_of(A1))|] ==> a~:internals(asig_of(A2))"; | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 165 | by (Asm_full_simp_tac 1); | 
| 4089 | 166 | by (best_tac (claset() addEs [equalityCE]) 1); | 
| 3078 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 167 | qed"ext2_is_not_int1"; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 168 | |
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 169 | val ext1_ext2_is_not_act2 = ext1_is_not_int2 RS int_and_ext_is_act; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 170 | val ext1_ext2_is_not_act1 = ext2_is_not_int1 RS int_and_ext_is_act; | 
| 
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
 mueller parents: diff
changeset | 171 |