src/HOL/UNITY/UNITY.ML
author paulson
Fri, 03 Apr 1998 12:34:33 +0200
changeset 4776 1f9362e769c1
child 5069 3ea049f7979d
permissions -rw-r--r--
New UNITY theory
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     1
(*  Title:      HOL/UNITY/UNITY
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     2
    ID:         $Id$
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     4
    Copyright   1998  University of Cambridge
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     5
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     6
The basic UNITY theory (revised version, based upon the "co" operator)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     7
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     8
From Misra, "A Logic for Concurrent Programming", 1994
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     9
*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    10
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    11
set proof_timing;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    12
HOL_quantifiers := false;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    13
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    14
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    15
(*CAN BOOLEAN SIMPLIFICATION BE AUTOMATED?*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    16
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    17
(** Rewrites rules to eliminate A.  Conditions can be satisfied by letting B
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    18
    be any set including A Int C and contained in A Un C, such as B=A or B=C.
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    19
**)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    20
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    21
goal thy "!!x. [| A Int C <= B; B <= A Un C |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    22
\              ==> (A Int B) Un (Compl A Int C) = B Un C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    23
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    24
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    25
goal thy "!!x. [| A Int C <= B; B <= A Un C |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    26
\              ==> (A Un B) Int (Compl A Un C) = B Int C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    27
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    28
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    29
(*The base B=A*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    30
goal thy "A Un (Compl A Int C) = A Un C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    31
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    32
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    33
goal thy "A Int (Compl A Un C) = A Int C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    34
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    35
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    36
(*The base B=C*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    37
goal thy "(A Int C) Un (Compl A Int C) = C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    38
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    39
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    40
goal thy "(A Un C) Int (Compl A Un C) = C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    41
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    42
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    43
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    44
(** More ad-hoc rules **)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    45
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    46
goal thy "A Un B - (A - B) = B";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    47
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    48
qed "Un_Diff_Diff";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    49
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    50
goal thy "A Int (B - C) Un C = A Int B Un C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    51
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    52
qed "Int_Diff_Un";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    53
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    54
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    55
open UNITY;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    56
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    57
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    58
(*** constrains ***)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    59
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    60
val prems = goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    61
    "(!!act s s'. [| act: Acts;  (s,s') : act;  s: A |] ==> s': A') \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    62
\    ==> constrains Acts A A'";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    63
by (blast_tac (claset() addIs prems) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    64
qed "constrainsI";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    65
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    66
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    67
    "!!Acts. [| constrains Acts A A'; act: Acts;  (s,s'): act;  s: A |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    68
\            ==> s': A'";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    69
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    70
qed "constrainsD";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    71
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    72
goalw thy [constrains_def] "constrains Acts {} B";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    73
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    74
qed "constrains_empty";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    75
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    76
goalw thy [constrains_def] "constrains Acts A UNIV";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    77
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    78
qed "constrains_UNIV";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    79
AddIffs [constrains_empty, constrains_UNIV];
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    80
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    81
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    82
    "!!Acts. [| constrains Acts A A'; A'<=B' |] ==> constrains Acts A B'";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    83
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    84
qed "constrains_weaken_R";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    85
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    86
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    87
    "!!Acts. [| constrains Acts A A'; B<=A |] ==> constrains Acts B A'";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    88
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    89
qed "constrains_weaken_L";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    90
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    91
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    92
   "!!Acts. [| constrains Acts A A'; B<=A; A'<=B' |] ==> constrains Acts B B'";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    93
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    94
qed "constrains_weaken";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    95
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    96
(*Set difference: UNUSED*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    97
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    98
  "!!C. [| constrains Acts (A-B) C; constrains Acts B C |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    99
\       ==> constrains Acts A C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   100
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   101
qed "constrains_Diff";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   102
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   103
(** Union **)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   104
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   105
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   106
    "!!Acts. [| constrains Acts A A'; constrains Acts B B' |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   107
\           ==> constrains Acts (A Un B) (A' Un B')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   108
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   109
qed "constrains_Un";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   110
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   111
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   112
    "!!Acts. ALL i:I. constrains Acts (A i) (A' i) \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   113
\    ==> constrains Acts (UN i:I. A i) (UN i:I. A' i)";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   114
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   115
qed "ball_constrains_UN";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   116
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   117
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   118
    "!!Acts. [| ALL i. constrains Acts (A i) (A' i) |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   119
\           ==> constrains Acts (UN i. A i) (UN i. A' i)";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   120
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   121
qed "all_constrains_UN";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   122
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   123
(** Intersection **)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   124
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   125
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   126
    "!!Acts. [| constrains Acts A A'; constrains Acts B B' |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   127
\           ==> constrains Acts (A Int B) (A' Int B')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   128
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   129
qed "constrains_Int";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   130
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   131
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   132
    "!!Acts. ALL i:I. constrains Acts (A i) (A' i) \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   133
\    ==> constrains Acts (INT i:I. A i) (INT i:I. A' i)";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   134
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   135
qed "ball_constrains_INT";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   136
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   137
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   138
    "!!Acts. [| ALL i. constrains Acts (A i) (A' i) |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   139
\           ==> constrains Acts (INT i. A i) (INT i. A' i)";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   140
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   141
qed "all_constrains_INT";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   142
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   143
goalw thy [stable_def, constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   144
    "!!Acts. [| stable Acts C; constrains Acts A (C Un A') |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   145
\           ==> constrains Acts (C Un A) (C Un A')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   146
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   147
qed "stable_constrains_Un";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   148
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   149
goalw thy [stable_def, constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   150
    "!!Acts. [| stable Acts C; constrains Acts (C Int A) A' |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   151
\           ==> constrains Acts (C Int A) (C Int A')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   152
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   153
qed "stable_constrains_Int";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   154
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   155
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   156
(*** stable ***)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   157
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   158
goalw thy [stable_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   159
    "!!Acts. constrains Acts A A ==> stable Acts A";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   160
by (assume_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   161
qed "stableI";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   162
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   163
goalw thy [stable_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   164
    "!!Acts. stable Acts A ==> constrains Acts A A";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   165
by (assume_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   166
qed "stableD";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   167
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   168
goalw thy [stable_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   169
    "!!Acts. [| stable Acts A; stable Acts A' |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   170
\           ==> stable Acts (A Un A')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   171
by (blast_tac (claset() addIs [constrains_Un]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   172
qed "stable_Un";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   173
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   174
goalw thy [stable_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   175
    "!!Acts. [| stable Acts A; stable Acts A' |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   176
\           ==> stable Acts (A Int A')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   177
by (blast_tac (claset() addIs [constrains_Int]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   178
qed "stable_Int";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   179
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   180
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   181
    "!!Acts. [| constrains Acts A A'; id: Acts |] ==> A<=A'";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   182
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   183
qed "constrains_imp_subset";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   184
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   185
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   186
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   187
    "!!Acts. [| id: Acts; constrains Acts A B; constrains Acts B C |]   \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   188
\           ==> constrains Acts A C";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   189
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   190
qed "constrains_trans";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   191
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   192
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   193
(*The Elimination Theorem.  The "free" m has become universally quantified!
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   194
  Should the premise be !!m instead of ALL m ?  Would make it harder to use
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   195
  in forward proof.*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   196
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   197
    "!!Acts. [| ALL m. constrains Acts {s. s x = m} (B m) |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   198
\           ==> constrains Acts {s. P(s x)} (UN m. {s. P(m)} Int B m)";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   199
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   200
qed "elimination";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   201
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   202
(*As above, but for the trivial case of a one-variable state, in which the
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   203
  state is identified with its one variable.*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   204
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   205
    "!!Acts. [| ALL m. constrains Acts {m} (B m) |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   206
\           ==> constrains Acts {s. P s} (UN m. {s. P(m)} Int B m)";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   207
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   208
qed "elimination_sing";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   209
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   210
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   211
goalw thy [constrains_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   212
   "!!Acts. [| constrains Acts A (A' Un B); constrains Acts B B'; id: Acts |] \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   213
\           ==> constrains Acts A (A' Un B')";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   214
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   215
qed "constrains_cancel";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   216
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   217
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   218
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   219
(*** Theoretical Results from Section 6 ***)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   220
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   221
goalw thy [constrains_def, strongest_rhs_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   222
    "constrains Acts A (strongest_rhs Acts A )";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   223
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   224
qed "constrains_strongest_rhs";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   225
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   226
goalw thy [constrains_def, strongest_rhs_def]
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   227
    "!!Acts. constrains Acts A B ==> strongest_rhs Acts A <= B";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   228
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   229
qed "strongest_rhs_is_strongest";