src/HOL/UNITY/UNITY.ML
changeset 5069 3ea049f7979d
parent 4776 1f9362e769c1
child 5111 8f4b72f0c15d
--- a/src/HOL/UNITY/UNITY.ML	Mon Jun 22 17:13:09 1998 +0200
+++ b/src/HOL/UNITY/UNITY.ML	Mon Jun 22 17:26:46 1998 +0200
@@ -18,36 +18,36 @@
     be any set including A Int C and contained in A Un C, such as B=A or B=C.
 **)
 
-goal thy "!!x. [| A Int C <= B; B <= A Un C |] \
+Goal "!!x. [| A Int C <= B; B <= A Un C |] \
 \              ==> (A Int B) Un (Compl A Int C) = B Un C";
 by (Blast_tac 1);
 
-goal thy "!!x. [| A Int C <= B; B <= A Un C |] \
+Goal "!!x. [| A Int C <= B; B <= A Un C |] \
 \              ==> (A Un B) Int (Compl A Un C) = B Int C";
 by (Blast_tac 1);
 
 (*The base B=A*)
-goal thy "A Un (Compl A Int C) = A Un C";
+Goal "A Un (Compl A Int C) = A Un C";
 by (Blast_tac 1);
 
-goal thy "A Int (Compl A Un C) = A Int C";
+Goal "A Int (Compl A Un C) = A Int C";
 by (Blast_tac 1);
 
 (*The base B=C*)
-goal thy "(A Int C) Un (Compl A Int C) = C";
+Goal "(A Int C) Un (Compl A Int C) = C";
 by (Blast_tac 1);
 
-goal thy "(A Un C) Int (Compl A Un C) = C";
+Goal "(A Un C) Int (Compl A Un C) = C";
 by (Blast_tac 1);
 
 
 (** More ad-hoc rules **)
 
-goal thy "A Un B - (A - B) = B";
+Goal "A Un B - (A - B) = B";
 by (Blast_tac 1);
 qed "Un_Diff_Diff";
 
-goal thy "A Int (B - C) Un C = A Int B Un C";
+Goal "A Int (B - C) Un C = A Int B Un C";
 by (Blast_tac 1);
 qed "Int_Diff_Un";
 
@@ -63,38 +63,38 @@
 by (blast_tac (claset() addIs prems) 1);
 qed "constrainsI";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| constrains Acts A A'; act: Acts;  (s,s'): act;  s: A |] \
 \            ==> s': A'";
 by (Blast_tac 1);
 qed "constrainsD";
 
-goalw thy [constrains_def] "constrains Acts {} B";
+Goalw [constrains_def] "constrains Acts {} B";
 by (Blast_tac 1);
 qed "constrains_empty";
 
-goalw thy [constrains_def] "constrains Acts A UNIV";
+Goalw [constrains_def] "constrains Acts A UNIV";
 by (Blast_tac 1);
 qed "constrains_UNIV";
 AddIffs [constrains_empty, constrains_UNIV];
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| constrains Acts A A'; A'<=B' |] ==> constrains Acts A B'";
 by (Blast_tac 1);
 qed "constrains_weaken_R";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| constrains Acts A A'; B<=A |] ==> constrains Acts B A'";
 by (Blast_tac 1);
 qed "constrains_weaken_L";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
    "!!Acts. [| constrains Acts A A'; B<=A; A'<=B' |] ==> constrains Acts B B'";
 by (Blast_tac 1);
 qed "constrains_weaken";
 
 (*Set difference: UNUSED*)
-goalw thy [constrains_def]
+Goalw [constrains_def]
   "!!C. [| constrains Acts (A-B) C; constrains Acts B C |] \
 \       ==> constrains Acts A C";
 by (Blast_tac 1);
@@ -102,19 +102,19 @@
 
 (** Union **)
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| constrains Acts A A'; constrains Acts B B' |]   \
 \           ==> constrains Acts (A Un B) (A' Un B')";
 by (Blast_tac 1);
 qed "constrains_Un";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. ALL i:I. constrains Acts (A i) (A' i) \
 \    ==> constrains Acts (UN i:I. A i) (UN i:I. A' i)";
 by (Blast_tac 1);
 qed "ball_constrains_UN";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| ALL i. constrains Acts (A i) (A' i) |] \
 \           ==> constrains Acts (UN i. A i) (UN i. A' i)";
 by (Blast_tac 1);
@@ -122,31 +122,31 @@
 
 (** Intersection **)
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| constrains Acts A A'; constrains Acts B B' |]   \
 \           ==> constrains Acts (A Int B) (A' Int B')";
 by (Blast_tac 1);
 qed "constrains_Int";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. ALL i:I. constrains Acts (A i) (A' i) \
 \    ==> constrains Acts (INT i:I. A i) (INT i:I. A' i)";
 by (Blast_tac 1);
 qed "ball_constrains_INT";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| ALL i. constrains Acts (A i) (A' i) |] \
 \           ==> constrains Acts (INT i. A i) (INT i. A' i)";
 by (Blast_tac 1);
 qed "all_constrains_INT";
 
-goalw thy [stable_def, constrains_def]
+Goalw [stable_def, constrains_def]
     "!!Acts. [| stable Acts C; constrains Acts A (C Un A') |]   \
 \           ==> constrains Acts (C Un A) (C Un A')";
 by (Blast_tac 1);
 qed "stable_constrains_Un";
 
-goalw thy [stable_def, constrains_def]
+Goalw [stable_def, constrains_def]
     "!!Acts. [| stable Acts C; constrains Acts (C Int A) A' |]   \
 \           ==> constrains Acts (C Int A) (C Int A')";
 by (Blast_tac 1);
@@ -155,35 +155,35 @@
 
 (*** stable ***)
 
-goalw thy [stable_def]
+Goalw [stable_def]
     "!!Acts. constrains Acts A A ==> stable Acts A";
 by (assume_tac 1);
 qed "stableI";
 
-goalw thy [stable_def]
+Goalw [stable_def]
     "!!Acts. stable Acts A ==> constrains Acts A A";
 by (assume_tac 1);
 qed "stableD";
 
-goalw thy [stable_def]
+Goalw [stable_def]
     "!!Acts. [| stable Acts A; stable Acts A' |]   \
 \           ==> stable Acts (A Un A')";
 by (blast_tac (claset() addIs [constrains_Un]) 1);
 qed "stable_Un";
 
-goalw thy [stable_def]
+Goalw [stable_def]
     "!!Acts. [| stable Acts A; stable Acts A' |]   \
 \           ==> stable Acts (A Int A')";
 by (blast_tac (claset() addIs [constrains_Int]) 1);
 qed "stable_Int";
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| constrains Acts A A'; id: Acts |] ==> A<=A'";
 by (Blast_tac 1);
 qed "constrains_imp_subset";
 
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| id: Acts; constrains Acts A B; constrains Acts B C |]   \
 \           ==> constrains Acts A C";
 by (Blast_tac 1);
@@ -193,7 +193,7 @@
 (*The Elimination Theorem.  The "free" m has become universally quantified!
   Should the premise be !!m instead of ALL m ?  Would make it harder to use
   in forward proof.*)
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| ALL m. constrains Acts {s. s x = m} (B m) |] \
 \           ==> constrains Acts {s. P(s x)} (UN m. {s. P(m)} Int B m)";
 by (Blast_tac 1);
@@ -201,14 +201,14 @@
 
 (*As above, but for the trivial case of a one-variable state, in which the
   state is identified with its one variable.*)
-goalw thy [constrains_def]
+Goalw [constrains_def]
     "!!Acts. [| ALL m. constrains Acts {m} (B m) |] \
 \           ==> constrains Acts {s. P s} (UN m. {s. P(m)} Int B m)";
 by (Blast_tac 1);
 qed "elimination_sing";
 
 
-goalw thy [constrains_def]
+Goalw [constrains_def]
    "!!Acts. [| constrains Acts A (A' Un B); constrains Acts B B'; id: Acts |] \
 \           ==> constrains Acts A (A' Un B')";
 by (Blast_tac 1);
@@ -218,12 +218,12 @@
 
 (*** Theoretical Results from Section 6 ***)
 
-goalw thy [constrains_def, strongest_rhs_def]
+Goalw [constrains_def, strongest_rhs_def]
     "constrains Acts A (strongest_rhs Acts A )";
 by (Blast_tac 1);
 qed "constrains_strongest_rhs";
 
-goalw thy [constrains_def, strongest_rhs_def]
+Goalw [constrains_def, strongest_rhs_def]
     "!!Acts. constrains Acts A B ==> strongest_rhs Acts A <= B";
 by (Blast_tac 1);
 qed "strongest_rhs_is_strongest";