1183 done |
1128 done |
1184 |
1129 |
1185 lemmas cpfd2sfds_simps = cpfd2sfds_open cpfd2sfds_execve cpfd2sfds_clone cpfd2sfds_kill cpfd2sfds_exit |
1130 lemmas cpfd2sfds_simps = cpfd2sfds_open cpfd2sfds_execve cpfd2sfds_clone cpfd2sfds_kill cpfd2sfds_exit |
1186 cpfd2sfds_closefd cpfd2sfds_other |
1131 cpfd2sfds_closefd cpfd2sfds_other |
1187 |
1132 |
1188 (********* ch2sshm simpset ********) |
|
1189 |
|
1190 lemma ch2sshm_createshm: |
|
1191 "valid (CreateShM p h # s) |
|
1192 \<Longrightarrow> ch2sshm (CreateShM p h # s) = (ch2sshm s) (h := |
|
1193 (case (sectxt_of_obj (CreateShM p h # s) (O_shm h)) of |
|
1194 Some sec \<Rightarrow> |
|
1195 Some (if (\<not> deleted (O_shm h) s \<and> h \<in> init_shms) then Init h else Created, sec) |
|
1196 | _ \<Rightarrow> None))" |
|
1197 apply (frule vd_cons, frule vt_grant_os) |
|
1198 apply (auto simp:ch2sshm_def sectxt_of_obj_simps dest!:current_has_sec' split:option.splits if_splits) |
|
1199 done |
|
1200 |
|
1201 lemma ch2sshm_other: |
|
1202 "\<lbrakk>valid (e # s); |
|
1203 \<forall> p h. e \<noteq> CreateShM p h; |
|
1204 h' \<in> current_shms (e # s)\<rbrakk> \<Longrightarrow> ch2sshm (e # s) h' = ch2sshm s h'" |
|
1205 apply (frule vd_cons, frule vt_grant_os) |
|
1206 apply (case_tac e) |
|
1207 apply (auto simp:ch2sshm_def sectxt_of_obj_simps dest!:current_has_sec' split:option.splits if_splits) |
|
1208 done |
|
1209 |
|
1210 lemmas ch2sshm_simps = ch2sshm_createshm ch2sshm_other |
|
1211 |
|
1212 lemma current_shm_has_sh: |
|
1213 "\<lbrakk>h \<in> current_shms s; valid s\<rbrakk> \<Longrightarrow> \<exists> sh. ch2sshm s h = Some sh" |
|
1214 by (auto simp:ch2sshm_def split:option.splits dest!:current_has_sec') |
|
1215 |
|
1216 lemma current_shm_has_sh': |
|
1217 "\<lbrakk>ch2sshm s h = None; valid s\<rbrakk> \<Longrightarrow> h \<notin> current_shms s" |
|
1218 by (auto dest:current_shm_has_sh) |
|
1219 |
|
1220 (********** cph2spshs simpset **********) |
|
1221 |
|
1222 lemma cph2spshs_attach: |
|
1223 "valid (Attach p h flag # s) \<Longrightarrow> |
|
1224 cph2spshs (Attach p h flag # s) = (cph2spshs s) (p := |
|
1225 (case (ch2sshm s h) of |
|
1226 Some sh \<Rightarrow> cph2spshs s p \<union> {(sh, flag)} |
|
1227 | _ \<Rightarrow> cph2spshs s p) )" |
|
1228 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1229 using ch2sshm_other[where e = "Attach p h flag" and s = s] |
|
1230 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1231 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 simp:cph2spshs_def) |
|
1232 apply (erule_tac x = ha in allE, frule procs_of_shm_prop1, simp, simp) |
|
1233 apply (erule_tac x = ha in allE, frule procs_of_shm_prop1, simp, simp) |
|
1234 apply (erule_tac x = ha in allE, frule procs_of_shm_prop1, simp, simp) |
|
1235 apply (erule_tac x = ha in allE, frule procs_of_shm_prop1, simp, simp) |
|
1236 apply (erule_tac x = ha in allE, frule procs_of_shm_prop1, simp, simp) |
|
1237 apply (case_tac "ha = h", simp, frule procs_of_shm_prop1, simp) |
|
1238 apply (rule_tac x = ha in exI, simp) |
|
1239 apply (rule_tac x = ha in exI, simp, drule procs_of_shm_prop1, simp, simp) |
|
1240 apply (rule_tac x = ha in exI, simp) |
|
1241 apply (frule procs_of_shm_prop1, simp, simp) |
|
1242 apply (rule impI, simp) |
|
1243 done |
|
1244 |
|
1245 lemma cph2spshs_detach: "valid (Detach p h # s) \<Longrightarrow> |
|
1246 cph2spshs (Detach p h # s) = (cph2spshs s) (p := |
|
1247 (case (ch2sshm s h, flag_of_proc_shm s p h) of |
|
1248 (Some sh, Some flag) \<Rightarrow> if (\<exists> h'. h' \<noteq> h \<and> (p,flag) \<in> procs_of_shm s h' \<and> ch2sshm s h' = Some sh) |
|
1249 then cph2spshs s p else cph2spshs s p - {(sh, flag)} |
|
1250 | _ \<Rightarrow> cph2spshs s p) )" |
|
1251 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1252 apply (case_tac "x = p") defer |
|
1253 using ch2sshm_other[where e = "Detach p h" and s = s] |
|
1254 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1255 dest!:current_shm_has_sh' procs_of_shm_prop4' dest:procs_of_shm_prop1 procs_of_shm_prop3 simp:cph2spshs_def) [1] |
|
1256 apply (rule_tac x = ha in exI, frule_tac h = ha in procs_of_shm_prop1, simp, simp) |
|
1257 apply (rule_tac x = ha in exI, frule_tac h = ha in procs_of_shm_prop1, simp, simp) |
|
1258 apply (rule impI, simp) |
|
1259 |
|
1260 apply (clarsimp) |
|
1261 apply (frule current_shm_has_sh, simp, erule exE) |
|
1262 apply (frule procs_of_shm_prop4, simp, simp) |
|
1263 apply (rule allI | rule conjI| erule conjE | erule exE | rule impI)+ |
|
1264 |
|
1265 apply (simp only:cph2spshs_def, rule set_eqI, rule iffI) |
|
1266 apply (erule CollectE | erule exE| erule conjE| rule CollectI)+ |
|
1267 apply (case_tac "ha = h", simp) |
|
1268 apply (rule_tac x = sha in exI, rule_tac x = flaga in exI, rule_tac x = ha in exI, simp) |
|
1269 using ch2sshm_other[where e = "Detach p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1270 |
|
1271 apply (erule CollectE | erule exE| erule conjE| rule CollectI)+ |
|
1272 apply (case_tac "ha = h", simp) |
|
1273 apply (rule_tac x = h' in exI, simp) |
|
1274 apply (frule_tac flag = flag and flag' = flaga in procs_of_shm_prop3, simp+) |
|
1275 apply (frule_tac flag = flaga in procs_of_shm_prop4, simp+) |
|
1276 using ch2sshm_other[where e = "Detach p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1277 apply (frule_tac h = h' in procs_of_shm_prop1, simp, simp) |
|
1278 apply (rule_tac x = ha in exI, simp, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1279 using ch2sshm_other[where e = "Detach p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1280 |
|
1281 apply (rule allI | rule conjI| erule conjE | erule exE | rule impI)+ |
|
1282 apply (simp only:cph2spshs_def, rule set_eqI, rule iffI) |
|
1283 apply (erule CollectE | erule exE| erule conjE| rule DiffI |rule CollectI)+ |
|
1284 apply (simp split:if_splits) |
|
1285 apply (rule_tac x = ha in exI, simp, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1286 using ch2sshm_other[where e = "Detach p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1287 apply (rule notI, simp split:if_splits) |
|
1288 apply (erule_tac x = ha in allE, simp, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1289 using ch2sshm_other[where e = "Detach p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1290 apply (erule CollectE | erule exE| erule conjE| erule DiffE |rule CollectI)+ |
|
1291 apply (simp split:if_splits) |
|
1292 apply (erule_tac x = ha in allE, simp, rule_tac x = ha in exI, simp) |
|
1293 apply (case_tac "ha = h", simp add:procs_of_shm_prop3, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1294 using ch2sshm_other[where e = "Detach p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1295 done |
|
1296 |
|
1297 lemma cph2spshs_deleteshm: |
|
1298 "valid (DeleteShM p h # s) \<Longrightarrow> |
|
1299 cph2spshs (DeleteShM p h # s) = (\<lambda> p'. |
|
1300 (case (ch2sshm s h, flag_of_proc_shm s p' h) of |
|
1301 (Some sh, Some flag) \<Rightarrow> if (\<exists> h'. h' \<noteq> h \<and> (p', flag) \<in> procs_of_shm s h' \<and> ch2sshm s h' = Some sh) |
|
1302 then cph2spshs s p' else cph2spshs s p' - {(sh, flag)} |
|
1303 | _ \<Rightarrow> cph2spshs s p') )" |
|
1304 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1305 |
|
1306 apply (clarsimp) |
|
1307 apply (frule current_shm_has_sh, simp, erule exE, simp, simp split:option.splits) |
|
1308 apply (rule conjI, rule impI) |
|
1309 using ch2sshm_other[where e = "DeleteShM p h" and s = s] |
|
1310 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1311 dest!:current_shm_has_sh' procs_of_shm_prop4' dest:procs_of_shm_prop1 procs_of_shm_prop3 simp:cph2spshs_def) [1] |
|
1312 apply (rule_tac x = ha in exI, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1313 apply (rule_tac x = ha in exI, simp) |
|
1314 apply (case_tac "ha = h", simp+, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1315 |
|
1316 apply (rule allI | rule conjI| erule conjE | erule exE | rule impI)+ |
|
1317 |
|
1318 apply (simp only:cph2spshs_def, rule set_eqI, rule iffI) |
|
1319 apply (erule CollectE | erule exE| erule conjE| rule CollectI)+ |
|
1320 apply (case_tac "ha = h", simp) |
|
1321 apply (rule_tac x = sha in exI, rule_tac x = flag in exI, rule_tac x = ha in exI, simp) |
|
1322 using ch2sshm_other[where e = "DeleteShM p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1323 |
|
1324 apply (erule CollectE | erule exE| erule conjE| rule CollectI)+ |
|
1325 apply (case_tac "ha = h", simp) |
|
1326 apply (rule_tac x = h' in exI, simp) |
|
1327 apply (frule_tac flag = flag in procs_of_shm_prop4, simp+) |
|
1328 using ch2sshm_other[where e = "DeleteShM p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1329 apply (frule_tac h = h' in procs_of_shm_prop1, simp, simp) |
|
1330 apply (rule_tac x = ha in exI, simp, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1331 using ch2sshm_other[where e = "DeleteShM p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1332 |
|
1333 apply (rule allI | rule conjI| erule conjE | erule exE | rule impI)+ |
|
1334 apply (simp only:cph2spshs_def, rule set_eqI, rule iffI) |
|
1335 apply (erule CollectE | erule exE| erule conjE| rule DiffI |rule CollectI)+ |
|
1336 apply (simp split:if_splits) |
|
1337 apply (rule_tac x = ha in exI, simp, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1338 using ch2sshm_other[where e = "DeleteShM p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1339 apply (rule notI, simp split:if_splits) |
|
1340 apply (erule_tac x = ha in allE, simp, frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1341 using ch2sshm_other[where e = "DeleteShM p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1342 apply (erule CollectE | erule exE| erule conjE| erule DiffE |rule CollectI)+ |
|
1343 apply (simp split:if_splits) |
|
1344 apply (erule_tac x = ha in allE, simp, rule_tac x = ha in exI, simp) |
|
1345 apply (case_tac "ha = h", simp add:procs_of_shm_prop4) |
|
1346 apply (frule_tac h = ha in procs_of_shm_prop1, simp+) |
|
1347 using ch2sshm_other[where e = "DeleteShM p h" and s = s] apply (simp add:procs_of_shm_prop1) |
|
1348 done |
|
1349 |
|
1350 lemma flag_of_proc_shm_prop1: |
|
1351 "\<lbrakk>flag_of_proc_shm s p h = Some flag; valid s\<rbrakk> \<Longrightarrow> (p, flag) \<in> procs_of_shm s h" |
|
1352 apply (induct s arbitrary:p) |
|
1353 apply (simp add:init_shmflag_has_proc) |
|
1354 apply (frule vt_grant_os, frule vd_cons, case_tac a, auto split:if_splits option.splits) |
|
1355 done |
|
1356 |
|
1357 lemma cph2spshs_clone: |
|
1358 "valid (Clone p p' fds shms # s) \<Longrightarrow> |
|
1359 cph2spshs (Clone p p' fds shms # s) = (cph2spshs s) (p' := |
|
1360 {(sh, flag) | h sh flag. h \<in> shms \<and> ch2sshm s h = Some sh \<and> flag_of_proc_shm s p h = Some flag} )" |
|
1361 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1362 using ch2sshm_other[where e = "Clone p p' fds shms" and s = s] |
|
1363 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1364 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 simp:cph2spshs_def) |
|
1365 apply (erule_tac x = h in allE, frule procs_of_shm_prop1, simp, simp add:procs_of_shm_prop4) |
|
1366 apply (rule_tac x = h in exI, simp, frule flag_of_proc_shm_prop1, simp+, simp add:procs_of_shm_prop1) |
|
1367 apply (rule_tac x = h in exI, simp, frule procs_of_shm_prop1, simp+)+ |
|
1368 done |
|
1369 |
|
1370 lemma cph2spshs_execve: |
|
1371 "valid (Execve p f fds # s) \<Longrightarrow> |
|
1372 cph2spshs (Execve p f fds # s) = (cph2spshs s) (p := {})" |
|
1373 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1374 using ch2sshm_other[where e = "Execve p f fds" and s = s] |
|
1375 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1376 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 simp:cph2spshs_def) |
|
1377 apply (rule_tac x = h in exI, simp add:procs_of_shm_prop1)+ |
|
1378 done |
|
1379 |
|
1380 lemma cph2spshs_kill: |
|
1381 "valid (Kill p p' # s) \<Longrightarrow> cph2spshs (Kill p p' # s) = (cph2spshs s) (p' := {})" |
|
1382 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1383 using ch2sshm_other[where e = "Kill p p'" and s = s] |
|
1384 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1385 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 simp:cph2spshs_def) |
|
1386 apply (rule_tac x = h in exI, simp add:procs_of_shm_prop1)+ |
|
1387 done |
|
1388 |
|
1389 lemma cph2spshs_exit: |
|
1390 "valid (Exit p # s) \<Longrightarrow> cph2spshs (Exit p # s) = (cph2spshs s) (p := {})" |
|
1391 apply (frule vd_cons, frule vt_grant_os, rule ext) |
|
1392 using ch2sshm_other[where e = "Exit p" and s = s] |
|
1393 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1394 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 simp:cph2spshs_def) |
|
1395 apply (rule_tac x = h in exI, simp add:procs_of_shm_prop1)+ |
|
1396 done |
|
1397 |
|
1398 lemma cph2spshs_createshm: |
|
1399 "valid (CreateShM p h # s) \<Longrightarrow> cph2spshs (CreateShM p h # s) = cph2spshs s" |
|
1400 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1401 apply (auto simp:cph2spshs_def) |
|
1402 using ch2sshm_createshm |
|
1403 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1404 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 simp:cph2spshs_def) |
|
1405 apply (rule_tac x = ha in exI, auto simp:procs_of_shm_prop1) |
|
1406 done |
|
1407 |
|
1408 lemma cph2spshs_other: |
|
1409 "\<lbrakk>valid (e # s); |
|
1410 \<forall> p h flag. e \<noteq> Attach p h flag; |
|
1411 \<forall> p h. e \<noteq> Detach p h; |
|
1412 \<forall> p h. e \<noteq> DeleteShM p h; |
|
1413 \<forall> p p' fds shms. e \<noteq> Clone p p' fds shms; |
|
1414 \<forall> p f fds. e \<noteq> Execve p f fds; |
|
1415 \<forall> p p'. e \<noteq> Kill p p'; |
|
1416 \<forall> p. e \<noteq> Exit p\<rbrakk> \<Longrightarrow> cph2spshs (e # s) = cph2spshs s" |
|
1417 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1418 unfolding cph2spshs_def |
|
1419 apply (rule set_eqI, rule iffI) |
|
1420 apply (erule CollectE | erule conjE| erule exE| rule conjI| rule impI| rule CollectI)+ |
|
1421 apply (frule procs_of_shm_prop1, simp, rule_tac x= sh in exI, rule_tac x = flag in exI, rule_tac x = h in exI) |
|
1422 apply (case_tac e) |
|
1423 using ch2sshm_other[where e = e and s = s] |
|
1424 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1425 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 |
|
1426 simp:ch2sshm_createshm) |
|
1427 apply (rule_tac x = h in exI, case_tac e) |
|
1428 using ch2sshm_other[where e = e and s = s] |
|
1429 apply (auto split del:t_open_must_flag.splits t_open_option_flag.splits split add:if_splits option.splits |
|
1430 dest!:current_shm_has_sh' dest: procs_of_shm_prop1 procs_of_shm_prop2 procs_of_shm_prop3 |
|
1431 simp:ch2sshm_createshm) |
|
1432 done |
|
1433 |
|
1434 lemmas cph2spshs_simps = cph2spshs_attach cph2spshs_detach cph2spshs_deleteshm cph2spshs_clone cph2spshs_execve |
|
1435 cph2spshs_exit cph2spshs_kill cph2spshs_other |
|
1436 |
|
1437 (******** cp2sproc simpset *********) |
|
1438 |
|
1439 lemma cp2sproc_clone: |
1133 lemma cp2sproc_clone: |
1440 "valid (Clone p p' fds shms # s) \<Longrightarrow> cp2sproc (Clone p p' fds shms # s) = (cp2sproc s) (p' := |
1134 "valid (Clone p p' fds # s) \<Longrightarrow> cp2sproc (Clone p p' fds # s) = (cp2sproc s) (p' := |
1441 case (sectxt_of_obj s (O_proc p)) of |
1135 case (sectxt_of_obj s (O_proc p)) of |
1442 Some sec \<Rightarrow> Some (Created, sec, |
1136 Some sec \<Rightarrow> Some (Created, sec, |
1443 {sfd. \<exists> fd \<in> fds. \<exists> f. file_of_proc_fd s p fd = Some f \<and> cfd2sfd s p fd = Some sfd}, |
1137 {sfd. \<exists> fd \<in> fds. \<exists> f. file_of_proc_fd s p fd = Some f \<and> cfd2sfd s p fd = Some sfd}) |
1444 {(sh, flag) | h sh flag. h \<in> shms \<and> ch2sshm s h = Some sh \<and> flag_of_proc_shm s p h = Some flag}) |
|
1445 | _ \<Rightarrow> None)" |
1138 | _ \<Rightarrow> None)" |
1446 apply (frule cph2spshs_clone, frule cpfd2sfds_clone) |
1139 apply (frule cpfd2sfds_clone) |
1447 apply (frule vd_cons, frule vt_grant_os, simp only:os_grant.simps) |
1140 apply (frule vd_cons, frule vt_grant_os, simp only:os_grant.simps) |
1448 apply ((erule exE| erule conjE)+, frule not_init_intro_proc, simp, rule ext, case_tac "x = p'", simp) |
1141 apply ((erule exE| erule conjE)+, frule not_init_intro_proc, simp, rule ext, case_tac "x = p'", simp) |
1449 apply (auto simp:cp2sproc_def sectxt_of_obj_simps dest!:current_has_sec' |
1142 apply (auto simp:cp2sproc_def sectxt_of_obj_simps dest!:current_has_sec' |
1450 dest:current_proc_has_sec split:option.splits if_splits) |
1143 dest:current_proc_has_sec split:option.splits if_splits) |
1451 done |
1144 done |
1452 |
1145 |
1453 lemma cp2sproc_other: |
1146 lemma cp2sproc_other: |
1454 "\<lbrakk>valid (e # s); |
1147 "\<lbrakk>valid (e # s); |
1455 \<forall> p f flags fd opt. e \<noteq> Open p f flags fd opt; |
1148 \<forall> p f flags fd opt. e \<noteq> Open p f flags fd opt; |
1456 \<forall> p fd. e \<noteq> CloseFd p fd; |
1149 \<forall> p fd. e \<noteq> CloseFd p fd; |
1457 \<forall> p h flag. e \<noteq> Attach p h flag; |
1150 \<forall> p p' fds. e \<noteq> Clone p p' fds; |
1458 \<forall> p h. e \<noteq> Detach p h; |
|
1459 \<forall> p h. e \<noteq> DeleteShM p h; |
|
1460 \<forall> p p' fds shms. e \<noteq> Clone p p' fds shms; |
|
1461 \<forall> p f fds. e \<noteq> Execve p f fds; |
1151 \<forall> p f fds. e \<noteq> Execve p f fds; |
1462 \<forall> p p'. e \<noteq> Kill p p'; |
1152 \<forall> p p'. e \<noteq> Kill p p'; |
1463 \<forall> p. e \<noteq> Exit p\<rbrakk> \<Longrightarrow> cp2sproc (e # s) = cp2sproc s" |
1153 \<forall> p. e \<noteq> Exit p\<rbrakk> \<Longrightarrow> cp2sproc (e # s) = cp2sproc s" |
1464 apply (frule cph2spshs_other, simp+, frule cpfd2sfds_other, simp+) |
1154 apply (frule cpfd2sfds_other, simp+) |
1465 apply (frule vt_grant_os, frule vd_cons, rule ext, case_tac e, simp_all) |
1155 apply (frule vt_grant_os, frule vd_cons, rule ext, case_tac e, simp_all) |
1466 apply (auto simp:cp2sproc_def sectxt_of_obj_simps dest!:current_has_sec' |
1156 apply (auto simp:cp2sproc_def sectxt_of_obj_simps dest!:current_has_sec' |
1467 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1157 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1468 done |
1158 done |
1469 |
1159 |
1492 Some sfd \<Rightarrow> (if (\<exists> fd' f'. fd' \<noteq> fd \<and> file_of_proc_fd s p fd' = Some f' \<and> cfd2sfd s p fd' = Some sfd) |
1181 Some sfd \<Rightarrow> (if (\<exists> fd' f'. fd' \<noteq> fd \<and> file_of_proc_fd s p fd' = Some f' \<and> cfd2sfd s p fd' = Some sfd) |
1493 then cp2sproc s p |
1182 then cp2sproc s p |
1494 else (case (sectxt_of_obj s (O_proc p)) of |
1183 else (case (sectxt_of_obj s (O_proc p)) of |
1495 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p) s \<and> p \<in> init_procs) |
1184 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p) s \<and> p \<in> init_procs) |
1496 then Init p else Created, |
1185 then Init p else Created, |
1497 sec, cpfd2sfds s p - {sfd}, cph2spshs s p) |
1186 sec, cpfd2sfds s p - {sfd}) |
1498 | _ \<Rightarrow> None)) |
1187 | _ \<Rightarrow> None)) |
1499 | _ \<Rightarrow> cp2sproc s p) |
1188 | _ \<Rightarrow> cp2sproc s p) |
1500 else cp2sproc s p)" |
1189 else cp2sproc s p)" |
1501 apply (frule cpfd2sfds_closefd, frule cph2spshs_other, simp, simp, simp, simp, simp, simp, simp) |
1190 apply (frule cpfd2sfds_closefd) |
1502 apply (frule vt_grant_os, frule vd_cons, rule ext) |
1191 apply (frule vt_grant_os, frule vd_cons, rule ext) |
1503 apply (case_tac "x = p") |
1192 apply (case_tac "x = p") |
1504 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
1193 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
1505 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
1194 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
1506 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1195 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1507 done |
1196 done |
1508 |
1197 |
1509 lemma cp2sproc_attach: |
|
1510 "valid (Attach p h flag # s) \<Longrightarrow> |
|
1511 cp2sproc (Attach p h flag # s) = (cp2sproc s) (p := |
|
1512 (case (ch2sshm s h) of |
|
1513 Some sh \<Rightarrow> (case (sectxt_of_obj s (O_proc p)) of |
|
1514 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p) s \<and> p \<in> init_procs) |
|
1515 then Init p else Created, |
|
1516 sec, cpfd2sfds s p, cph2spshs s p \<union> {(sh, flag)}) |
|
1517 | _ \<Rightarrow> None) |
|
1518 | _ \<Rightarrow> cp2sproc s p) )" |
|
1519 apply (frule cph2spshs_attach, frule cpfd2sfds_other, simp, simp, simp, simp, simp, simp) |
|
1520 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1521 apply (case_tac "x = p") |
|
1522 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
|
1523 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
|
1524 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
|
1525 done |
|
1526 |
|
1527 lemma cp2sproc_detach: |
|
1528 "valid (Detach p h # s) \<Longrightarrow> |
|
1529 cp2sproc (Detach p h # s) = (cp2sproc s) (p := |
|
1530 (case (ch2sshm s h, flag_of_proc_shm s p h) of |
|
1531 (Some sh, Some flag) \<Rightarrow> if (\<exists> h'. h' \<noteq> h \<and> (p,flag) \<in> procs_of_shm s h' \<and> ch2sshm s h' = Some sh) |
|
1532 then cp2sproc s p |
|
1533 else (case (sectxt_of_obj s (O_proc p)) of |
|
1534 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p) s \<and> p \<in> init_procs) |
|
1535 then Init p else Created, sec, |
|
1536 cpfd2sfds s p, cph2spshs s p - {(sh, flag)}) |
|
1537 | None \<Rightarrow> None) |
|
1538 | _ \<Rightarrow> cp2sproc s p) )" |
|
1539 apply (frule cph2spshs_detach, frule cpfd2sfds_other, simp, simp, simp, simp, simp, simp) |
|
1540 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1541 apply (case_tac "x = p") |
|
1542 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
|
1543 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
|
1544 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
|
1545 done |
|
1546 |
|
1547 lemma cp2sproc_deleteshm: |
|
1548 "valid (DeleteShM p h # s) \<Longrightarrow> |
|
1549 cp2sproc (DeleteShM p h # s) = (\<lambda> p'. |
|
1550 (case (ch2sshm s h, flag_of_proc_shm s p' h) of |
|
1551 (Some sh, Some flag) \<Rightarrow> if (\<exists> h'. h' \<noteq> h \<and> (p', flag) \<in> procs_of_shm s h' \<and> ch2sshm s h' = Some sh) |
|
1552 then cp2sproc s p' |
|
1553 else (case (sectxt_of_obj s (O_proc p')) of |
|
1554 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p') s \<and> p' \<in> init_procs) |
|
1555 then Init p' else Created, sec, |
|
1556 cpfd2sfds s p', cph2spshs s p' - {(sh, flag)}) |
|
1557 | None \<Rightarrow> None) |
|
1558 | _ \<Rightarrow> cp2sproc s p') )" |
|
1559 apply (frule cph2spshs_deleteshm, frule cpfd2sfds_other, simp, simp, simp, simp, simp, simp) |
|
1560 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1561 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
|
1562 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
|
1563 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
|
1564 done |
|
1565 |
|
1566 lemma cp2sproc_execve: |
1198 lemma cp2sproc_execve: |
1567 "valid (Execve p f fds # s) \<Longrightarrow> |
1199 "valid (Execve p f fds # s) \<Longrightarrow> |
1568 cp2sproc (Execve p f fds # s) = (cp2sproc s) (p := |
1200 cp2sproc (Execve p f fds # s) = (cp2sproc s) (p := |
1569 (case (sectxt_of_obj (Execve p f fds # s) (O_proc p)) of |
1201 (case (sectxt_of_obj (Execve p f fds # s) (O_proc p)) of |
1570 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p) s \<and> p \<in> init_procs) then Init p else Created, sec, |
1202 Some sec \<Rightarrow> Some (if (\<not> deleted (O_proc p) s \<and> p \<in> init_procs) then Init p else Created, sec, |
1571 {sfd. \<exists> fd \<in> fds. \<exists> f. file_of_proc_fd s p fd = Some f \<and> cfd2sfd s p fd = Some sfd}, {}) |
1203 {sfd. \<exists> fd \<in> fds. \<exists> f. file_of_proc_fd s p fd = Some f \<and> cfd2sfd s p fd = Some sfd}) |
1572 | _ \<Rightarrow> None) )" |
1204 | _ \<Rightarrow> None) )" |
1573 apply (frule cph2spshs_execve, frule cpfd2sfds_execve) |
1205 apply (frule cpfd2sfds_execve) |
1574 apply (frule vt_grant_os, frule vd_cons, rule ext) |
1206 apply (frule vt_grant_os, frule vd_cons, rule ext) |
1575 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
1207 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
1576 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
1208 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
1577 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1209 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1578 done |
1210 done |
1579 |
1211 |
1580 lemma cp2sproc_kill: |
1212 lemma cp2sproc_kill: |
1581 "\<lbrakk>valid (Kill p p' # s); p'' \<noteq> p'\<rbrakk> \<Longrightarrow> |
1213 "\<lbrakk>valid (Kill p p' # s); p'' \<noteq> p'\<rbrakk> \<Longrightarrow> |
1582 cp2sproc (Kill p p' # s) p'' = (cp2sproc s) p''" |
1214 cp2sproc (Kill p p' # s) p'' = (cp2sproc s) p''" |
1583 apply (frule cph2spshs_kill, frule cpfd2sfds_kill) |
1215 apply (frule cpfd2sfds_kill) |
1584 apply (frule vt_grant_os, frule vd_cons) |
1216 apply (frule vt_grant_os, frule vd_cons) |
1585 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
1217 apply (auto simp:cp2sproc_def sectxt_of_obj_simps current_files_simps |
1586 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
1218 dest!:current_has_sec' dest!:current_file_has_sfile' dest:is_file_in_current is_dir_in_current |
1587 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1219 dest:current_proc_has_sec not_deleted_init_proc split:option.splits if_splits) |
1588 done |
1220 done |
1605 lemma cp2sproc_exit': |
1237 lemma cp2sproc_exit': |
1606 "\<lbrakk>valid (Exit p # s); p' \<in> current_procs (Exit p # s)\<rbrakk> \<Longrightarrow> |
1238 "\<lbrakk>valid (Exit p # s); p' \<in> current_procs (Exit p # s)\<rbrakk> \<Longrightarrow> |
1607 cp2sproc (Exit p # s) p' = (cp2sproc s) p'" |
1239 cp2sproc (Exit p # s) p' = (cp2sproc s) p'" |
1608 by (drule_tac p'= p' in cp2sproc_exit, simp+) |
1240 by (drule_tac p'= p' in cp2sproc_exit, simp+) |
1609 |
1241 |
1610 lemmas cp2sproc_simps = cp2sproc_open cp2sproc_closefd cp2sproc_attach cp2sproc_detach cp2sproc_deleteshm |
1242 lemmas cp2sproc_simps = cp2sproc_open cp2sproc_closefd cp2sproc_clone cp2sproc_execve |
1611 cp2sproc_clone cp2sproc_execve cp2sproc_kill cp2sproc_exit cp2sproc_other |
1243 cp2sproc_kill cp2sproc_exit cp2sproc_other |
1612 |
1244 |
1613 lemma current_proc_has_sp: |
1245 lemma current_proc_has_sp: |
1614 "\<lbrakk>p \<in> current_procs s; valid s\<rbrakk> \<Longrightarrow> \<exists> sp. cp2sproc s p = Some sp" |
1246 "\<lbrakk>p \<in> current_procs s; valid s\<rbrakk> \<Longrightarrow> \<exists> sp. cp2sproc s p = Some sp" |
1615 by (auto simp:cp2sproc_def split:option.splits dest!:current_has_sec') |
1247 by (auto simp:cp2sproc_def split:option.splits dest!:current_has_sec') |
1616 |
1248 |
1617 lemma current_proc_has_sp': |
1249 lemma current_proc_has_sp': |
1618 "\<lbrakk>cp2sproc s p = None; valid s\<rbrakk> \<Longrightarrow> p \<notin> current_procs s" |
1250 "\<lbrakk>cp2sproc s p = None; valid s\<rbrakk> \<Longrightarrow> p \<notin> current_procs s" |
1619 by (auto dest:current_proc_has_sp) |
1251 by (auto dest:current_proc_has_sp) |
1620 |
|
1621 |
|
1622 |
|
1623 (* simpset for cf2sfiles *) |
|
1624 |
|
1625 lemma cf2sfiles_open: |
|
1626 "\<lbrakk>valid (Open p f flag fd opt # s); f' \<in> current_files (Open p f flag fd opt # s)\<rbrakk> |
|
1627 \<Longrightarrow> cf2sfiles (Open p f flag fd opt # s) f' = ( |
|
1628 if (f' = f \<and> opt \<noteq> None) |
|
1629 then (case cf2sfile (Open p f flag fd opt # s) f of |
|
1630 Some sf \<Rightarrow> {sf} |
|
1631 | _ \<Rightarrow> {} ) |
|
1632 else cf2sfiles s f')" |
|
1633 apply (frule vt_grant_os, frule vd_cons) |
|
1634 apply (auto simp:cf2sfiles_def cf2sfile_open_none cf2sfile_simps same_inode_files_open |
|
1635 split:if_splits option.splits dest!:current_file_has_sfile' dest:cf2sfile_open) |
|
1636 apply (rule_tac x = "f'a" in bexI, drule same_inode_files_prop1, simp add:cf2sfile_open_some1, simp)+ |
|
1637 done |
|
1638 |
|
1639 lemma cf2sfiles_other: |
|
1640 "\<lbrakk>valid (e # s); |
|
1641 \<forall> p f flag fd opt. e \<noteq> Open p f flag fd opt; |
|
1642 \<forall> p fd. e \<noteq> CloseFd p fd; |
|
1643 \<forall> p f. e \<noteq> UnLink p f; |
|
1644 \<forall> p f f'. e \<noteq> LinkHard p f f'\<rbrakk> \<Longrightarrow> cf2sfiles (e # s) = cf2sfiles s" |
|
1645 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1646 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI) |
|
1647 apply (drule Set.CollectD, erule bexE, rule CollectI) |
|
1648 apply (rule_tac x = f' in bexI, case_tac e) |
|
1649 apply (auto simp:cf2sfiles_def cf2sfile_simps same_inode_files_simps current_files_simps |
|
1650 split:if_splits option.splits dest!:current_file_has_sfile' dest:same_inode_files_prop1 cf2sfile_other') |
|
1651 apply (drule_tac f' = f' in cf2sfile_rmdir) |
|
1652 apply (simp add:current_files_simps same_inode_files_prop1 same_inode_files_prop3 dir_is_empty_def)+ |
|
1653 |
|
1654 apply (rule_tac x = f' in bexI, case_tac e) |
|
1655 apply (auto simp:cf2sfiles_def cf2sfile_simps same_inode_files_simps current_files_simps |
|
1656 split:if_splits option.splits dest!:current_file_has_sfile' dest:same_inode_files_prop1 cf2sfile_other') |
|
1657 apply (drule_tac f' = f' in cf2sfile_rmdir) |
|
1658 apply (simp add:current_files_simps same_inode_files_prop1 same_inode_files_prop3 dir_is_empty_def)+ |
|
1659 done |
|
1660 |
|
1661 lemma cf2sfile_linkhard1': |
|
1662 "\<lbrakk>valid (LinkHard p oldf f # s); f' \<in> same_inode_files s f''\<rbrakk> |
|
1663 \<Longrightarrow> cf2sfile (LinkHard p oldf f# s) f' = cf2sfile s f'" |
|
1664 apply (drule same_inode_files_prop1) |
|
1665 by (simp add:cf2sfile_linkhard1) |
|
1666 |
|
1667 lemma cf2sfiles_linkhard: |
|
1668 "valid (LinkHard p oldf f # s) \<Longrightarrow> cf2sfiles (LinkHard p oldf f # s) = (\<lambda> f'. |
|
1669 if (f' = f \<or> f' \<in> same_inode_files s oldf) |
|
1670 then (case (cf2sfile (LinkHard p oldf f # s) f) of |
|
1671 Some sf \<Rightarrow> cf2sfiles s oldf \<union> {sf} |
|
1672 | _ \<Rightarrow> {}) |
|
1673 else cf2sfiles s f')" |
|
1674 apply (frule vt_grant_os, frule vd_cons, rule ext) |
|
1675 apply (auto simp:cf2sfiles_def cf2sfile_linkhard1' same_inode_files_linkhard current_files_linkhard |
|
1676 split:if_splits option.splits dest!:current_file_has_sfile' current_has_sec' dest:same_inode_files_prop1) |
|
1677 done |
|
1678 |
|
1679 lemma cf2sfile_unlink': |
|
1680 "\<lbrakk>valid (UnLink p f # s); f' \<in> same_inode_files (UnLink p f # s) f''\<rbrakk> |
|
1681 \<Longrightarrow> cf2sfile (UnLink p f # s) f' = cf2sfile s f'" |
|
1682 apply (drule same_inode_files_prop1) |
|
1683 by (simp add:cf2sfile_unlink) |
|
1684 |
|
1685 lemma cf2sfiles_unlink: |
|
1686 "\<lbrakk>valid (UnLink p f # s); f' \<in> current_files (UnLink p f # s)\<rbrakk> \<Longrightarrow> cf2sfiles (UnLink p f # s) f' = ( |
|
1687 if (f' \<in> same_inode_files s f \<and> proc_fd_of_file s f = {} \<and> |
|
1688 (\<forall> f'' \<in> same_inode_files s f. f'' \<noteq> f \<longrightarrow> cf2sfile s f'' \<noteq> cf2sfile s f)) then |
|
1689 (case (cf2sfile s f) of |
|
1690 Some sf \<Rightarrow> cf2sfiles s f' - {sf} |
|
1691 | _ \<Rightarrow> {}) |
|
1692 else cf2sfiles s f')" |
|
1693 apply (frule vt_grant_os, frule vd_cons, simp add:current_files_simps split:if_splits) |
|
1694 apply (rule conjI, clarify, frule is_file_has_sfile', simp, erule exE, simp) |
|
1695 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1696 apply (erule bexE, frule_tac f' = f' in same_inode_files_unlink) |
|
1697 apply (simp add:current_files_unlink, simp, erule conjE) |
|
1698 apply (erule_tac x = f'a in ballE, frule_tac f' = "f'a" in cf2sfile_unlink) |
|
1699 apply (simp add:current_files_unlink same_inode_files_prop1, simp) |
|
1700 apply (rule_tac x = f'a in bexI, simp, simp) |
|
1701 apply (drule_tac f = f and f' = f' and f'' = f'a in same_inode_files_prop4, simp+) |
|
1702 apply (erule conjE|erule exE|erule bexE)+ |
|
1703 apply (case_tac "f'a = f", simp) |
|
1704 apply (frule_tac f' = f' in same_inode_files_unlink, simp add:current_files_unlink) |
|
1705 apply (frule_tac f' = f'a in cf2sfile_unlink, simp add:current_files_unlink same_inode_files_prop1) |
|
1706 apply (rule_tac x = f'a in bexI, simp, simp) |
|
1707 |
|
1708 apply (rule impI)+ |
|
1709 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1710 apply (erule bexE, frule_tac f' = f' in same_inode_files_unlink) |
|
1711 apply (simp add:current_files_unlink, simp, (erule conjE)+) |
|
1712 apply (rule_tac x = f'a in bexI, frule_tac f' = "f'a" in cf2sfile_unlink) |
|
1713 apply (simp add:current_files_unlink same_inode_files_prop1, simp, simp) |
|
1714 apply (drule CollectD, erule bexE, frule_tac f' = f' in same_inode_files_unlink) |
|
1715 apply (simp add:current_files_unlink, simp) |
|
1716 apply (case_tac "f'a = f", simp) |
|
1717 apply (frule_tac f = f' and f' = f in same_inode_files_prop5, simp) |
|
1718 apply (erule bexE, erule conjE) |
|
1719 apply (rule_tac x = f'' in bexI) |
|
1720 apply (drule_tac f' = f'' in cf2sfile_unlink, simp add:current_files_unlink same_inode_files_prop1) |
|
1721 apply (simp, simp, erule same_inode_files_prop4, simp) |
|
1722 apply (rule_tac x = f'a in bexI) |
|
1723 apply (drule_tac f' = f'a in cf2sfile_unlink, simp add:current_files_unlink same_inode_files_prop1) |
|
1724 apply (simp, simp) |
|
1725 |
|
1726 |
|
1727 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1728 apply (erule bexE, frule_tac f' = f' in same_inode_files_unlink) |
|
1729 apply (simp add:current_files_unlink, simp) |
|
1730 apply (rule_tac x = f'a in bexI) |
|
1731 apply (frule_tac f' = f'a in cf2sfile_unlink) |
|
1732 apply (simp add:same_inode_files_prop1 current_files_unlink, simp, simp) |
|
1733 apply (drule CollectD, erule bexE, frule_tac f' = f' in same_inode_files_unlink) |
|
1734 apply (simp add:current_files_unlink, simp) |
|
1735 apply (rule_tac x = f'a in bexI) |
|
1736 apply (frule_tac f' = f'a in cf2sfile_unlink) |
|
1737 apply (simp add:same_inode_files_prop1 current_files_unlink, simp, simp) |
|
1738 done |
|
1739 |
|
1740 lemma cf2sfiles_closefd: |
|
1741 "\<lbrakk>valid (CloseFd p fd # s); f' \<in> current_files (CloseFd p fd # s)\<rbrakk> \<Longrightarrow> cf2sfiles (CloseFd p fd # s) f' = ( |
|
1742 case (file_of_proc_fd s p fd) of |
|
1743 Some f \<Rightarrow> if (f' \<in> same_inode_files s f \<and> proc_fd_of_file s f = {(p, fd)} \<and> f \<in> files_hung_by_del s \<and> |
|
1744 (\<forall> f'' \<in> same_inode_files s f. f'' \<noteq> f \<longrightarrow> cf2sfile s f'' \<noteq> cf2sfile s f)) |
|
1745 then (case (cf2sfile s f) of |
|
1746 Some sf \<Rightarrow> cf2sfiles s f' - {sf} |
|
1747 | _ \<Rightarrow> {}) |
|
1748 else cf2sfiles s f' |
|
1749 | _ \<Rightarrow> cf2sfiles s f')" |
|
1750 |
|
1751 apply (frule vt_grant_os, frule vd_cons, case_tac "file_of_proc_fd s p fd") |
|
1752 apply (simp_all add:current_files_simps split:if_splits) |
|
1753 |
|
1754 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1755 apply (erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1756 apply (simp add:current_files_closefd, simp) |
|
1757 apply (rule_tac x = f'a in bexI) |
|
1758 apply (frule_tac f = f'a in cf2sfile_closefd) |
|
1759 apply (simp add:same_inode_files_prop1 current_files_closefd, simp, simp) |
|
1760 apply (drule CollectD, erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1761 apply (simp add:current_files_closefd, simp) |
|
1762 apply (rule_tac x = f'a in bexI) |
|
1763 apply (frule_tac f = f'a in cf2sfile_closefd) |
|
1764 apply (simp add:same_inode_files_prop1 current_files_closefd, simp, simp) |
|
1765 |
|
1766 apply (rule conjI, clarify, frule file_of_pfd_is_file, simp) |
|
1767 apply (frule is_file_has_sfile', simp, erule exE, simp) |
|
1768 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1769 apply (erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1770 apply (simp add:current_files_closefd, simp, erule conjE) |
|
1771 apply (erule_tac x = f'a in ballE, frule_tac f = "f'a" in cf2sfile_closefd) |
|
1772 apply (simp add:current_files_closefd same_inode_files_prop1, simp) |
|
1773 apply (rule_tac x = f'a in bexI, simp, simp) |
|
1774 apply (drule_tac f = a and f' = f' and f'' = f'a in same_inode_files_prop4, simp+) |
|
1775 apply (erule conjE|erule exE|erule bexE)+ |
|
1776 apply (case_tac "f'a = a", simp) |
|
1777 apply (frule_tac f' = f' in same_inode_files_closefd, simp add:current_files_closefd, simp) |
|
1778 apply (frule_tac f = f'a in cf2sfile_closefd, simp add:current_files_closefd same_inode_files_prop1) |
|
1779 apply (rule_tac x = f'a in bexI, simp, simp) |
|
1780 |
|
1781 apply (rule impI)+ |
|
1782 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1783 apply (erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1784 apply (simp add:current_files_closefd, simp, (erule conjE)+) |
|
1785 apply (rule_tac x = f'a in bexI, frule_tac f = f'a in cf2sfile_closefd) |
|
1786 apply (simp add:current_files_closefd same_inode_files_prop1, simp, simp) |
|
1787 apply (drule CollectD, erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1788 apply (simp add:current_files_closefd, simp) |
|
1789 apply (case_tac "f'a = a", simp) |
|
1790 apply (frule_tac f = f' and f' = a in same_inode_files_prop5, simp) |
|
1791 apply (erule bexE, erule conjE) |
|
1792 apply (rule_tac x = f'' in bexI) |
|
1793 apply (drule_tac f = f'' in cf2sfile_closefd, simp add:current_files_closefd same_inode_files_prop1) |
|
1794 apply (simp, simp, erule same_inode_files_prop4, simp) |
|
1795 apply (rule_tac x = f'a in bexI) |
|
1796 apply (drule_tac f = f'a in cf2sfile_closefd, simp add:current_files_closefd same_inode_files_prop1) |
|
1797 apply (simp, simp) |
|
1798 |
|
1799 apply (rule conjI, clarify) |
|
1800 |
|
1801 apply (rule impI) |
|
1802 apply (case_tac "a \<in> files_hung_by_del s", simp_all) |
|
1803 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1804 apply (erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1805 apply (simp add:current_files_closefd, simp) |
|
1806 apply (rule_tac x = f'a in bexI) |
|
1807 apply (frule_tac f = f'a in cf2sfile_closefd) |
|
1808 apply (simp add:same_inode_files_prop1 current_files_closefd, simp, simp) |
|
1809 apply (drule CollectD, erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1810 apply (simp add:current_files_closefd, simp) |
|
1811 apply (rule_tac x = f'a in bexI) |
|
1812 apply (frule_tac f = f'a in cf2sfile_closefd) |
|
1813 apply (simp add:same_inode_files_prop1 current_files_closefd, simp, simp) |
|
1814 apply (simp add:cf2sfiles_def, rule set_eqI, rule iffI, drule CollectD) |
|
1815 apply (erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1816 apply (simp add:current_files_closefd, simp) |
|
1817 apply (rule_tac x = f'a in bexI) |
|
1818 apply (frule_tac f = f'a in cf2sfile_closefd) |
|
1819 apply (simp add:same_inode_files_prop1 current_files_closefd, simp, simp) |
|
1820 apply (drule CollectD, erule bexE, frule_tac f' = f' in same_inode_files_closefd) |
|
1821 apply (simp add:current_files_closefd, simp) |
|
1822 apply (rule_tac x = f'a in bexI) |
|
1823 apply (frule_tac f = f'a in cf2sfile_closefd) |
|
1824 apply (simp add:same_inode_files_prop1 current_files_closefd, simp, simp) |
|
1825 done |
|
1826 |
|
1827 lemmas cf2sfiles_simps = cf2sfiles_open cf2sfiles_linkhard cf2sfiles_other |
|
1828 cf2sfiles_unlink cf2sfiles_closefd |
|
1829 |
|
1830 |
1252 |
1831 (* simpset for co2sobj *) |
1253 (* simpset for co2sobj *) |
1832 |
1254 |
1833 lemma co2sobj_execve: |
1255 lemma co2sobj_execve: |
1834 "\<lbrakk>valid (Execve p f fds # s); alive (Execve p f fds # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Execve p f fds # s) obj = ( |
1256 "\<lbrakk>valid (Execve p f fds # s); alive (Execve p f fds # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Execve p f fds # s) obj = ( |
1835 if (obj = O_proc p) |
1257 if (obj = O_proc p) |
1836 then (case (cp2sproc (Execve p f fds # s) p) of |
1258 then (case (cp2sproc (Execve p f fds # s) p) of |
1837 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s \<or> O_file f \<in> Tainted s)) |
1259 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> tainted s \<or> O_file f \<in> tainted s)) |
1838 | _ \<Rightarrow> None) |
1260 | _ \<Rightarrow> None) |
1839 else co2sobj s obj )" |
1261 else co2sobj s obj )" |
1840 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1262 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1841 apply (simp_all add:current_files_simps cf2sfiles_other ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1263 apply (simp_all add:current_files_simps cq2smsgq_other cf2sfile_other) |
1842 apply (case_tac "cp2sproc (Execve p f fds # s) p") |
1264 apply (case_tac "cp2sproc (Execve p f fds # s) p") |
1843 apply (drule current_proc_has_sp', simp, simp) |
1265 apply (drule current_proc_has_sp', simp, simp) |
1844 apply (simp (no_asm_simp) add:cp2sproc_execve tainted_eq_Tainted split:option.splits) |
1266 apply (simp (no_asm_simp) add:cp2sproc_execve split:option.splits) |
|
1267 apply (simp add:is_file_simps, frule_tac s = s in is_file_has_sfile', simp, erule exE, simp) |
|
1268 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
|
1269 apply (simp add:is_file_in_current) |
1845 apply (simp add:is_dir_simps, frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1270 apply (simp add:is_dir_simps, frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1846 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1271 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1847 apply (simp add:is_dir_in_current) |
1272 apply (simp add:is_dir_in_current) |
1848 done |
1273 done |
1849 |
1274 |
1850 lemma co2sobj_execve': |
1275 lemma co2sobj_execve': |
1851 "\<lbrakk>valid (Execve p f fds # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Execve p f fds # s) obj = ( |
1276 "\<lbrakk>valid (Execve p f fds # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Execve p f fds # s) obj = ( |
1852 if (obj = O_proc p) |
1277 if (obj = O_proc p) |
1853 then (case (cp2sproc (Execve p f fds # s) p) of |
1278 then (case (cp2sproc (Execve p f fds # s) p) of |
1854 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s \<or> O_file f \<in> Tainted s)) |
1279 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> tainted s \<or> O_file f \<in> tainted s)) |
1855 | _ \<Rightarrow> None) |
1280 | _ \<Rightarrow> None) |
1856 else co2sobj s obj )" |
1281 else co2sobj s obj )" |
1857 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1282 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1858 apply (simp_all add:current_files_simps cf2sfiles_other ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1283 apply (simp_all add:current_files_simps cf2sfile_other cq2smsgq_other) |
1859 apply (case_tac "cp2sproc (Execve p f fds # s) p") |
1284 apply (case_tac "cp2sproc (Execve p f fds # s) p") |
1860 apply (drule current_proc_has_sp', simp, simp) |
1285 apply (drule current_proc_has_sp', simp, simp) |
1861 apply (simp (no_asm_simp) add:cp2sproc_execve tainted_eq_Tainted split:option.splits) |
1286 apply (simp (no_asm_simp) add:cp2sproc_execve split:option.splits) |
|
1287 apply (frule_tac s = s in is_file_has_sfile', simp, erule exE, simp) |
|
1288 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
|
1289 apply (simp add:is_file_in_current) |
1862 apply (frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1290 apply (frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1863 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1291 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1864 apply (simp add:is_dir_in_current) |
1292 apply (simp add:is_dir_in_current) |
1865 done |
1293 done |
1866 |
1294 |
1867 lemma co2sobj_clone': |
1295 lemma co2sobj_clone': |
1868 "\<lbrakk>valid (Clone p p' fds shms # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Clone p p' fds shms # s) obj = ( |
1296 "\<lbrakk>valid (Clone p p' fds # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Clone p p' fds # s) obj = ( |
1869 if (obj = O_proc p') |
1297 if (obj = O_proc p') |
1870 then (case (cp2sproc (Clone p p' fds shms # s) p') of |
1298 then (case (cp2sproc (Clone p p' fds # s) p') of |
1871 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s)) |
1299 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> tainted s)) |
1872 | _ \<Rightarrow> None) |
1300 | _ \<Rightarrow> None) |
1873 else co2sobj s obj )" |
1301 else co2sobj s obj )" |
1874 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1302 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1875 apply (simp_all add:current_files_simps cf2sfiles_other ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1303 apply (simp_all add:current_files_simps cf2sfile_other cq2smsgq_other ) |
1876 apply (case_tac "cp2sproc (Clone p p' fds shms # s) p'") |
1304 apply (case_tac "cp2sproc (Clone p p' fds # s) p'") |
1877 apply (drule current_proc_has_sp', simp, simp) |
1305 apply (drule current_proc_has_sp', simp, simp) |
1878 apply ((erule conjE)+, frule_tac p = p in current_proc_has_sec, simp, erule exE, simp) |
1306 apply ((erule conjE)+, frule_tac p = p in current_proc_has_sec, simp, erule exE, simp) |
1879 apply (rule conjI, rule impI, simp) |
1307 apply (simp (no_asm_simp) add:cp2sproc_clone split:option.splits) |
1880 apply (simp (no_asm_simp) add:cp2sproc_clone tainted_eq_Tainted split:option.splits) |
1308 apply (case_tac "nat = p'", simp, simp) |
1881 |
1309 apply (frule_tac s = s in is_file_has_sfile', simp, erule exE, simp) |
|
1310 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
|
1311 apply (simp add:is_file_in_current) |
1882 apply (frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1312 apply (frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1883 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1313 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1884 apply (simp add:is_dir_in_current) |
1314 apply (simp add:is_dir_in_current) |
1885 done |
1315 done |
1886 |
1316 |
1887 lemma co2sobj_clone: |
1317 lemma co2sobj_clone: |
1888 "\<lbrakk>valid (Clone p p' fds shms # s); alive (Clone p p' fds shms # s) obj\<rbrakk> |
1318 "\<lbrakk>valid (Clone p p' fds # s); alive (Clone p p' fds # s) obj\<rbrakk> |
1889 \<Longrightarrow> co2sobj (Clone p p' fds shms # s) obj = ( |
1319 \<Longrightarrow> co2sobj (Clone p p' fds # s) obj = ( |
1890 if (obj = O_proc p') |
1320 if (obj = O_proc p') |
1891 then (case (cp2sproc (Clone p p' fds shms # s) p') of |
1321 then (case (cp2sproc (Clone p p' fds # s) p') of |
1892 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s)) |
1322 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> tainted s)) |
1893 | _ \<Rightarrow> None) |
1323 | _ \<Rightarrow> None) |
1894 else co2sobj s obj )" |
1324 else co2sobj s obj )" |
1895 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1325 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1896 apply (simp_all add:current_files_simps cf2sfiles_other ch2sshm_other |
1326 apply (simp_all add:current_files_simps cf2sfile_other cq2smsgq_other) |
1897 cq2smsgq_other tainted_eq_Tainted) |
|
1898 apply (rule conjI, rule impI, simp) |
1327 apply (rule conjI, rule impI, simp) |
1899 apply (case_tac "cp2sproc (Clone p p' fds shms # s) p'") |
1328 apply (case_tac "cp2sproc (Clone p p' fds # s) p'") |
1900 apply (drule current_proc_has_sp', simp, simp) |
1329 apply (drule current_proc_has_sp', simp, simp) |
1901 apply ((erule conjE)+, frule_tac p = p in current_proc_has_sec, simp, erule exE, simp) |
1330 apply ((erule conjE)+, frule_tac p = p in current_proc_has_sec, simp, erule exE, simp) |
1902 apply (simp add:tainted_eq_Tainted, rule impI, rule notI) |
1331 apply (rule impI,rule notI, drule tainted_in_current, simp+) |
1903 apply (drule Tainted_in_current, simp+) |
|
1904 apply (rule impI, simp) |
1332 apply (rule impI, simp) |
1905 apply (drule current_proc_has_sp, simp, (erule exE|erule conjE)+) |
1333 apply (drule current_proc_has_sp, simp, (erule exE|erule conjE)+) |
1906 apply (simp (no_asm_simp) add:cp2sproc_clone tainted_eq_Tainted Tainted_in_current split:option.splits) |
1334 apply (simp (no_asm_simp) add:cp2sproc_clone tainted_in_current split:option.splits) |
1907 |
1335 |
|
1336 apply (simp add:is_file_simps, frule_tac s = s in is_file_has_sfile', simp, erule exE, simp) |
|
1337 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
|
1338 apply (simp add:is_file_in_current) |
1908 apply (simp add:is_dir_simps, frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1339 apply (simp add:is_dir_simps, frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1909 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1340 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1910 apply (simp add:is_dir_in_current) |
1341 apply (simp add:is_dir_in_current) |
1911 done |
1342 done |
1912 |
1343 |
1913 lemma co2sobj_ptrace: |
1344 lemma co2sobj_ptrace: |
1914 "\<lbrakk>valid (Ptrace p p' # s); alive s obj\<rbrakk>\<Longrightarrow> co2sobj (Ptrace p p' # s) obj = ( |
1345 "\<lbrakk>valid (Ptrace p p' # s); alive s obj\<rbrakk>\<Longrightarrow> co2sobj (Ptrace p p' # s) obj = ( |
1915 case obj of |
1346 case obj of |
1916 O_proc p'' \<Rightarrow> if (info_flow_shm s p' p'') |
1347 O_proc p'' \<Rightarrow> if (p'' = p') |
1917 then (case (cp2sproc s p'') of |
1348 then (case (cp2sproc s p'') of |
1918 Some sp \<Rightarrow> Some (S_proc sp (O_proc p'' \<in> Tainted s \<or> O_proc p \<in> Tainted s)) |
1349 Some sp \<Rightarrow> Some (S_proc sp (O_proc p'' \<in> tainted s \<or> O_proc p \<in> tainted s)) |
1919 | _ \<Rightarrow> None) |
1350 | _ \<Rightarrow> None) |
1920 else if (info_flow_shm s p p'') |
1351 else if (p'' = p) |
1921 then (case (cp2sproc s p'') of |
1352 then (case (cp2sproc s p'') of |
1922 Some sp \<Rightarrow> Some (S_proc sp (O_proc p'' \<in> Tainted s \<or> O_proc p' \<in> Tainted s)) |
1353 Some sp \<Rightarrow> Some (S_proc sp (O_proc p'' \<in> tainted s \<or> O_proc p' \<in> tainted s)) |
1923 | _ \<Rightarrow> None) |
1354 | _ \<Rightarrow> None) |
1924 else co2sobj s (O_proc p'') |
1355 else co2sobj s (O_proc p'') |
1925 | _ \<Rightarrow> co2sobj s obj)" |
1356 | _ \<Rightarrow> co2sobj s obj)" |
1926 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1357 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1927 apply (simp_all add:current_files_simps ch2sshm_other cq2smsgq_other cf2sfiles_other tainted_eq_Tainted) |
1358 apply (simp_all add:current_files_simps cq2smsgq_other cf2sfile_other) |
1928 |
1359 |
1929 apply (auto simp:cp2sproc_other tainted_eq_Tainted split:option.splits |
1360 apply (auto simp:cp2sproc_other split:option.splits |
1930 dest!:current_proc_has_sec' current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
1361 dest!:current_proc_has_sec' current_proc_has_sp')[1] |
1931 |
1362 |
|
1363 apply (frule_tac s = s in is_file_has_sfile', simp, erule exE, simp) |
|
1364 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
|
1365 apply (simp add:is_file_in_current) |
1932 apply (frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1366 apply (frule_tac s = s in is_dir_has_sdir', simp, erule exE, simp) |
1933 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1367 apply (frule_tac ff = list in cf2sfile_other', simp_all) |
1934 apply (simp add:is_dir_in_current) |
1368 apply (simp add:is_dir_in_current) |
1935 done |
1369 done |
1936 |
1370 |
1937 lemma co2sobj_open: |
1371 lemma co2sobj_open: |
1938 "\<lbrakk>valid (Open p f flag fd opt # s); alive (Open p f flag fd opt # s) obj\<rbrakk> |
1372 "\<lbrakk>valid (Open p f flag fd opt # s); alive (Open p f flag fd opt # s) obj\<rbrakk> |
1939 \<Longrightarrow> co2sobj (Open p f flag fd opt # s) obj = (case obj of |
1373 \<Longrightarrow> co2sobj (Open p f flag fd opt # s) obj = (case obj of |
1940 O_file f' \<Rightarrow> if (f' = f \<and> opt \<noteq> None) |
1374 O_file f' \<Rightarrow> if (f' = f \<and> opt \<noteq> None) |
1941 then (case (cf2sfile (Open p f flag fd opt # s) f) of |
1375 then (case (cf2sfile (Open p f flag fd opt # s) f) of |
1942 Some sf \<Rightarrow> Some (S_file {sf} (O_proc p \<in> Tainted s)) |
1376 Some sf \<Rightarrow> Some (S_file sf (O_proc p \<in> tainted s)) |
1943 | _ \<Rightarrow> None) |
1377 | _ \<Rightarrow> None) |
1944 else co2sobj s (O_file f') |
1378 else co2sobj s (O_file f') |
1945 | O_proc p' \<Rightarrow> if (p' = p) |
1379 | O_proc p' \<Rightarrow> if (p' = p) |
1946 then (case (cp2sproc (Open p f flag fd opt # s) p) of |
1380 then (case (cp2sproc (Open p f flag fd opt # s) p) of |
1947 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s)) |
1381 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> tainted s)) |
1948 | _ \<Rightarrow> None) |
1382 | _ \<Rightarrow> None) |
1949 else co2sobj s (O_proc p') |
1383 else co2sobj s (O_proc p') |
1950 | _ \<Rightarrow> co2sobj s obj )" |
1384 | _ \<Rightarrow> co2sobj s obj )" |
1951 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1385 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1952 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits |
1386 apply (auto simp:cp2sproc_simps split:option.splits dest!:current_proc_has_sp')[1] |
1953 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
|
1954 |
1387 |
1955 apply (simp split:if_splits t_object.splits) |
1388 apply (simp split:if_splits t_object.splits) |
1956 apply (rule conjI, rule impI, erule conjE, erule exE, simp, (erule exE|erule conjE)+) |
1389 apply (rule conjI, rule impI, erule conjE, erule exE, simp, (erule exE|erule conjE)+) |
1957 apply (case_tac "cf2sfile (Open p f flag fd (Some y) # s) f") |
1390 apply (case_tac "cf2sfile (Open p f flag fd (Some y) # s) f") |
1958 apply (drule current_file_has_sfile', simp, simp add:current_files_simps, simp) |
1391 apply (drule current_file_has_sfile', simp, simp add:current_files_simps, simp) |
1959 apply (frule_tac f' = f in cf2sfiles_open, simp add:current_files_simps) |
1392 apply (frule_tac f' = f in cf2sfile_open, simp add:current_files_simps) |
1960 apply (simp add:tainted_eq_Tainted) |
1393 apply (rule impI, rule notI, drule tainted_in_current, simp, simp add:is_file_in_current) |
1961 apply (rule impI, rule notI, drule Tainted_in_current, simp, simp add:is_file_in_current) |
1394 apply (rule impI, simp add:cf2sfile_open is_file_in_current split:option.splits) |
1962 apply (rule impI, simp add:tainted_eq_Tainted cf2sfiles_open is_file_in_current split:option.splits) |
1395 |
1963 |
1396 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
1964 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
1965 |
1397 |
1966 apply (frule is_dir_in_current) |
1398 apply (frule is_dir_in_current) |
1967 apply (frule_tac f' = list in cf2sfile_open) |
1399 apply (frule_tac f' = list in cf2sfile_open) |
1968 apply (simp add:current_files_simps split:option.splits) |
1400 apply (simp add:current_files_simps split:option.splits) |
1969 apply (simp split:if_splits option.splits) |
1401 apply (simp split:if_splits option.splits) |
1971 |
1403 |
1972 lemma co2sobj_readfile: |
1404 lemma co2sobj_readfile: |
1973 "\<lbrakk>valid (ReadFile p fd # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (ReadFile p fd # s) obj = ( |
1405 "\<lbrakk>valid (ReadFile p fd # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (ReadFile p fd # s) obj = ( |
1974 case obj of |
1406 case obj of |
1975 O_proc p' \<Rightarrow> (case (file_of_proc_fd s p fd) of |
1407 O_proc p' \<Rightarrow> (case (file_of_proc_fd s p fd) of |
1976 Some f \<Rightarrow> (if (info_flow_shm s p p' \<and> O_file f \<in> Tainted s) |
1408 Some f \<Rightarrow> (if (p' = p \<and> O_file f \<in> tainted s) |
1977 then (case (cp2sproc s p') of |
1409 then (case (cp2sproc s p') of |
1978 Some sp \<Rightarrow> Some (S_proc sp True) |
1410 Some sp \<Rightarrow> Some (S_proc sp True) |
1979 | _ \<Rightarrow> None) |
1411 | _ \<Rightarrow> None) |
1980 else co2sobj s obj) |
1412 else co2sobj s obj) |
1981 | _ \<Rightarrow> None) |
1413 | _ \<Rightarrow> None) |
1982 | _ \<Rightarrow> co2sobj s obj)" |
1414 | _ \<Rightarrow> co2sobj s obj)" |
1983 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1415 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1984 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits |
1416 apply (auto simp:cp2sproc_simps split:option.splits dest!:current_proc_has_sp')[1] |
1985 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
1417 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
1986 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
1987 |
1418 |
1988 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' |
1419 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' |
1989 simp:current_files_simps cf2sfiles_simps cf2sfile_simps |
1420 simp:current_files_simps cf2sfile_simps |
1990 dest:is_file_in_current is_dir_in_current) |
1421 dest:is_file_in_current is_dir_in_current) |
1991 done |
1422 done |
1992 |
1423 |
1993 lemma co2sobj_writefile: |
1424 lemma co2sobj_writefile: |
1994 "\<lbrakk>valid (WriteFile p fd # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (WriteFile p fd # s) obj = ( |
1425 "\<lbrakk>valid (WriteFile p fd # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (WriteFile p fd # s) obj = ( |
1995 case obj of |
1426 case obj of |
1996 O_file f' \<Rightarrow> (case (file_of_proc_fd s p fd) of |
1427 O_file f' \<Rightarrow> (case (file_of_proc_fd s p fd) of |
1997 Some f \<Rightarrow> (if (f \<in> same_inode_files s f') |
1428 Some f \<Rightarrow> (if (f' = f) |
1998 then Some (S_file (cf2sfiles s f') |
1429 then (case cf2sfile s f of |
1999 (O_file f' \<in> Tainted s \<or> O_proc p \<in> Tainted s)) |
1430 Some sf \<Rightarrow> Some (S_file sf (O_file f \<in> tainted s \<or> O_proc p \<in> tainted s)) |
|
1431 | _ \<Rightarrow> None) |
2000 else co2sobj s obj) |
1432 else co2sobj s obj) |
2001 | _ \<Rightarrow> None) |
1433 | _ \<Rightarrow> None) |
2002 | _ \<Rightarrow> co2sobj s obj)" |
1434 | _ \<Rightarrow> co2sobj s obj)" |
2003 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1435 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2004 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1436 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
2005 |
1437 |
2006 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
1438 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
2007 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
1439 simp:current_files_simps cf2sfile_simps cp2sproc_simps |
2008 same_inode_files_prop6 |
|
2009 dest:is_file_in_current is_dir_in_current) |
1440 dest:is_file_in_current is_dir_in_current) |
2010 |
1441 done |
2011 (* should delete has_same_inode !?!?*) |
|
2012 by (auto simp:same_inode_files_def is_file_def has_same_inode_def split:if_splits option.splits) |
|
2013 |
1442 |
2014 lemma co2sobj_closefd: |
1443 lemma co2sobj_closefd: |
2015 "\<lbrakk>valid (CloseFd p fd # s); alive (CloseFd p fd # s) obj\<rbrakk> \<Longrightarrow> co2sobj (CloseFd p fd # s) obj = ( |
1444 "\<lbrakk>valid (CloseFd p fd # s); alive (CloseFd p fd # s) obj\<rbrakk> \<Longrightarrow> co2sobj (CloseFd p fd # s) obj = ( |
2016 case obj of |
1445 case obj of |
2017 O_file f' \<Rightarrow> (case (file_of_proc_fd s p fd) of |
1446 O_proc p' \<Rightarrow> (if (p = p') |
2018 Some f \<Rightarrow> (if (f' \<in> same_inode_files s f \<and> proc_fd_of_file s f = {(p, fd)} \<and> |
|
2019 f \<in> files_hung_by_del s \<and> (\<forall> f'' \<in> same_inode_files s f. |
|
2020 f'' \<noteq> f \<longrightarrow> cf2sfile s f'' \<noteq> cf2sfile s f)) |
|
2021 then (case (cf2sfile s f, co2sobj s (O_file f')) of |
|
2022 (Some sf, Some (S_file sfs b)) \<Rightarrow> Some (S_file (sfs - {sf}) b) |
|
2023 | _ \<Rightarrow> None) |
|
2024 else co2sobj s obj) |
|
2025 | _ \<Rightarrow> co2sobj s obj) |
|
2026 | O_proc p' \<Rightarrow> (if (p = p') |
|
2027 then (case (cp2sproc (CloseFd p fd # s) p) of |
1447 then (case (cp2sproc (CloseFd p fd # s) p) of |
2028 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s)) |
1448 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> tainted s)) |
2029 | _ \<Rightarrow> None) |
1449 | _ \<Rightarrow> None) |
2030 else co2sobj s obj) |
1450 else co2sobj s obj) |
2031 | _ \<Rightarrow> co2sobj s obj) " |
1451 | _ \<Rightarrow> co2sobj s obj) " |
2032 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1452 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2033 apply (simp_all add:current_files_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1453 apply (simp_all add:current_files_simps cq2smsgq_other) |
2034 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits if_splits |
1454 apply (auto simp:cp2sproc_simps split:option.splits if_splits dest!:current_proc_has_sp')[1] |
2035 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
|
2036 |
1455 |
2037 apply (frule is_file_in_current) |
1456 apply (frule is_file_in_current) |
2038 apply (case_tac "file_of_proc_fd s p fd") |
1457 apply (case_tac "file_of_proc_fd s p fd") |
2039 apply (simp add:tainted_eq_Tainted) |
1458 apply (simp add:current_files_simps is_file_simps tainted.simps) |
2040 apply (drule_tac f' = list in cf2sfiles_closefd, simp add:current_files_closefd, simp) |
1459 apply (drule_tac f = list in cf2sfile_closefd, simp add:current_files_simps) |
2041 apply (frule_tac f' = list in cf2sfiles_closefd, simp) |
1460 apply (simp split:option.splits) |
2042 apply (simp add:is_file_simps current_files_simps) |
1461 apply (frule_tac f = list in cf2sfile_closefd, simp) |
2043 apply (auto simp add:tainted_eq_Tainted cf2sfile_closefd split:if_splits option.splits |
1462 apply (simp split:option.splits) |
2044 dest!:current_file_has_sfile' dest:hung_file_in_current)[1] |
1463 apply (simp add:is_file_simps current_files_simps split:if_splits) |
|
1464 apply (rule impI, simp) |
2045 |
1465 |
2046 apply (simp add:is_dir_simps, frule is_dir_in_current) |
1466 apply (simp add:is_dir_simps, frule is_dir_in_current) |
2047 apply (frule_tac f = list in cf2sfile_closefd) |
1467 apply (frule_tac f = list in cf2sfile_closefd) |
2048 apply (clarsimp simp:current_files_closefd split:option.splits) |
1468 apply (clarsimp simp:current_files_closefd split:option.splits) |
2049 apply (drule file_of_pfd_is_file', simp+) |
1469 apply (drule file_of_pfd_is_file', simp+) |
2050 done |
1470 done |
2051 |
1471 |
2052 lemma co2sobj_unlink: |
1472 lemma co2sobj_unlink: |
2053 "\<lbrakk>valid (UnLink p f # s); alive (UnLink p f # s) obj\<rbrakk> \<Longrightarrow> co2sobj (UnLink p f # s) obj = ( |
1473 "\<lbrakk>valid (UnLink p f # s); alive (UnLink p f # s) obj\<rbrakk> |
2054 case obj of |
1474 \<Longrightarrow> co2sobj (UnLink p f # s) obj = co2sobj s obj" |
2055 O_file f' \<Rightarrow> if (f' \<in> same_inode_files s f \<and> proc_fd_of_file s f = {} \<and> |
1475 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2056 (\<forall> f'' \<in> same_inode_files s f. f'' \<noteq> f \<longrightarrow> cf2sfile s f'' \<noteq> cf2sfile s f)) |
1476 apply (simp_all add:current_files_simps cq2smsgq_other) |
2057 then (case (cf2sfile s f, co2sobj s (O_file f')) of |
1477 apply (auto simp:cp2sproc_simps split:option.splits if_splits dest!:current_proc_has_sp')[1] |
2058 (Some sf, Some (S_file sfs b)) \<Rightarrow> Some (S_file (sfs - {sf}) b) |
|
2059 | _ \<Rightarrow> None) |
|
2060 else co2sobj s obj |
|
2061 | _ \<Rightarrow> co2sobj s obj)" |
|
2062 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
|
2063 apply (simp_all add:current_files_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
2064 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits if_splits |
|
2065 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
|
2066 apply (frule is_file_in_current) |
1478 apply (frule is_file_in_current) |
2067 apply (frule_tac f' = list in cf2sfile_unlink, simp) |
1479 apply (frule_tac f' = list in cf2sfile_unlink, simp) |
2068 apply (frule_tac f' = list in cf2sfiles_unlink, simp) |
1480 apply (simp add:is_file_simps current_files_simps split:option.splits if_splits) |
2069 apply (simp add:is_file_simps current_files_simps) |
|
2070 apply (auto simp add:tainted_eq_Tainted is_file_in_current split:if_splits option.splits |
|
2071 dest!:current_file_has_sfile')[1] |
|
2072 |
1481 |
2073 apply (simp add:is_dir_simps, frule is_dir_in_current) |
1482 apply (simp add:is_dir_simps, frule is_dir_in_current) |
2074 apply (frule_tac f' = list in cf2sfile_unlink) |
1483 apply (frule_tac f' = list in cf2sfile_unlink) |
2075 apply (clarsimp simp:current_files_unlink split:option.splits) |
1484 apply (clarsimp simp:current_files_unlink split:option.splits) |
2076 apply (drule file_dir_conflict, simp+) |
1485 apply (drule file_dir_conflict, simp+) |
2077 done |
1486 done |
2078 |
1487 |
2079 lemma co2sobj_rmdir: |
1488 lemma co2sobj_rmdir: |
2080 "\<lbrakk>valid (Rmdir p f # s); alive (Rmdir p f # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Rmdir p f # s) obj = co2sobj s obj" |
1489 "\<lbrakk>valid (Rmdir p f # s); alive (Rmdir p f # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Rmdir p f # s) obj = co2sobj s obj" |
2081 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1490 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2082 apply (simp_all add:current_files_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1491 apply (simp_all add:current_files_simps cq2smsgq_other) |
2083 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits if_splits |
1492 apply (auto simp:cp2sproc_simps split:option.splits if_splits dest!:current_proc_has_sp')[1] |
2084 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
|
2085 apply (simp add:is_file_simps dir_is_empty_def) |
1493 apply (simp add:is_file_simps dir_is_empty_def) |
2086 apply (case_tac "f = list", drule file_dir_conflict, simp, simp) |
1494 apply (case_tac "f = list", drule file_dir_conflict, simp, simp) |
2087 apply (simp add:cf2sfiles_other) |
1495 apply (frule_tac f' = list in cf2sfile_rmdir, simp add:is_file_in_current current_files_simps) |
2088 apply (auto simp:cf2sfile_simps dest:is_dir_in_current) |
1496 apply (simp split:option.splits) |
|
1497 apply (auto simp:cf2sfile_simps cf2sfile_other dest:is_dir_in_current) |
2089 done |
1498 done |
2090 |
1499 |
2091 lemma co2sobj_mkdir: |
1500 lemma co2sobj_mkdir: |
2092 "\<lbrakk>valid (Mkdir p f i # s); alive (Mkdir p f i # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Mkdir p f i # s) obj = ( |
1501 "\<lbrakk>valid (Mkdir p f i # s); alive (Mkdir p f i # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Mkdir p f i # s) obj = ( |
2093 if (obj = O_dir f) |
1502 if (obj = O_dir f) |
2094 then (case (cf2sfile (Mkdir p f i # s) f) of |
1503 then (case (cf2sfile (Mkdir p f i # s) f) of |
2095 Some sf \<Rightarrow> Some (S_dir sf) |
1504 Some sf \<Rightarrow> Some (S_dir sf) |
2096 | _ \<Rightarrow> None) |
1505 | _ \<Rightarrow> None) |
2097 else co2sobj s obj)" |
1506 else co2sobj s obj)" |
2098 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1507 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2099 apply (simp_all add:current_files_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1508 apply (simp_all add:current_files_simps cq2smsgq_other) |
2100 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits if_splits |
1509 apply (auto simp:cp2sproc_simps split:option.splits if_splits dest!:current_proc_has_sp')[1] |
2101 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
1510 apply (case_tac "f = list", simp add:is_file_simps is_file_in_current) |
2102 apply (frule_tac cf2sfiles_other, simp+) |
1511 apply (frule_tac f' = list in cf2sfile_mkdir) |
|
1512 apply (simp add:is_file_in_current) |
|
1513 apply (simp split:option.splits) |
|
1514 |
2103 apply (frule is_dir_in_current, rule impI, simp add:current_files_mkdir) |
1515 apply (frule is_dir_in_current, rule impI, simp add:current_files_mkdir) |
2104 apply (frule current_file_has_sfile, simp, erule exE, simp) |
1516 apply (frule current_file_has_sfile, simp, erule exE, simp) |
2105 apply (drule cf2sfile_mkdir1, simp+) |
1517 apply (drule cf2sfile_mkdir1, simp+) |
2106 done |
1518 done |
2107 |
1519 |
2108 |
|
2109 lemma co2sobj_linkhard: |
|
2110 "\<lbrakk>valid (LinkHard p oldf f # s); alive (LinkHard p oldf f # s) obj\<rbrakk> |
|
2111 \<Longrightarrow> co2sobj (LinkHard p oldf f # s) obj = ( |
|
2112 case obj of |
|
2113 O_file f' \<Rightarrow> if (f' = f \<or> f' \<in> same_inode_files s oldf) |
|
2114 then (case (cf2sfile (LinkHard p oldf f # s) f) of |
|
2115 Some sf \<Rightarrow> Some (S_file (cf2sfiles s oldf \<union> {sf}) (O_file oldf \<in> Tainted s)) |
|
2116 | _ \<Rightarrow> None) |
|
2117 else co2sobj s obj |
|
2118 | _ \<Rightarrow> co2sobj s obj)" |
|
2119 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
|
2120 apply (simp_all add:current_files_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
2121 apply (auto simp:cp2sproc_simps tainted_eq_Tainted split:option.splits if_splits |
|
2122 dest!:current_proc_has_sp' intro:info_flow_shm_Tainted)[1] |
|
2123 apply (frule_tac cf2sfiles_linkhard, simp+) |
|
2124 apply (frule_tac f' = f in cf2sfile_linkhard, simp add:current_files_linkhard) |
|
2125 apply (auto simp:is_file_simps sectxt_of_obj_simps current_files_simps is_file_in_current same_inodes_Tainted |
|
2126 split:option.splits if_splits dest:Tainted_in_current |
|
2127 dest!:current_has_sec' current_file_has_sfile')[1] |
|
2128 |
|
2129 apply (frule is_dir_in_current, simp add:current_files_linkhard is_dir_simps is_dir_in_current) |
|
2130 apply (frule is_dir_in_current) |
|
2131 apply (frule current_file_has_sfile, simp) |
|
2132 apply (drule cf2sfile_linkhard1, simp+) |
|
2133 done |
|
2134 |
|
2135 lemma co2sobj_truncate: |
1520 lemma co2sobj_truncate: |
2136 "\<lbrakk>valid (Truncate p f len # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Truncate p f len # s) obj = ( |
1521 "\<lbrakk>valid (Truncate p f len # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Truncate p f len # s) obj = ( |
2137 case obj of |
1522 case obj of |
2138 O_file f' \<Rightarrow> if (f' \<in> same_inode_files s f \<and> len > 0) |
1523 O_file f' \<Rightarrow> if (f' = f \<and> len > 0) |
2139 then Some (S_file (cf2sfiles s f') (O_file f' \<in> Tainted s \<or> O_proc p \<in> Tainted s)) |
1524 then (case cf2sfile s f of |
|
1525 Some sf \<Rightarrow> Some (S_file sf (O_file f' \<in> tainted s \<or> O_proc p \<in> tainted s)) |
|
1526 | _ \<Rightarrow> None) |
2140 else co2sobj s obj |
1527 else co2sobj s obj |
2141 | _ \<Rightarrow> co2sobj s obj)" |
1528 | _ \<Rightarrow> co2sobj s obj)" |
2142 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1529 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2143 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1530 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
2144 |
1531 |
2145 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
1532 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
2146 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
1533 simp:current_files_simps cf2sfile_simps cp2sproc_simps |
2147 same_inode_files_prop6 |
|
2148 dest:is_file_in_current is_dir_in_current) |
1534 dest:is_file_in_current is_dir_in_current) |
2149 done |
1535 done |
2150 |
1536 |
2151 lemma co2sobj_kill: |
1537 lemma co2sobj_kill: |
2152 "\<lbrakk>valid (Kill p p' # s); alive (Kill p p' # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Kill p p' # s) obj = co2sobj s obj" |
1538 "\<lbrakk>valid (Kill p p' # s); alive (Kill p p' # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Kill p p' # s) obj = co2sobj s obj" |
2153 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1539 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2154 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1540 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
2155 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
1541 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
2156 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
1542 simp:current_files_simps cf2sfile_simps cp2sproc_simps |
2157 same_inode_files_prop6 |
|
2158 dest:is_file_in_current is_dir_in_current) |
1543 dest:is_file_in_current is_dir_in_current) |
2159 done |
1544 done |
2160 |
1545 |
2161 lemma co2sobj_exit: |
1546 lemma co2sobj_exit: |
2162 "\<lbrakk>valid (Exit p # s); alive (Exit p # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Exit p # s) obj = co2sobj s obj" |
1547 "\<lbrakk>valid (Exit p # s); alive (Exit p # s) obj\<rbrakk> \<Longrightarrow> co2sobj (Exit p # s) obj = co2sobj s obj" |
2163 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1548 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2164 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1549 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other ) |
2165 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
1550 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
2166 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
1551 simp:current_files_simps cf2sfile_simps cp2sproc_simps |
2167 same_inode_files_prop6 |
|
2168 dest:is_file_in_current is_dir_in_current) |
1552 dest:is_file_in_current is_dir_in_current) |
2169 done |
1553 done |
2170 |
1554 |
2171 lemma co2sobj_createmsgq: |
1555 lemma co2sobj_createmsgq: |
2172 "\<lbrakk>valid (CreateMsgq p q # s); alive (CreateMsgq p q # s) obj\<rbrakk> \<Longrightarrow> co2sobj (CreateMsgq p q # s) obj = ( |
1556 "\<lbrakk>valid (CreateMsgq p q # s); alive (CreateMsgq p q # s) obj\<rbrakk> \<Longrightarrow> co2sobj (CreateMsgq p q # s) obj = ( |
2207 case obj of |
1589 case obj of |
2208 O_msgq q' \<Rightarrow> if (q' = q) then (case (cq2smsgq (RecvMsg p q m # s) q) of |
1590 O_msgq q' \<Rightarrow> if (q' = q) then (case (cq2smsgq (RecvMsg p q m # s) q) of |
2209 Some sq \<Rightarrow> Some (S_msgq sq) |
1591 Some sq \<Rightarrow> Some (S_msgq sq) |
2210 | _ \<Rightarrow> None) |
1592 | _ \<Rightarrow> None) |
2211 else co2sobj s obj |
1593 else co2sobj s obj |
2212 | O_proc p' \<Rightarrow> if (info_flow_shm s p p' \<and> O_msg q m \<in> Tainted s) |
1594 | O_proc p' \<Rightarrow> if (p' = p \<and> O_msg q m \<in> tainted s) |
2213 then (case (cp2sproc s p') of |
1595 then (case (cp2sproc s p') of |
2214 Some sp \<Rightarrow> Some (S_proc sp True) |
1596 Some sp \<Rightarrow> Some (S_proc sp True) |
2215 | _ \<Rightarrow> None) |
1597 | _ \<Rightarrow> None) |
2216 else co2sobj s obj |
1598 else co2sobj s obj |
2217 | _ \<Rightarrow> co2sobj s obj)" |
1599 | _ \<Rightarrow> co2sobj s obj)" |
2218 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1600 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2219 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1601 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
2220 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
1602 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
2221 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
1603 simp:current_files_simps cf2sfile_simps cp2sproc_simps |
2222 same_inode_files_prop6 |
|
2223 dest!:current_has_smsgq' |
1604 dest!:current_has_smsgq' |
2224 dest:is_file_in_current is_dir_in_current cq2smsg_recvmsg) |
1605 dest:is_file_in_current is_dir_in_current cq2smsg_recvmsg) |
2225 done |
1606 done |
2226 |
1607 |
2227 lemma co2sobj_removemsgq: |
1608 lemma co2sobj_removemsgq: |
2228 "\<lbrakk>valid (RemoveMsgq p q # s); alive (RemoveMsgq p q # s) obj\<rbrakk> |
1609 "\<lbrakk>valid (RemoveMsgq p q # s); alive (RemoveMsgq p q # s) obj\<rbrakk> |
2229 \<Longrightarrow> co2sobj (RemoveMsgq p q # s) obj = co2sobj s obj" |
1610 \<Longrightarrow> co2sobj (RemoveMsgq p q # s) obj = co2sobj s obj" |
2230 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
1611 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
2231 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
1612 apply (simp_all add:current_files_simps is_dir_simps cq2smsgq_other) |
2232 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
1613 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
2233 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
1614 simp:current_files_simps cf2sfile_simps cp2sproc_simps |
2234 same_inode_files_prop6 |
|
2235 dest!:current_has_smsgq' |
1615 dest!:current_has_smsgq' |
2236 dest:is_file_in_current is_dir_in_current cq2smsg_removemsgq) |
1616 dest:is_file_in_current is_dir_in_current cq2smsg_removemsgq) |
2237 done |
1617 done |
2238 |
1618 |
2239 lemma co2sobj_createshm: |
|
2240 "\<lbrakk>valid (CreateShM p h # s); alive (CreateShM p h # s) obj\<rbrakk> \<Longrightarrow> co2sobj (CreateShM p h # s) obj = ( |
|
2241 case obj of |
|
2242 O_shm h' \<Rightarrow> if (h' = h) then (case (ch2sshm (CreateShM p h # s) h) of |
|
2243 Some sh \<Rightarrow> Some (S_shm sh) |
|
2244 | _ \<Rightarrow> None) |
|
2245 else co2sobj s obj |
|
2246 | _ \<Rightarrow> co2sobj s obj)" |
|
2247 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
|
2248 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
2249 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
|
2250 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
|
2251 same_inode_files_prop6 ch2sshm_simps |
|
2252 dest!:current_shm_has_sh' |
|
2253 dest:is_file_in_current is_dir_in_current) |
|
2254 done |
|
2255 |
|
2256 lemma co2sobj_detach: |
|
2257 "\<lbrakk>valid (Detach p h # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Detach p h # s) obj = ( |
|
2258 case obj of |
|
2259 O_proc p' \<Rightarrow> if (p' = p) then (case (cp2sproc (Detach p h # s) p) of |
|
2260 Some sp \<Rightarrow> Some (S_proc sp (O_proc p \<in> Tainted s)) |
|
2261 | _ \<Rightarrow> None) |
|
2262 else co2sobj s obj |
|
2263 | _ \<Rightarrow> co2sobj s obj)" |
|
2264 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
|
2265 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
2266 |
|
2267 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
|
2268 simp:current_files_simps cf2sfiles_simps cf2sfile_simps cp2sproc_simps tainted_eq_Tainted |
|
2269 same_inode_files_prop6 ch2sshm_simps |
|
2270 dest!:current_shm_has_sh' |
|
2271 dest:is_file_in_current is_dir_in_current) |
|
2272 done |
|
2273 |
|
2274 lemma co2sobj_deleteshm: |
|
2275 "\<lbrakk>valid (DeleteShM p h # s); alive (DeleteShM p h # s) obj\<rbrakk> \<Longrightarrow> co2sobj (DeleteShM p h # s) obj = ( |
|
2276 case obj of |
|
2277 O_proc p' \<Rightarrow> (case (cp2sproc (DeleteShM p h # s) p') of |
|
2278 Some sp \<Rightarrow> Some (S_proc sp (O_proc p' \<in> Tainted s)) |
|
2279 | _ \<Rightarrow> None) |
|
2280 | _ \<Rightarrow> co2sobj s obj)" |
|
2281 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
|
2282 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
2283 |
|
2284 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' current_proc_has_sp' |
|
2285 simp:current_files_simps cf2sfiles_simps cf2sfile_simps tainted_eq_Tainted |
|
2286 same_inode_files_prop6 ch2sshm_simps |
|
2287 dest!:current_shm_has_sh' |
|
2288 dest:is_file_in_current is_dir_in_current) |
|
2289 done |
|
2290 |
1619 |
2291 declare Product_Type.split_paired_Ex Product_Type.split_paired_All [simp del] |
1620 declare Product_Type.split_paired_Ex Product_Type.split_paired_All [simp del] |
2292 |
|
2293 lemma info_flow_shm_prop1: |
|
2294 "p \<in> current_procs s \<Longrightarrow> info_flow_shm s p p" |
|
2295 by (simp add:info_flow_shm_def) |
|
2296 |
|
2297 lemma co2sobj_attach: |
|
2298 "\<lbrakk>valid (Attach p h flag # s); alive s obj\<rbrakk> \<Longrightarrow> co2sobj (Attach p h flag # s) obj = ( |
|
2299 case obj of |
|
2300 O_proc p' \<Rightarrow> if (info_flow_shm s p p') |
|
2301 then (case (cp2sproc (Attach p h flag # s) p') of |
|
2302 Some sp \<Rightarrow> Some (S_proc sp (O_proc p' \<in> Tainted s \<or> |
|
2303 (\<exists> p''. O_proc p'' \<in> Tainted s \<and> (p'', SHM_RDWR) \<in> procs_of_shm s h))) |
|
2304 | _ \<Rightarrow> None) |
|
2305 else if (\<exists> p'' flag'. (p'', flag') \<in> procs_of_shm s h \<and> flag = SHM_RDWR \<and> O_proc p \<in> Tainted s \<and> |
|
2306 info_flow_shm s p'' p') |
|
2307 then (case (cp2sproc s p') of |
|
2308 Some sp \<Rightarrow> Some (S_proc sp True) |
|
2309 | _ \<Rightarrow> None) |
|
2310 else co2sobj s obj |
|
2311 | _ \<Rightarrow> co2sobj s obj)" |
|
2312 apply (frule vt_grant_os, frule vd_cons, case_tac obj) |
|
2313 apply (simp_all add:current_files_simps is_dir_simps ch2sshm_other cq2smsgq_other tainted_eq_Tainted) |
|
2314 |
|
2315 apply (rule conjI|rule impI|erule exE)+ |
|
2316 apply (simp split:option.splits del:split_paired_Ex) |
|
2317 apply (rule impI, frule current_proc_has_sp, simp) |
|
2318 apply ((erule exE)+, auto simp:tainted_eq_Tainted intro:info_flow_shm_Tainted)[1] |
|
2319 apply (rule impI, simp add:tainted_eq_Tainted split:option.splits del:split_paired_Ex) |
|
2320 apply (auto simp:info_flow_shm_prop1 cp2sproc_attach dest!:current_proc_has_sp')[1] |
|
2321 |
|
2322 apply (case_tac "cp2sproc (Attach p h flag # s) nat") |
|
2323 apply (drule current_proc_has_sp', simp+) |
|
2324 |
|
2325 apply (rule conjI|erule exE|erule conjE|rule impI)+ |
|
2326 apply (simp add:tainted_eq_Tainted) |
|
2327 apply (auto simp:info_flow_shm_prop1 cp2sproc_attach intro:info_flow_shm_Tainted dest!:current_proc_has_sp')[1] |
|
2328 apply (auto simp:info_flow_shm_prop1 cp2sproc_attach tainted_eq_Tainted intro:info_flow_shm_Tainted dest!:current_proc_has_sp' |
|
2329 split:option.splits if_splits)[1] |
|
2330 |
|
2331 |
|
2332 apply (auto split:if_splits option.splits dest!:current_file_has_sfile' |
|
2333 simp:current_files_simps cf2sfiles_simps cf2sfile_simps tainted_eq_Tainted |
|
2334 same_inode_files_prop6 |
|
2335 dest:is_file_in_current is_dir_in_current) |
|
2336 done |
|
2337 |
|
2338 |
1621 |
2339 lemma co2sobj_other: |
1622 lemma co2sobj_other: |
2340 "\<lbrakk>valid (e # s); alive (e # s) obj; |
1623 "\<lbrakk>valid (e # s); alive (e # s) obj; |
2341 \<forall> p f fds. e \<noteq> Execve p f fds; |
1624 \<forall> p f fds. e \<noteq> Execve p f fds; |
2342 \<forall> p p' fds shms. e \<noteq> Clone p p' fds shms; |
1625 \<forall> p p' fds. e \<noteq> Clone p p' fds; |
2343 \<forall> p p'. e \<noteq> Ptrace p p'; |
1626 \<forall> p p'. e \<noteq> Ptrace p p'; |
2344 \<forall> p f flags fd opt. e \<noteq> Open p f flags fd opt; |
1627 \<forall> p f flags fd opt. e \<noteq> Open p f flags fd opt; |
2345 \<forall> p fd. e \<noteq> ReadFile p fd; |
1628 \<forall> p fd. e \<noteq> ReadFile p fd; |
2346 \<forall> p fd. e \<noteq> WriteFile p fd; |
1629 \<forall> p fd. e \<noteq> WriteFile p fd; |
2347 \<forall> p fd. e \<noteq> CloseFd p fd; |
1630 \<forall> p fd. e \<noteq> CloseFd p fd; |
2348 \<forall> p f. e \<noteq> UnLink p f; |
1631 \<forall> p f. e \<noteq> UnLink p f; |
2349 \<forall> p f. e \<noteq> Rmdir p f; |
1632 \<forall> p f. e \<noteq> Rmdir p f; |
2350 \<forall> p f i. e \<noteq> Mkdir p f i; |
1633 \<forall> p f i. e \<noteq> Mkdir p f i; |
2351 \<forall> p f f'. e \<noteq> LinkHard p f f'; |
|
2352 \<forall> p f len. e \<noteq> Truncate p f len; |
1634 \<forall> p f len. e \<noteq> Truncate p f len; |
2353 \<forall> p q. e \<noteq> CreateMsgq p q; |
1635 \<forall> p q. e \<noteq> CreateMsgq p q; |
2354 \<forall> p q m. e \<noteq> SendMsg p q m; |
1636 \<forall> p q m. e \<noteq> SendMsg p q m; |
2355 \<forall> p q m. e \<noteq> RecvMsg p q m; |
1637 \<forall> p q m. e \<noteq> RecvMsg p q m; |
2356 \<forall> p q. e \<noteq> RemoveMsgq p q; |
1638 \<forall> p q. e \<noteq> RemoveMsgq p q\<rbrakk> |
2357 \<forall> p h. e \<noteq> CreateShM p h; |
1639 \<Longrightarrow> co2sobj (e # s) obj = co2sobj s obj" |
2358 \<forall> p h flag. e \<noteq> Attach p h flag; |
|
2359 \<forall> p h. e \<noteq> Detach p h; |
|
2360 \<forall> p h. e \<noteq> DeleteShM p h |
|
2361 \<rbrakk> \<Longrightarrow> co2sobj (e # s) obj = co2sobj s obj" |
|
2362 apply (frule vt_grant, case_tac e) |
1640 apply (frule vt_grant, case_tac e) |
2363 apply (auto intro:co2sobj_kill co2sobj_exit) |
1641 apply (auto intro:co2sobj_kill co2sobj_exit) |
2364 done |
1642 done |
2365 |
1643 |
2366 lemmas co2sobj_simps = co2sobj_execve co2sobj_clone co2sobj_ptrace co2sobj_open co2sobj_readfile |
1644 lemmas co2sobj_simps = co2sobj_execve co2sobj_clone co2sobj_ptrace co2sobj_open co2sobj_readfile |
2367 co2sobj_writefile co2sobj_closefd co2sobj_unlink co2sobj_rmdir co2sobj_mkdir co2sobj_linkhard |
1645 co2sobj_writefile co2sobj_closefd co2sobj_unlink co2sobj_rmdir co2sobj_mkdir |
2368 co2sobj_truncate co2sobj_kill co2sobj_exit co2sobj_createmsgq co2sobj_sendmsg co2sobj_recvmsg |
1646 co2sobj_truncate co2sobj_kill co2sobj_exit co2sobj_createmsgq co2sobj_sendmsg co2sobj_recvmsg |
2369 co2sobj_removemsgq co2sobj_attach co2sobj_detach co2sobj_createshm co2sobj_deleteshm |
1647 co2sobj_removemsgq |
2370 |
|
2371 |
|
2372 |
1648 |
2373 end |
1649 end |
2374 |
1650 |
2375 (*<*) |
1651 (*<*) |
2376 end |
1652 end |