diff -r 95f1e700b712 -r 57bf0cecb366 src/ZF/UNITY/ClientImpl.thy --- a/src/ZF/UNITY/ClientImpl.thy Tue Mar 06 16:46:27 2012 +0000 +++ b/src/ZF/UNITY/ClientImpl.thy Tue Mar 06 17:01:37 2012 +0000 @@ -91,7 +91,7 @@ declare client_ask_act_def [THEN def_act_simp, simp] lemma client_prog_ok_iff: - "\G \ program. (client_prog ok G) <-> + "\G \ program. (client_prog ok G) \ (G \ preserves(lift(rel)) & G \ preserves(lift(ask)) & G \ preserves(lift(tok)) & client_prog \ Allowed(G))" by (auto simp add: ok_iff_Allowed client_prog_def [THEN def_prg_Allowed]) @@ -117,7 +117,7 @@ (*Safety property 1: ask, rel are increasing: (24) *) lemma client_prog_Increasing_ask_rel: -"client_prog: program guarantees Incr(lift(ask)) Int Incr(lift(rel))" +"client_prog: program guarantees Incr(lift(ask)) \ Incr(lift(rel))" apply (unfold guar_def) apply (auto intro!: increasing_imp_Increasing simp add: client_prog_ok_iff Increasing.increasing_def preserves_imp_prefix) @@ -137,7 +137,7 @@ lemma ask_Bounded_lemma: "[| client_prog ok G; G \ program |] ==> client_prog \ G \ - Always({s \ state. s`tok \ NbT} Int + Always({s \ state. s`tok \ NbT} \ {s \ state. \elt \ set_of_list(s`ask). elt \ NbT})" apply (rotate_tac -1) apply (auto simp add: client_prog_ok_iff) @@ -209,7 +209,7 @@ done lemma strict_prefix_is_prefix: - " \ strict_prefix(A) <-> \ prefix(A) & xs\ys" + " \ strict_prefix(A) \ \ prefix(A) & xs\ys" apply (unfold strict_prefix_def id_def lam_def) apply (auto dest: prefix_type [THEN subsetD]) done @@ -298,7 +298,7 @@ lemma client_prog_Allowed: "Allowed(client_prog) = - preserves(lift(rel)) Int preserves(lift(ask)) Int preserves(lift(tok))" + preserves(lift(rel)) \ preserves(lift(ask)) \ preserves(lift(tok))" apply (cut_tac v = "lift (ask)" in preserves_type) apply (auto simp add: Allowed_def client_prog_def [THEN def_prg_Allowed] cons_Int_distrib safety_prop_Acts_iff)