sound_defs_prop.thy
author chunhan
Thu, 13 Jun 2013 22:51:03 +0800
changeset 8 2dab4bbb6684
parent 6 4294abb1f38c
permissions -rw-r--r--
fixed typos
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1
dcde836219bc add thy files
chunhan
parents:
diff changeset
     1
theory sound_defs_prop
dcde836219bc add thy files
chunhan
parents:
diff changeset
     2
imports rc_theory Main os_rc obj2sobj_prop
dcde836219bc add thy files
chunhan
parents:
diff changeset
     3
begin
dcde836219bc add thy files
chunhan
parents:
diff changeset
     4
dcde836219bc add thy files
chunhan
parents:
diff changeset
     5
context tainting_s_sound begin
dcde836219bc add thy files
chunhan
parents:
diff changeset
     6
dcde836219bc add thy files
chunhan
parents:
diff changeset
     7
lemma not_both_I:
dcde836219bc add thy files
chunhan
parents:
diff changeset
     8
  "not_both_sproc (SProc sp srp) sobj \<Longrightarrow> not_both_sproc sobj' sobj"
dcde836219bc add thy files
chunhan
parents:
diff changeset
     9
by (case_tac sobj, auto)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    10
dcde836219bc add thy files
chunhan
parents:
diff changeset
    11
lemma not_both_I_file:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    12
  "not_both_sproc (SFile sf srf) sobj \<Longrightarrow> not_both_sproc (SFile sf' srf') sobj"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    13
by (case_tac sobj, auto)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    14
dcde836219bc add thy files
chunhan
parents:
diff changeset
    15
lemma not_both_I_ipc:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    16
  "not_both_sproc (SIPC si sri) sobj \<Longrightarrow> not_both_sproc (SIPC si' sri') sobj"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    17
by (case_tac sobj, auto)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    18
dcde836219bc add thy files
chunhan
parents:
diff changeset
    19
lemma intact_imp_butp:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    20
  "\<lbrakk>p \<in> init_processes; initp_intact s\<rbrakk> \<Longrightarrow> initp_intact_butp s p "
dcde836219bc add thy files
chunhan
parents:
diff changeset
    21
by (auto simp:initp_intact_def initp_intact_butp_def initp_alter_def)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    22
dcde836219bc add thy files
chunhan
parents:
diff changeset
    23
lemma no_sproc_imp_intact:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    24
  "\<lbrakk>not_both_sproc (SProc sp srp) sobj; initp_intact_but s sobj\<rbrakk> \<Longrightarrow> initp_intact s"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    25
by (case_tac sobj, simp_all)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    26
dcde836219bc add thy files
chunhan
parents:
diff changeset
    27
lemma initp_intact_but_nil:"initp_intact_but [] (init_obj2sobj obj)"  
dcde836219bc add thy files
chunhan
parents:
diff changeset
    28
apply (case_tac obj)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    29
apply (auto simp:initp_intact_def initp_intact_butp_def initp_alter_def split:option.splits)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    30
apply (rule_tac x = nat in exI) using init_proc_has_role 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    31
by (auto simp:bidirect_in_init_def)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    32
dcde836219bc add thy files
chunhan
parents:
diff changeset
    33
lemma init_alterp_exec:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    34
  "\<lbrakk>initp_alter s p; p \<in> init_processes; valid (Execute p f # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
    35
  \<Longrightarrow> initp_alter (Execute p f # Clone p (new_proc s) # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    36
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons, frule_tac \<tau> = s in valid_os)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    37
apply (clarsimp simp add:initp_alter_def simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    38
apply (subgoal_tac "p' \<noteq> new_proc s") defer apply (rule notI,simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    39
apply (case_tac "p' = p")
dcde836219bc add thy files
chunhan
parents:
diff changeset
    40
apply (rule_tac x = "new_proc s" in exI) defer
dcde836219bc add thy files
chunhan
parents:
diff changeset
    41
apply (rule_tac x = p' in exI)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    42
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    43
           split:option.splits dest!:current_proc_has_sproc')
dcde836219bc add thy files
chunhan
parents:
diff changeset
    44
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
    45
dcde836219bc add thy files
chunhan
parents:
diff changeset
    46
lemma init_alterp_chown:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    47
  "\<lbrakk>initp_alter s p; p \<in> init_processes; valid (ChangeOwner p u # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
    48
  \<Longrightarrow> initp_alter (ChangeOwner p u # Clone p (new_proc s) # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    49
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons, frule_tac \<tau> = s in valid_os)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    50
apply (clarsimp simp add:initp_alter_def simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    51
apply (subgoal_tac "p' \<noteq> new_proc s") defer apply (rule notI,simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    52
apply (case_tac "p' = p")
dcde836219bc add thy files
chunhan
parents:
diff changeset
    53
apply (rule_tac x = "new_proc s" in exI) defer
dcde836219bc add thy files
chunhan
parents:
diff changeset
    54
apply (rule_tac x = p' in exI)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    55
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    56
           split:option.splits dest!:current_proc_has_sproc')
dcde836219bc add thy files
chunhan
parents:
diff changeset
    57
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
    58
dcde836219bc add thy files
chunhan
parents:
diff changeset
    59
lemma init_alterp_crole:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    60
  "\<lbrakk>initp_alter s p; p \<in> init_processes; valid (ChangeRole p r # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
    61
  \<Longrightarrow> initp_alter (ChangeRole p r # Clone p (new_proc s) # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    62
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons, frule_tac \<tau> = s in valid_os)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    63
apply (clarsimp simp add:initp_alter_def simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    64
apply (subgoal_tac "p' \<noteq> new_proc s") defer apply (rule notI,simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    65
apply (case_tac "p' = p")
dcde836219bc add thy files
chunhan
parents:
diff changeset
    66
apply (rule_tac x = "new_proc s" in exI) defer
dcde836219bc add thy files
chunhan
parents:
diff changeset
    67
apply (rule_tac x = p' in exI)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    68
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    69
           split:option.splits dest!:current_proc_has_sproc')
dcde836219bc add thy files
chunhan
parents:
diff changeset
    70
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
    71
dcde836219bc add thy files
chunhan
parents:
diff changeset
    72
lemma init_alterp_other:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    73
  "\<lbrakk>initp_alter s p; valid (e # s); \<forall> p f. e \<noteq> Execute p f;
dcde836219bc add thy files
chunhan
parents:
diff changeset
    74
    \<forall> p u. e \<noteq> ChangeOwner p u; \<forall> p r. e \<noteq> ChangeRole p r; no_del_event (e # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
    75
  \<Longrightarrow> initp_alter (e # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    76
apply (frule valid_cons, frule valid_os)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    77
apply (clarsimp simp add:initp_alter_def simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    78
apply (subgoal_tac "p' \<noteq> new_proc s") defer apply (rule notI,simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    79
apply (rule_tac x = p' in exI, case_tac e)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    80
apply (auto simp add: cp2sproc_simps' simp del:cp2sproc.simps split:option.splits)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    81
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
    82
dcde836219bc add thy files
chunhan
parents:
diff changeset
    83
lemma initp_intact_butp_I_exec:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    84
  "\<lbrakk>initp_intact_butp s p; p \<in> init_processes; valid (Execute p f # Clone p (new_proc s) # s); 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    85
    no_del_event s\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
    86
  \<Longrightarrow> initp_intact_butp (Execute p f # Clone p (new_proc s) # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
    87
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    88
apply (auto simp add:initp_intact_def initp_intact_butp_def 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    89
            simp del:obj2sobj.simps init_obj2sobj.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    90
               intro:init_alterp_exec)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    91
apply (erule_tac x = pa in allE)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    92
apply (subgoal_tac "pa \<noteq> (new_proc s)")
dcde836219bc add thy files
chunhan
parents:
diff changeset
    93
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
    94
           split:option.splits dest!:current_proc_has_sproc')[1]
dcde836219bc add thy files
chunhan
parents:
diff changeset
    95
apply (rule notI, simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
    96
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
    97
dcde836219bc add thy files
chunhan
parents:
diff changeset
    98
lemma initp_intact_butp_I_chown:
dcde836219bc add thy files
chunhan
parents:
diff changeset
    99
  "\<lbrakk>initp_intact_butp s p; p \<in> init_processes; no_del_event s;
dcde836219bc add thy files
chunhan
parents:
diff changeset
   100
   valid (ChangeOwner p u # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   101
  \<Longrightarrow> initp_intact_butp (ChangeOwner p u # Clone p (new_proc s) # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   102
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   103
apply (auto simp add:initp_intact_def initp_intact_butp_def 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   104
            simp del:obj2sobj.simps init_obj2sobj.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   105
               intro:init_alterp_chown)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   106
apply (erule_tac x = pa in allE)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   107
apply (subgoal_tac "pa \<noteq> (new_proc s)")
dcde836219bc add thy files
chunhan
parents:
diff changeset
   108
apply (auto simp:cp2sproc_simps simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   109
           split:option.splits dest!:current_proc_has_sproc')[1]
dcde836219bc add thy files
chunhan
parents:
diff changeset
   110
apply (rule notI, simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   111
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   112
dcde836219bc add thy files
chunhan
parents:
diff changeset
   113
lemma initp_intact_butp_I_crole:
dcde836219bc add thy files
chunhan
parents:
diff changeset
   114
  "\<lbrakk>initp_intact_butp s p; p \<in> init_processes; 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   115
    valid (ChangeRole p r # Clone p (new_proc s) # s); no_del_event s\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   116
  \<Longrightarrow> initp_intact_butp (ChangeRole p r # Clone p (new_proc s) # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   117
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   118
apply (auto simp add:initp_intact_def initp_intact_butp_def 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   119
            simp del:obj2sobj.simps init_obj2sobj.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   120
               intro:init_alterp_crole)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   121
apply (erule_tac x = pa in allE)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   122
apply (subgoal_tac "pa \<noteq> (new_proc s)")
dcde836219bc add thy files
chunhan
parents:
diff changeset
   123
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   124
           split:option.splits dest!:current_proc_has_sproc')[1]
dcde836219bc add thy files
chunhan
parents:
diff changeset
   125
apply (rule notI, simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   126
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   127
dcde836219bc add thy files
chunhan
parents:
diff changeset
   128
lemma initp_intact_butp_I_others:
dcde836219bc add thy files
chunhan
parents:
diff changeset
   129
  "\<lbrakk>initp_intact_butp s p; valid (e # s); \<forall> p f. e \<noteq> Execute p f;
dcde836219bc add thy files
chunhan
parents:
diff changeset
   130
    \<forall> p u. e \<noteq> ChangeOwner p u; \<forall> p r. e \<noteq> ChangeRole p r; no_del_event (e # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   131
  \<Longrightarrow> initp_intact_butp (e # s) p"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   132
apply (frule valid_os, frule valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   133
apply (simp add:initp_intact_butp_def init_alterp_other 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   134
            del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   135
apply (rule impI|rule allI|erule conjE|rule conjI)+
dcde836219bc add thy files
chunhan
parents:
diff changeset
   136
apply (drule_tac obj = "Proc pa" in nodel_imp_exists, simp, simp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   137
apply (frule no_del_event_cons_D, drule_tac obj = "Proc pa" and s = s in nodel_imp_exists, simp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   138
apply (subgoal_tac "pa \<noteq> new_proc s") defer apply (rule notI,simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   139
apply (rotate_tac 6, erule_tac x = pa in allE, case_tac e)
6
4294abb1f38c update scripts with no new_* in admissable-check
chunhan
parents: 1
diff changeset
   140
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps dest:nodel_imp_exists[where obj = "Proc pa"]
1
dcde836219bc add thy files
chunhan
parents:
diff changeset
   141
           split:option.splits dest!:current_proc_has_sproc')
6
4294abb1f38c update scripts with no new_* in admissable-check
chunhan
parents: 1
diff changeset
   142
apply (drule_tac obj = "Proc nat2" in nodel_imp_exists, simp, simp)+
1
dcde836219bc add thy files
chunhan
parents:
diff changeset
   143
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   144
dcde836219bc add thy files
chunhan
parents:
diff changeset
   145
lemma initp_intact_I_exec:
dcde836219bc add thy files
chunhan
parents:
diff changeset
   146
  "\<lbrakk>initp_intact s; valid (Execute (new_proc s) f # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   147
  \<Longrightarrow> initp_intact (Execute (new_proc s) f # Clone p (new_proc s) # s)"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   148
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   149
apply (auto simp add:initp_intact_def 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   150
            simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   151
apply (erule_tac x = pa in allE)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   152
apply (subgoal_tac "pa \<noteq> (new_proc s)")
dcde836219bc add thy files
chunhan
parents:
diff changeset
   153
apply (auto simp:cp2sproc_simps' cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   154
           split:option.splits dest!:current_proc_has_sproc')[1]
dcde836219bc add thy files
chunhan
parents:
diff changeset
   155
apply (rule notI, simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   156
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   157
dcde836219bc add thy files
chunhan
parents:
diff changeset
   158
lemma initp_intact_I_chown:
dcde836219bc add thy files
chunhan
parents:
diff changeset
   159
  "\<lbrakk>initp_intact s; valid (ChangeOwner (new_proc s) u # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   160
  \<Longrightarrow> initp_intact (ChangeOwner (new_proc s) u # Clone p (new_proc s) # s)"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   161
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   162
apply (auto simp add:initp_intact_def 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   163
            simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   164
apply (erule_tac x = pa in allE)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   165
apply (subgoal_tac "pa \<noteq> (new_proc s)")
dcde836219bc add thy files
chunhan
parents:
diff changeset
   166
apply (auto simp:cp2sproc_simps cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   167
           split:option.splits dest!:current_proc_has_sproc')[1]
dcde836219bc add thy files
chunhan
parents:
diff changeset
   168
apply (rule notI, simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   169
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   170
dcde836219bc add thy files
chunhan
parents:
diff changeset
   171
lemma initp_intact_I_crole:
dcde836219bc add thy files
chunhan
parents:
diff changeset
   172
  "\<lbrakk>initp_intact s; valid (ChangeRole (new_proc s) r # Clone p (new_proc s) # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   173
  \<Longrightarrow> initp_intact (ChangeRole (new_proc s) r # Clone p (new_proc s) # s)"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   174
apply (frule valid_cons, frule_tac \<tau> = s in valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   175
apply (auto simp add:initp_intact_def initp_intact_butp_def 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   176
            simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   177
apply (erule_tac x = pa in allE)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   178
apply (subgoal_tac "pa \<noteq> (new_proc s)")
dcde836219bc add thy files
chunhan
parents:
diff changeset
   179
apply (auto simp:cp2sproc_simps' cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   180
           split:option.splits dest!:current_proc_has_sproc')[1]
dcde836219bc add thy files
chunhan
parents:
diff changeset
   181
apply (rule notI, simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   182
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   183
dcde836219bc add thy files
chunhan
parents:
diff changeset
   184
lemma initp_intact_I_others:
dcde836219bc add thy files
chunhan
parents:
diff changeset
   185
  "\<lbrakk>initp_intact s; valid (e # s); \<forall> p f. e \<noteq> Execute p f;
dcde836219bc add thy files
chunhan
parents:
diff changeset
   186
    \<forall> p u. e \<noteq> ChangeOwner p u; \<forall> p r. e \<noteq> ChangeRole p r; no_del_event (e # s)\<rbrakk>
dcde836219bc add thy files
chunhan
parents:
diff changeset
   187
  \<Longrightarrow> initp_intact (e # s)"
dcde836219bc add thy files
chunhan
parents:
diff changeset
   188
apply (frule valid_os, frule valid_cons)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   189
apply (clarsimp simp add:initp_intact_def simp del:obj2sobj.simps init_obj2sobj.simps)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   190
apply (frule no_del_event_cons_D, drule_tac obj = "Proc p" and s = s in nodel_imp_exists, simp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   191
apply (subgoal_tac "p \<noteq> new_proc s") defer apply (rule notI,simp add:np_notin_curp)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   192
apply (erule_tac x = p in allE, case_tac e)
dcde836219bc add thy files
chunhan
parents:
diff changeset
   193
apply (auto simp:cp2sproc_simps' simp del:cp2sproc.simps 
dcde836219bc add thy files
chunhan
parents:
diff changeset
   194
           split:option.splits dest!:current_proc_has_sproc')
6
4294abb1f38c update scripts with no new_* in admissable-check
chunhan
parents: 1
diff changeset
   195
apply (drule_tac obj = "Proc nat2" in nodel_imp_exists, simp, simp)+
1
dcde836219bc add thy files
chunhan
parents:
diff changeset
   196
done
dcde836219bc add thy files
chunhan
parents:
diff changeset
   197
dcde836219bc add thy files
chunhan
parents:
diff changeset
   198
end
dcde836219bc add thy files
chunhan
parents:
diff changeset
   199
dcde836219bc add thy files
chunhan
parents:
diff changeset
   200
end