src/ZF/UNITY/Comp.ML
author paulson
Fri, 24 May 2002 16:55:28 +0200
changeset 13178 bc54319f6875
parent 12484 7ad150f5fc10
child 13339 0f89104dd377
permissions -rw-r--r--
new quantifier lemmas
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
Goalw [component_def] 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    32
   "F:program ==> SKIP component F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    33
by (res_inst_tac [("x", "F")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    34
by (force_tac (claset() addIs [Join_SKIP_left], simpset()) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    35
qed "component_SKIP";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    36
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    37
Goalw [component_def] 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    38
"F:program ==> F component F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    39
by (res_inst_tac  [("x", "F")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    40
by (force_tac (claset() addIs [Join_SKIP_right], simpset()) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    41
qed "component_refl";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    42
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    43
Addsimps [component_SKIP, component_refl];
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    44
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    45
Goal "F component SKIP ==> programify(F) = SKIP";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    46
by (rtac program_equalityI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    47
by (ALLGOALS(asm_full_simp_tac (simpset() addsimps [component_eq_subset])));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    48
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    49
qed "SKIP_minimal";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    50
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    51
Goalw [component_def] "F component (F Join G)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    52
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    53
qed "component_Join1";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    54
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    55
Goalw [component_def] "G component (F Join G)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    56
by (simp_tac (simpset() addsimps [Join_commute]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    57
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    58
qed "component_Join2";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    59
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    60
Goal "F component G ==> F Join G = G";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    61
by (auto_tac (claset(), simpset() 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    62
        addsimps [component_def, Join_left_absorb]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    63
qed "Join_absorb1";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    64
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    65
Goal "G component F ==> F Join G = F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    66
by (auto_tac (claset(), simpset() addsimps Join_ac@[component_def]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    67
qed "Join_absorb2";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    68
12220
9dc4e8fec63d last-minute tidying
paulson
parents: 12195
diff changeset
    69
Goal "H:program==>(JOIN(I,F) component H) <-> (ALL i:I. F(i) component H)";
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    70
by (case_tac "I=0" 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    71
by (Force_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    72
by (asm_simp_tac (simpset() addsimps [component_eq_subset]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    73
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    74
by (dres_inst_tac [("c", "xb"), ("A", "AllowedActs(H)")] subsetD 2);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    75
by (REPEAT(blast_tac (claset() addSEs [not_emptyE]) 1));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    76
qed "JN_component_iff";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    77
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
    78
Goalw [component_def] "i:I ==> F(i) component (JN i:I. (F(i)))";
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    79
by (blast_tac (claset() addIs [JN_absorb]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    80
qed "component_JN";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    81
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    82
Goalw [component_def] "[| F component G; G component H |] ==> F component H";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    83
by (blast_tac (claset() addIs [Join_assoc RS sym]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    84
qed "component_trans";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    85
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
    86
Goal "[| F:program; G:program |] ==>(F component G & G  component F) --> F = G";
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    87
by (asm_simp_tac (simpset() addsimps [component_eq_subset]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    88
by (Clarify_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    89
by (rtac program_equalityI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    90
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    91
qed "component_antisym";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    92
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    93
Goal "H:program ==> ((F Join G) component H) <-> (F component H & G component H)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    94
by (asm_simp_tac (simpset() addsimps [component_eq_subset]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    95
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    96
qed "Join_component_iff";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    97
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
    98
Goal "[| F component G; G:A co B; F:program |] ==> F : A co B";
12484
7ad150f5fc10 isatool expandshort;
wenzelm
parents: 12220
diff changeset
    99
by (ftac constrainsD2 1);
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   100
by (rotate_tac ~1 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   101
by (auto_tac (claset(), 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   102
              simpset() addsimps [constrains_def, component_eq_subset]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   103
qed "component_constrains";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   104
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   105
(* Used in Guar.thy to show that programs are partially ordered*)
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   106
(* bind_thm ("program_less_le", strict_component_def RS meta_eq_to_obj_eq);*)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   107
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   108
(*** preserves ***)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   109
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   110
val prems = Goalw [preserves_def] 
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   111
"ALL z. F:stable({s:state. f(s) = z})  ==> F:preserves(f)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   112
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   113
by (blast_tac (claset() addDs [stableD2]) 1);
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   114
qed "preserves_aux";
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   115
bind_thm("preservesI", allI RS preserves_aux);
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   116
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   117
Goalw [preserves_def, stable_def, constrains_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   118
     "[| F:preserves(f);  act : Acts(F);  <s,t> : act |] ==> f(s) = f(t)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   119
by (subgoal_tac "s:state & t:state" 1);
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   120
by (blast_tac (claset() addSDs [Acts_type RS subsetD]) 2);
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   121
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   122
by (dres_inst_tac [("x", "f(s)")] spec 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   123
by (dres_inst_tac [("x", "act")] bspec 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   124
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   125
qed "preserves_imp_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   126
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   127
Goalw [preserves_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   128
"(F Join G : preserves(v)) <->  \
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   129
\     (programify(F) : preserves(v) & programify(G) : preserves(v))";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   130
by (auto_tac (claset(), simpset() addsimps [INT_iff]));
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   131
qed "Join_preserves";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   132
 
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   133
Goal "(JOIN(I,F): preserves(v)) <-> (ALL i:I. programify(F(i)):preserves(v))";
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   134
by (auto_tac (claset(), simpset() addsimps [JN_stable, preserves_def, INT_iff]));
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   135
qed "JN_preserves";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   136
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   137
Goal "SKIP : preserves(v)";
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   138
by (auto_tac (claset(), simpset() addsimps [preserves_def, INT_iff]));
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   139
qed "SKIP_preserves";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   140
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   141
AddIffs [Join_preserves, JN_preserves, SKIP_preserves];
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   142
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   143
(** Added by Sidi **)
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   144
(** component_of **)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   145
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   146
(*  component_of is stronger than component *)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   147
Goalw [component_def, component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   148
"F component_of H ==> F component H";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   149
by (Blast_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   150
qed "component_of_imp_component";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   151
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   152
(* component_of satisfies many of component's properties *)
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   153
Goalw [component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   154
"F:program ==> F component_of F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   155
by (res_inst_tac [("x", "SKIP")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   156
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   157
qed "component_of_refl";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   158
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   159
Goalw [component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   160
"F:program ==>SKIP component_of F";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   161
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   162
by (res_inst_tac [("x", "F")] exI 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   163
by Auto_tac;
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   164
qed "component_of_SKIP";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   165
Addsimps [component_of_refl, component_of_SKIP];
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   166
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   167
Goalw [component_of_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   168
"[| F component_of G; G component_of H |] ==> F component_of H";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   169
by (blast_tac (claset() addIs [Join_assoc RS sym]) 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   170
qed "component_of_trans";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   171
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   172
(** localize **)
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   173
Goalw [localize_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   174
 "Init(localize(v,F)) = Init(F)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   175
by (Simp_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   176
qed "localize_Init_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   177
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   178
Goalw [localize_def]
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   179
 "Acts(localize(v,F)) = Acts(F)";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   180
by (Simp_tac 1);
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   181
qed "localize_Acts_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   182
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   183
Goalw [localize_def]
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   184
 "AllowedActs(localize(v,F)) = AllowedActs(F) Int (UN G:preserves(v). Acts(G))";
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   185
by (rtac equalityI 1);
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   186
by (auto_tac (claset() addDs [Acts_type RS subsetD], simpset()));
11479
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   187
qed "localize_AllowedActs_eq";
697dcaaf478f new ZF/UNITY theory
paulson
parents:
diff changeset
   188
12195
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   189
AddIffs [localize_Init_eq, localize_Acts_eq, localize_AllowedActs_eq];
ed2893765a08 *** empty log message ***
ehmety
parents: 11479
diff changeset
   190