src/HOL/UNITY/Comp.ML
author paulson
Thu, 26 Aug 1999 11:36:04 +0200
changeset 7361 477e1bdf230f
parent 7340 a22efb7a522b
child 7386 1048bc161c05
permissions -rw-r--r--
changed "guar" back to "guarantees" (sorry)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     1
(*  Title:      HOL/UNITY/Comp.thy
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     2
    ID:         $Id$
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     4
    Copyright   1998  University of Cambridge
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     5
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     6
Composition
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     7
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     8
From Chandy and Sanders, "Reasoning About Program Composition"
a12b25c53df1 composition theory
paulson
parents:
diff changeset
     9
*)
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    10
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    11
(*** component ***)
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    12
6738
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    13
Goalw [component_def]
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    14
     "H component F | H component G ==> H component (F Join G)";
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    15
by Auto_tac;
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    16
by (res_inst_tac [("x", "G Join Ga")] exI 1);
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    17
by (res_inst_tac [("x", "G Join F")] exI 2);
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    18
by (auto_tac (claset(), simpset() addsimps Join_ac));
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    19
qed "componentI";
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    20
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
    21
Goalw [component_def]
6738
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    22
     "(F component G) = (Init G <= Init F & Acts F <= Acts G)";
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    23
by (force_tac (claset() addSIs [exI, program_equalityI], 
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    24
	       simpset() addsimps [Acts_Join]) 1);
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    25
qed "component_eq_subset";
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    26
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    27
Goalw [component_def] "SKIP component F";
6012
1894bfc4aee9 Addition of the States component; parts of Comp not working
paulson
parents: 5968
diff changeset
    28
by (force_tac (claset() addIs [Join_SKIP_left], simpset()) 1);
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
    29
qed "component_SKIP";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
    30
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    31
Goalw [component_def] "F component F";
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    32
by (blast_tac (claset() addIs [Join_SKIP_right]) 1);
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    33
qed "component_refl";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    34
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
    35
AddIffs [component_SKIP, component_refl];
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    36
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    37
Goal "F component SKIP ==> F = SKIP";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    38
by (auto_tac (claset() addSIs [program_equalityI],
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    39
	      simpset() addsimps [component_eq_subset]));
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    40
qed "SKIP_minimal";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    41
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    42
Goalw [component_def] "F component (F Join G)";
5968
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    43
by (Blast_tac 1);
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    44
qed "component_Join1";
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    45
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    46
Goalw [component_def] "G component (F Join G)";
5968
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    47
by (simp_tac (simpset() addsimps [Join_commute]) 1);
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    48
by (Blast_tac 1);
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    49
qed "component_Join2";
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    50
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    51
Goalw [component_def] "i : I ==> (F i) component (JN i:I. (F i))";
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    52
by (blast_tac (claset() addIs [JN_absorb]) 1);
5968
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    53
qed "component_JN";
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
    54
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    55
Goalw [component_def] "[| F component G; G component H |] ==> F component H";
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    56
by (blast_tac (claset() addIs [Join_assoc RS sym]) 1);
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    57
qed "component_trans";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    58
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    59
Goal "[| F component G; G component F |] ==> F=G";
6738
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    60
by (full_simp_tac (simpset() addsimps [component_eq_subset]) 1);
06189132c67b component_eq_subset: a neat characterization of "component"
paulson
parents: 6703
diff changeset
    61
by (blast_tac (claset() addSIs [program_equalityI]) 1);
6703
paulson
parents: 6646
diff changeset
    62
qed "component_antisym";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    63
5804
8e0a4c4fd67b Revising the Client proof as suggested by Michel Charpentier. New lemmas
paulson
parents: 5706
diff changeset
    64
Goalw [component_def]
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    65
      "F component H = (EX G. F Join G = H & Disjoint F G)";
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    66
by (blast_tac (claset() addSIs [Diff_Disjoint, Join_Diff2]) 1);
5804
8e0a4c4fd67b Revising the Client proof as suggested by Michel Charpentier. New lemmas
paulson
parents: 5706
diff changeset
    67
qed "component_eq";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    68
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    69
Goal "((F Join G) component H) = (F component H & G component H)";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    70
by (simp_tac (simpset() addsimps [component_eq_subset, Acts_Join]) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    71
by (Blast_tac 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    72
qed "Join_component_iff";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
    73
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    74
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    75
(*** existential properties ***)
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    76
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    77
Goalw [ex_prop_def]
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    78
     "[| ex_prop X; finite GG |] ==> GG Int X ~= {} --> (JN G:GG. G) : X";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    79
by (etac finite_induct 1);
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    80
by (auto_tac (claset(), simpset() addsimps [Int_insert_left]));
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    81
qed_spec_mp "ex1";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    82
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    83
Goalw [ex_prop_def]
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    84
     "ALL GG. finite GG & GG Int X ~= {} --> (JN G:GG. G) : X ==> ex_prop X";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    85
by (Clarify_tac 1);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    86
by (dres_inst_tac [("x", "{F,G}")] spec 1);
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
    87
by Auto_tac;
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    88
qed "ex2";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    89
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    90
(*Chandy & Sanders take this as a definition*)
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
    91
Goal "ex_prop X = (ALL GG. finite GG & GG Int X ~= {} --> (JN G:GG. G) : X)";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    92
by (blast_tac (claset() addIs [ex1,ex2]) 1);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    93
qed "ex_prop_finite";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    94
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    95
(*Their "equivalent definition" given at the end of section 3*)
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
    96
Goal "ex_prop X = (ALL G. G:X = (ALL H. G component H --> H: X))";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
    97
by Auto_tac;
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
    98
by (rewrite_goals_tac [ex_prop_def, component_def]);
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
    99
by (Blast_tac 1);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   100
by Safe_tac;
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   101
by (stac Join_commute 2);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   102
by (ALLGOALS Blast_tac);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   103
qed "ex_prop_equiv";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   104
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   105
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   106
(*** universal properties ***)
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   107
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   108
Goalw [uv_prop_def]
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   109
     "[| uv_prop X; finite GG |] ==> GG <= X --> (JN G:GG. G) : X";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   110
by (etac finite_induct 1);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   111
by (auto_tac (claset(), simpset() addsimps [Int_insert_left]));
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   112
qed_spec_mp "uv1";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   113
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   114
Goalw [uv_prop_def]
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   115
     "ALL GG. finite GG & GG <= X --> (JN G:GG. G) : X  ==> uv_prop X";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   116
by (rtac conjI 1);
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   117
by (Clarify_tac 2);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   118
by (dres_inst_tac [("x", "{F,G}")] spec 2);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   119
by (dres_inst_tac [("x", "{}")] spec 1);
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   120
by Auto_tac;
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   121
qed "uv2";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   122
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   123
(*Chandy & Sanders take this as a definition*)
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   124
Goal "uv_prop X = (ALL GG. finite GG & GG <= X --> (JN G:GG. G) : X)";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   125
by (blast_tac (claset() addIs [uv1,uv2]) 1);
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   126
qed "uv_prop_finite";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   127
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   128
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   129
(*** guarantees ***)
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   130
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   131
val prems = Goal
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   132
     "(!!G. [| F Join G : X;  Disjoint F G |] ==> F Join G : Y) \
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   133
\     ==> F : X guarantees Y";
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   134
by (simp_tac (simpset() addsimps [guar_def, component_eq]) 1);
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   135
by (blast_tac (claset() addIs prems) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   136
qed "guaranteesI";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   137
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   138
Goalw [guar_def, component_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   139
     "[| F : X guarantees Y;  F Join G : X |] ==> F Join G : Y";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   140
by (Blast_tac 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   141
qed "guaranteesD";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   142
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   143
(*This version of guaranteesD matches more easily in the conclusion*)
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   144
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   145
     "[| F : X guarantees Y;  H : X;  F component H |] ==> H : Y";
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   146
by (Blast_tac 1);
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   147
qed "component_guaranteesD";
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   148
5668
9ddc4e836d3e moved a theorem
paulson
parents: 5637
diff changeset
   149
(*This equation is more intuitive than the official definition*)
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   150
Goal "(F : X guarantees Y) = \
5968
06f9dbfff032 renamed vars
paulson
parents: 5804
diff changeset
   151
\     (ALL G. F Join G : X & Disjoint F G --> F Join G : Y)";
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   152
by (simp_tac (simpset() addsimps [guar_def, component_eq]) 1);
5668
9ddc4e836d3e moved a theorem
paulson
parents: 5637
diff changeset
   153
by (Blast_tac 1);
9ddc4e836d3e moved a theorem
paulson
parents: 5637
diff changeset
   154
qed "guarantees_eq";
9ddc4e836d3e moved a theorem
paulson
parents: 5637
diff changeset
   155
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   156
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   157
     "[| F: X guarantees X'; Y <= X; X' <= Y' |] ==> F: Y guarantees Y'";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   158
by (Blast_tac 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   159
qed "guarantees_weaken";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   160
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   161
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   162
     "[| F: X guarantees Y; F component F' |] ==> F': X guarantees Y";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   163
by (blast_tac (claset() addIs [component_trans]) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   164
qed "guarantees_weaken_prog";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   165
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   166
Goalw [guar_def] "X <= Y ==> X guarantees Y = UNIV";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   167
by (Blast_tac 1);
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   168
qed "subset_imp_guarantees_UNIV";
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   169
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   170
(*Equivalent to subset_imp_guarantees_UNIV but more intuitive*)
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   171
Goalw [guar_def] "X <= Y ==> F : X guarantees Y";
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   172
by (Blast_tac 1);
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   173
qed "subset_imp_guarantees";
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   174
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   175
(*Remark at end of section 4.1*)
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   176
Goalw [guar_def] "ex_prop Y = (Y = UNIV guarantees Y)";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   177
by (simp_tac (simpset() addsimps [ex_prop_equiv]) 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   178
by (blast_tac (claset() addEs [equalityE]) 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   179
qed "ex_prop_equiv2";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   180
6822
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   181
(** Distributive laws.  Re-orient to perform miniscoping **)
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   182
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   183
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   184
     "(UN i:I. X i) guarantees Y = (INT i:I. X i guarantees Y)";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   185
by (Blast_tac 1);
6822
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   186
qed "guarantees_UN_left";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   187
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   188
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   189
    "(X Un Y) guarantees Z = (X guarantees Z) Int (Y guarantees Z)";
6822
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   190
by (Blast_tac 1);
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   191
qed "guarantees_Un_left";
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   192
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   193
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   194
     "X guarantees (INT i:I. Y i) = (INT i:I. X guarantees Y i)";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   195
by (Blast_tac 1);
6822
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   196
qed "guarantees_INT_right";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   197
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   198
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   199
    "Z guarantees (X Int Y) = (Z guarantees X) Int (Z guarantees Y)";
6822
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   200
by (Blast_tac 1);
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   201
qed "guarantees_Int_right";
8932f33259d4 guarantees -> guar
paulson
parents: 6738
diff changeset
   202
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   203
Goalw [guar_def] "(X guarantees Y) = (UNIV guarantees (-X Un Y))";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   204
by (Blast_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   205
qed "shunting";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   206
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   207
Goalw [guar_def] "(X guarantees Y) = -Y guarantees -X";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   208
by (Blast_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   209
qed "contrapositive";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   210
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   211
(** The following two can be expressed using intersection and subset, which
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   212
    is more faithful to the text but looks cryptic.
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   213
**)
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   214
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   215
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   216
    "[| F : V guarantees X;  F : (X Int Y) guarantees Z |]\
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   217
\    ==> F : (V Int Y) guarantees Z";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   218
by (Blast_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   219
qed "combining1";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   220
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   221
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   222
    "[| F : V guarantees (X Un Y);  F : Y guarantees Z |]\
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   223
\    ==> F : V guarantees (X Un Z)";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   224
by (Blast_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   225
qed "combining2";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   226
6646
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   227
(** The following two follow Chandy-Sanders, but the use of object-quantifiers
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   228
    does not suit Isabelle... **)
3ea726909fff "component" now an infix
paulson
parents: 6299
diff changeset
   229
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   230
(*Premise should be (!!i. i: I ==> F: X guarantees Y i) *)
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   231
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   232
     "ALL i:I. F : X guarantees (Y i) ==> F : X guarantees (INT i:I. Y i)";
5630
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   233
by (Blast_tac 1);
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   234
qed "all_guarantees";
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   235
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   236
(*Premises should be [| F: X guarantees Y i; i: I |] *)
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   237
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   238
     "EX i:I. F : X guarantees (Y i) ==> F : X guarantees (UN i:I. Y i)";
5630
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   239
by (Blast_tac 1);
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   240
qed "ex_guarantees";
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   241
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   242
(*** Additional guarantees laws, by lcp ***)
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   243
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   244
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   245
    "[| F: U guarantees V;  G: X guarantees Y |] \
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   246
\    ==> F Join G: (U Int X) guarantees (V Int Y)";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   247
by (simp_tac (simpset() addsimps [Join_component_iff]) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   248
by (Blast_tac 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   249
qed "guarantees_Join_Int";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   250
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   251
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   252
    "[| F: U guarantees V;  G: X guarantees Y |]  \
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   253
\    ==> F Join G: (U Un X) guarantees (V Un Y)";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   254
by (simp_tac (simpset() addsimps [Join_component_iff]) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   255
by (Blast_tac 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   256
qed "guarantees_Join_Un";
5630
fc2c299187c0 new guarantees laws
paulson
parents: 5620
diff changeset
   257
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   258
Goal "((JOIN I F) component H) = (ALL i: I. F i component H)";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   259
by (simp_tac (simpset() addsimps [component_eq_subset, Acts_JN]) 1);
5804
8e0a4c4fd67b Revising the Client proof as suggested by Michel Charpentier. New lemmas
paulson
parents: 5706
diff changeset
   260
by (Blast_tac 1);
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   261
qed "JN_component_iff";
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   262
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   263
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   264
    "[| ALL i:I. F i : X i guarantees Y i |] \
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   265
\    ==> (JOIN I F) : (INTER I X) guarantees (INTER I Y)";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   266
by (simp_tac (simpset() addsimps [JN_component_iff]) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   267
by (Blast_tac 1);
7340
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   268
bind_thm ("guarantees_JN_INT", ballI RS result());
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   269
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   270
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   271
    "[| ALL i:I. F i : X i guarantees Y i |] \
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   272
\    ==> (JOIN I F) : (UNION I X) guarantees (UNION I Y)";
6833
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   273
by (simp_tac (simpset() addsimps [JN_component_iff]) 1);
15d6c121d75f many new guarantees laws
paulson
parents: 6822
diff changeset
   274
by (Blast_tac 1);
7340
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   275
bind_thm ("guarantees_JN_UN", ballI RS result());
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   276
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   277
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   278
(*** guarantees laws for breaking down the program, by lcp ***)
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   279
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   280
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   281
    "F: X guarantees Y | G: X guarantees Y ==> F Join G: X guarantees Y";
7340
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   282
by (simp_tac (simpset() addsimps [Join_component_iff]) 1);
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   283
by (Blast_tac 1);
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   284
qed "guarantees_Join_I";
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   285
7361
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   286
Goalw [guar_def]
477e1bdf230f changed "guar" back to "guarantees" (sorry)
paulson
parents: 7340
diff changeset
   287
     "[| i : I;  F i: X guarantees Y |] ==> (JN i:I. (F i)) : X guarantees Y";
7340
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   288
by (simp_tac (simpset() addsimps [JN_component_iff]) 1);
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   289
by (Blast_tac 1);
a22efb7a522b new guarantees laws; also better natural deduction style for old ones
paulson
parents: 6833
diff changeset
   290
qed "guarantees_JN_I";
5637
a06006a320a1 new rule
paulson
parents: 5630
diff changeset
   291
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   292
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   293
(*** well-definedness ***)
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   294
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   295
Goalw [welldef_def] "F Join G: welldef ==> F: welldef";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   296
by Auto_tac;
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   297
qed "Join_welldef_D1";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   298
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   299
Goalw [welldef_def] "F Join G: welldef ==> G: welldef";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   300
by Auto_tac;
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   301
qed "Join_welldef_D2";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   302
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   303
(*** refinement ***)
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   304
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   305
Goalw [refines_def] "F refines F wrt X";
5597
a12b25c53df1 composition theory
paulson
parents:
diff changeset
   306
by (Blast_tac 1);
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   307
qed "refines_refl";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   308
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   309
Goalw [refines_def]
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   310
     "[| H refines G wrt X;  G refines F wrt X |] ==> H refines F wrt X";
6012
1894bfc4aee9 Addition of the States component; parts of Comp not working
paulson
parents: 5968
diff changeset
   311
by Auto_tac;
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   312
qed "refines_trans";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   313
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   314
Goalw [strict_ex_prop_def]
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   315
     "strict_ex_prop X \
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   316
\     ==> (ALL H. F Join H : X --> G Join H : X) = (F:X --> G:X)";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   317
by (Blast_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   318
qed "strict_ex_refine_lemma";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   319
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   320
Goalw [strict_ex_prop_def]
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   321
     "strict_ex_prop X \
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   322
\     ==> (ALL H. F Join H : welldef & F Join H : X --> G Join H : X) = \
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   323
\         (F: welldef Int X --> G:X)";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   324
by Safe_tac;
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   325
by (eres_inst_tac [("x","SKIP"), ("P", "%H. ?PP H --> ?RR H")] allE 1);
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   326
by (auto_tac (claset() addDs [Join_welldef_D1, Join_welldef_D2], simpset()));
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   327
qed "strict_ex_refine_lemma_v";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   328
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   329
Goal "[| strict_ex_prop X;  \
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   330
\        ALL H. F Join H : welldef Int X --> G Join H : welldef |] \
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   331
\     ==> (G refines F wrt X) = (G iso_refines F wrt X)";
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   332
by (res_inst_tac [("x","SKIP")] allE 1
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   333
    THEN assume_tac 1);
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   334
by (asm_full_simp_tac
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   335
    (simpset() addsimps [refines_def, iso_refines_def,
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   336
			 strict_ex_refine_lemma_v]) 1);
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   337
qed "ex_refinement_thm";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   338
6012
1894bfc4aee9 Addition of the States component; parts of Comp not working
paulson
parents: 5968
diff changeset
   339
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   340
Goalw [strict_uv_prop_def]
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   341
     "strict_uv_prop X \
6295
351b3c2b0d83 removed the infernal States, eqStates, compatible, etc.
paulson
parents: 6018
diff changeset
   342
\     ==> (ALL H. F Join H : X --> G Join H : X) = (F:X --> G:X)";
5612
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   343
by (Blast_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   344
qed "strict_uv_refine_lemma";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   345
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   346
Goalw [strict_uv_prop_def]
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   347
     "strict_uv_prop X \
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   348
\     ==> (ALL H. F Join H : welldef & F Join H : X --> G Join H : X) = \
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   349
\         (F: welldef Int X --> G:X)";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   350
by Safe_tac;
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   351
by (eres_inst_tac [("x","SKIP"), ("P", "%H. ?PP H --> ?RR H")] allE 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   352
by (auto_tac (claset() addDs [Join_welldef_D1, Join_welldef_D2],
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   353
	      simpset()));
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   354
qed "strict_uv_refine_lemma_v";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   355
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   356
Goal "[| strict_uv_prop X;  \
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   357
\        ALL H. F Join H : welldef Int X --> G Join H : welldef |] \
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   358
\     ==> (G refines F wrt X) = (G iso_refines F wrt X)";
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   359
by (res_inst_tac [("x","SKIP")] allE 1
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   360
    THEN assume_tac 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   361
by (asm_full_simp_tac (simpset() addsimps [refines_def, iso_refines_def,
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   362
					   strict_uv_refine_lemma_v]) 1);
e981ca6f7332 Finished proofs to end of section 5.1 of Chandy and Sanders
paulson
parents: 5597
diff changeset
   363
qed "uv_refinement_thm";