src/ZF/UNITY/Comp.ML
author paulson
Wed, 08 Aug 2001 14:33:10 +0200
changeset 11479 697dcaaf478f
child 12195 ed2893765a08
permissions -rw-r--r--
new ZF/UNITY theory
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     1
(*  Title:      ZF/UNITY/Comp.ML
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     2
    ID:         $Id$
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     3
    Author:     Sidi O Ehmety, Computer Laboratory
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     4
    Copyright   1998  University of Cambridge
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     5
Composition
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     6
From Chandy and Sanders, "Reasoning About Program Composition"
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     7
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     8
Revised by Sidi Ehmety on January 2001
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
     9
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    10
*)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    11
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    12
(*** component and strict_component relations ***)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    13
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    14
Goalw [component_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    15
     "H component F | H component G ==> H component (F Join G)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    16
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    17
by (res_inst_tac [("x", "Ga Join G")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    18
by (res_inst_tac [("x", "G Join F")] exI 2);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    19
by (auto_tac (claset(), simpset() addsimps Join_ac));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    20
qed "componentI";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    21
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    22
Goalw [component_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    23
     "G:program ==> (F component G) <-> \
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    24
\  (Init(G) <= Init(F) & Acts(F) <= Acts(G) & AllowedActs(G) <= AllowedActs(F))";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    25
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    26
by (rtac exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    27
by (rtac program_equalityI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    28
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    29
qed "component_eq_subset";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    30
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    31
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    32
Goalw [component_def] 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    33
   "F:program ==> SKIP component F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    34
by (res_inst_tac [("x", "F")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    35
by (force_tac (claset() addIs [Join_SKIP_left], simpset()) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    36
qed "component_SKIP";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    37
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    38
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    39
Goalw [component_def] 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    40
"F:program ==> F component F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    41
by (res_inst_tac  [("x", "F")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    42
by (force_tac (claset() addIs [Join_SKIP_right], simpset()) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    43
qed "component_refl";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    44
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    45
Addsimps [component_SKIP, component_refl];
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    46
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    47
Goal "F component SKIP ==> programify(F) = SKIP";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    48
by (rtac program_equalityI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    49
by (ALLGOALS(asm_full_simp_tac (simpset() addsimps [component_eq_subset])));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    50
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    51
qed "SKIP_minimal";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    52
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    53
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    54
Goalw [component_def] "F component (F Join G)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    55
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    56
qed "component_Join1";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    57
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    58
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    59
Goalw [component_def] "G component (F Join G)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    60
by (simp_tac (simpset() addsimps [Join_commute]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    61
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    62
qed "component_Join2";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    63
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    64
Goal "F component G ==> F Join G = G";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    65
by (auto_tac (claset(), simpset() 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    66
        addsimps [component_def, Join_left_absorb]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    67
qed "Join_absorb1";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    68
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    69
Goal "G component F ==> F Join G = F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    70
by (auto_tac (claset(), simpset() addsimps Join_ac@[component_def]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    71
qed "Join_absorb2";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    72
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    73
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    74
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    75
Goal "H:program ==> \
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    76
\  (JOIN(I,F) component H) <-> (ALL i:I. F(i) component H)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    77
by (case_tac "I=0" 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    78
by (Force_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    79
by (asm_simp_tac (simpset() addsimps [component_eq_subset]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    80
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    81
by (dres_inst_tac [("c", "xb"), ("A", "AllowedActs(H)")] subsetD 2);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    82
by (REPEAT(blast_tac (claset() addSEs [not_emptyE]) 1));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    83
qed "JN_component_iff";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    84
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    85
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    86
Goalw [component_def] "i : I ==> F(i) component (JN i:I. (F(i)))";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    87
by (blast_tac (claset() addIs [JN_absorb]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    88
qed "component_JN";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    89
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    90
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    91
Goalw [component_def] "[| F component G; G component H |] ==> F component H";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    92
by (blast_tac (claset() addIs [Join_assoc RS sym]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    93
qed "component_trans";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    94
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    95
Goal "[| F:program; G:program |] ==> \
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    96
\ (F  component G & G  component F) --> F = G";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    97
by (asm_simp_tac (simpset() addsimps [component_eq_subset]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    98
by (Clarify_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    99
by (rtac program_equalityI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   100
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   101
qed "component_antisym";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   102
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   103
Goal "H:program ==> ((F Join G) component H) <-> (F component H & G component H)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   104
by (asm_simp_tac (simpset() addsimps [component_eq_subset]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   105
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   106
qed "Join_component_iff";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   107
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   108
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   109
Goal "[| F component G; G:A co B; F:program |] ==> F : A co B";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   110
by (forward_tac [constrainsD2] 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   111
by (rotate_tac ~1 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   112
by (auto_tac (claset(), 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   113
              simpset() addsimps [constrains_def, component_eq_subset]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   114
qed "component_constrains";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   115
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   116
(*Used in Guar.thy to show that programs are partially ordered*)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   117
(* bind_thm ("program_less_le", strict_component_def RS meta_eq_to_obj_eq);*)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   118
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   119
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   120
(*** preserves ***)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   121
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   122
val prems = 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   123
Goalw [preserves_def] 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   124
"ALL z. F:stable({s:state. f(s) = z})  ==> F:preserves(f)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   125
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   126
by (blast_tac (claset() addDs [stableD2]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   127
bind_thm("preservesI", allI RS result());
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   128
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   129
Goalw [preserves_def, stable_def, constrains_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   130
     "[| F:preserves(f);  act : Acts(F);  <s,t> : act |] ==> f(s) = f(t)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   131
by (subgoal_tac "s:state & t:state" 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   132
by (blast_tac (claset() addSDs [ActsD]) 2);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   133
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   134
by (dres_inst_tac [("x", "f(s)")] spec 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   135
by (dres_inst_tac [("x", "act")] bspec 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   136
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   137
qed "preserves_imp_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   138
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   139
Goalw [preserves_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   140
"(F Join G : preserves(v)) <->  \
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   141
\     (programify(F) : preserves(v) & programify(G) : preserves(v))";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   142
by (auto_tac (claset(), simpset() addsimps [INT_iff]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   143
qed "Join_preserves";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   144
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   145
 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   146
Goal "(JOIN(I,F): preserves(v)) <-> (ALL i:I. programify(F(i)):preserves(v))";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   147
by (auto_tac (claset(), simpset() addsimps 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   148
             [JN_stable, preserves_def, INT_iff]@state_simps));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   149
qed "JN_preserves";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   150
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   151
Goal "SKIP : preserves(v)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   152
by (auto_tac (claset(), simpset() 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   153
           addsimps [preserves_def, INT_iff]@state_simps));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   154
qed "SKIP_preserves";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   155
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   156
AddIffs [Join_preserves, JN_preserves, SKIP_preserves];
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   157
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   158
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   159
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   160
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   161
(** component_of **)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   162
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   163
(*  component_of is stronger than component *)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   164
Goalw [component_def, component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   165
"F component_of H ==> F component H";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   166
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   167
qed "component_of_imp_component";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   168
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   169
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   170
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   171
(* component_of satisfies many of the <='s properties *)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   172
Goalw [component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   173
"F:program ==> F component_of F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   174
by (res_inst_tac [("x", "SKIP")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   175
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   176
qed "component_of_refl";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   177
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   178
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   179
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   180
Goalw [component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   181
"F:program ==>SKIP component_of F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   182
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   183
by (res_inst_tac [("x", "F")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   184
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   185
qed "component_of_SKIP";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   186
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   187
Addsimps [component_of_refl, component_of_SKIP];
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   188
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   189
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   190
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   191
Goalw [component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   192
"[| F component_of G; G component_of H |] ==> F component_of H";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   193
by (blast_tac (claset() addIs [Join_assoc RS sym]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   194
qed "component_of_trans";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   195
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   196
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   197
(** localize **)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   198
Goalw [localize_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   199
 "Init(localize(v,F)) = Init(F)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   200
by (Simp_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   201
qed "localize_Init_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   202
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   203
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   204
Goalw [localize_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   205
 "Acts(localize(v,F)) = Acts(F)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   206
by (Simp_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   207
qed "localize_Acts_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   208
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   209
Goalw [localize_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   210
 "AllowedActs(localize(v,F)) = AllowedActs(F Int (UN G:preserves(v). Acts(G)))";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   211
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   212
qed "localize_AllowedActs_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   213
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   214
Addsimps [localize_Init_eq, localize_Acts_eq, localize_AllowedActs_eq];