diff -r 566b0d1c3669 -r 259a50be4381 Static.thy --- a/Static.thy Sun Jun 16 08:05:37 2013 +0800 +++ b/Static.thy Mon Jun 24 09:01:42 2013 +0800 @@ -463,9 +463,16 @@ where "info_flow_sproc_sshms shms shms' \ (\ sh flag'. (sh, SHM_RDWR) \ shms \ (sh, flag') \ shms')" +(* fun info_flow_sshm :: "t_sproc \ t_sproc \ bool" where "info_flow_sshm (pi,sec,fds,shms) (pi',sec',fds',shms') = info_flow_sproc_sshms shms shms'" +*) +inductive info_flow_sshm :: "t_sproc \ t_sproc \ bool" +where + "info_flow_sshm sp sp" +| "\info_flow_sshm sp (pi,sec,fds,shms); info_flow_sproc_sshms shms shms'\ + \ info_flow_sshm sp (pi',sec',fds',shms')" definition update_ss_shms :: "t_static_state \ t_sproc \ bool \ t_static_state" where