Datasets:

Modalities:
Text
Languages:
English
Libraries:
Datasets
License:
File size: 3,044 Bytes
4365a98
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
(*  Title:       OAWN_SOS_Labels.thy
    License:     BSD 2-Clause. See LICENSE.
    Author:      Timothy Bourke
*)

section "Configure the inv-cterms tactic for open sequential processes"

theory OAWN_SOS_Labels
imports OAWN_SOS Inv_Cterms
begin

lemma oelimder_guard:
  assumes "p = {l}\<langle>fg\<rangle> qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}\<langle>fg\<rangle> p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemma oelimder_assign:
  assumes "p = {l}\<lbrakk>fa\<rbrakk> qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}\<lbrakk>fa\<rbrakk> p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemma oelimder_ucast:
  assumes "p = {l}unicast(fip, fmsg).q1 \<triangleright> q2"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' pp' where "p = {l}unicast(fip, fmsg).p' \<triangleright> pp'"
                   and "case a of unicast _ _ \<Rightarrow> l' \<in> labels \<Gamma> q1
                                        | _ \<Rightarrow> l' \<in> labels \<Gamma> q2"
  using assms by simp (erule oseqpTEs, auto)

lemma oelimder_bcast:
  assumes "p = {l}broadcast(fmsg).qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}broadcast(fmsg). p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemma oelimder_gcast:
  assumes "p = {l}groupcast(fips, fmsg).qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}groupcast(fips, fmsg). p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemma oelimder_send:
  assumes "p = {l}send(fmsg).qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}send(fmsg). p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemma oelimder_deliver:
  assumes "p = {l}deliver(fdata).qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}deliver(fdata).p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemma oelimder_receive:
  assumes "p = {l}receive(fmsg).qq"
      and "l' \<in> labels \<Gamma> q"
      and "((\<sigma>, p), a, (\<sigma>', q)) \<in> oseqp_sos \<Gamma> i"
  obtains p' where "p = {l}receive(fmsg).p'"
               and "l' \<in> labels \<Gamma> qq"
  using assms by auto

lemmas oelimders =
   oelimder_guard
   oelimder_assign
   oelimder_ucast
   oelimder_bcast
   oelimder_gcast
   oelimder_send
   oelimder_deliver
   oelimder_receive

declare
  oseqpTEs [cterms_seqte]
  oelimders [cterms_elimders]

end