Finite_current.thy
author chunhan
Mon, 30 Dec 2013 12:01:09 +0800
changeset 84 cebdef333899
parent 72 526ba0410662
permissions -rw-r--r--
cfd2sfd, OF_create flag should not be in the sfd, cause all-duplicated sfd could not have this flag
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     1
theory Finite_current
72
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
     2
imports Main Valid_prop Flask Flask_type Proc_fd_of_file_prop
1
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     3
begin
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     4
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     5
context flask begin
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     6
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     7
lemma finite_cf: "valid \<tau> \<Longrightarrow> finite (current_files \<tau>)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     8
apply (induct \<tau>)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
     9
apply (simp add:current_files_def inum_of_file.simps)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    10
apply (rule_tac B = "init_files" in finite_subset)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    11
apply (clarsimp dest!:inof_has_file_tag, simp add:init_finite_sets)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    12
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    13
apply (frule vt_grant_os, frule vd_cons, simp, case_tac a)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    14
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    15
apply (auto simp:current_files_def os_grant.simps inum_of_file.simps split:if_splits option.splits)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    16
apply (rule_tac B = "insert list {f. \<exists>i. inum_of_file \<tau> f = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    17
apply (rule_tac B = "{f. \<exists>i. inum_of_file \<tau> f = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    18
apply (rule_tac B = "{f. \<exists>i. inum_of_file \<tau> f = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    19
apply (rule_tac B = "{f. \<exists>i. inum_of_file \<tau> f = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    20
apply (rule_tac B = "insert list {f. \<exists>i. inum_of_file \<tau> f = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    21
apply (rule_tac B = "insert list2 {f. \<exists>i. inum_of_file \<tau> f = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    22
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    23
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    24
lemma finite_cp: "finite (current_procs \<tau>)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    25
apply (induct \<tau>)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    26
apply (simp add:current_procs.simps init_finite_sets)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    27
apply (case_tac a, auto simp:current_procs.simps)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    28
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    29
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    30
lemma finite_cfd: "valid \<tau> \<Longrightarrow> finite (current_proc_fds \<tau> p)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    31
apply (induct \<tau> arbitrary:p)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    32
apply (simp add:current_proc_fds.simps init_finite_sets)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    33
apply (frule vd_cons, frule vt_grant_os, case_tac a, auto simp:current_proc_fds.simps)
72
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    34
apply (erule finite_subset)
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    35
apply (frule_tac s = \<tau> and p = nat in file_fds_subset_pfds)
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    36
apply (erule finite_subset, simp)
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    37
apply (erule finite_subset)
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    38
apply (frule_tac s = \<tau> and p = nat1 in file_fds_subset_pfds)
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    39
apply (erule finite_subset, simp)
526ba0410662 fixed bugs
chunhan
parents: 1
diff changeset
    40
done
1
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    41
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    42
lemma finite_pair: "\<lbrakk>finite A; finite B\<rbrakk> \<Longrightarrow> finite {(x, y). x \<in> A \<and> y \<in> B}"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    43
by auto
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    44
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    45
lemma finite_UN_I': "\<lbrakk>finite X; \<forall> x. x \<in> X \<longrightarrow> finite (f x)\<rbrakk> \<Longrightarrow> finite {(x, y). x \<in> X \<and> y \<in> f x}"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    46
apply (frule_tac B = f in finite_UN_I, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    47
apply (drule_tac finite_pair, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    48
apply (rule_tac B = "{(x, y). x \<in> X \<and> y \<in> (\<Union>a\<in>X. f a)}" in finite_subset, auto)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    49
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    50
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    51
lemma finite_init_netobjs: "finite init_sockets"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    52
apply (subgoal_tac "finite {(p, fd). p \<in> init_procs \<and> fd \<in> init_fds_of_proc p}")
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    53
apply (rule_tac B = "{(p, fd). p \<in> init_procs \<and> fd \<in> init_fds_of_proc p}" in finite_subset)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    54
apply (clarsimp dest!:init_socket_has_inode, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    55
using init_finite_sets finite_UN_I'
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    56
by (metis Collect_mem_eq SetCompr_Sigma_eq internal_split_def) 
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    57
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    58
lemma finite_cn_aux: "valid \<tau> \<Longrightarrow> finite {s. \<exists>i. inum_of_socket \<tau> s = Some i}"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    59
apply (induct \<tau>)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    60
apply (rule_tac B = "init_sockets" in finite_subset)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    61
apply (clarsimp simp:inum_of_socket.simps dest!:inos_has_sock_tag, simp add:finite_init_netobjs)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    62
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    63
apply (frule vd_cons, frule vt_grant_os, simp, case_tac a)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    64
apply (auto split:option.splits if_splits) 
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    65
apply (rule_tac B = "{s. \<exists>i. inum_of_socket \<tau> s = Some i}" in finite_subset, clarsimp split:if_splits, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    66
apply (rule_tac B = "{s. \<exists>i. inum_of_socket \<tau> s = Some i} \<union> {(p, fd). \<exists> i. inum_of_socket \<tau> (nat1, fd) = Some i \<and> p = nat2 \<and> fd \<in> set1}" in finite_subset, clarsimp split:if_splits)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    67
apply (simp only:finite_Un, rule conjI, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    68
apply (rule_tac B = "{(p, fd). \<exists> i. inum_of_socket \<tau> (nat1, fd) = Some i \<and> p = nat2}" in finite_subset, clarsimp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    69
apply (drule_tac h = "\<lambda> (p, fd). if (p = nat1) then (nat2, fd) else (p, fd)" in finite_imageI)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    70
apply (rule_tac B = "((\<lambda>(p, fd). if p = nat1 then (nat2, fd) else (p, fd)) ` {a. \<exists>i. inum_of_socket \<tau> a = Some i})" in finite_subset) 
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    71
apply (rule subsetI,erule CollectE, case_tac x, simp, (erule exE|erule conjE)+)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    72
unfolding image_def
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    73
apply (rule CollectI, rule_tac x = "(nat1, b)" in bexI, simp+)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    74
apply (rule_tac B = "{s. \<exists>i. inum_of_socket \<tau> s = Some i}" in finite_subset, clarsimp split:if_splits, simp)+
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    75
apply (rule_tac B = "insert (nat1, nat2) {s. \<exists>i. inum_of_socket \<tau> s = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    76
apply (rule_tac B = "insert (nat1, nat4) {s. \<exists>i. inum_of_socket \<tau> s = Some i}" in finite_subset, clarsimp, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    77
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    78
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    79
lemma finite_cn: "valid \<tau> \<Longrightarrow> finite (current_sockets \<tau>)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    80
apply (simp add:current_sockets_def inum_of_socket.simps)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    81
using finite_cn_aux[where \<tau> = \<tau>] by auto
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    82
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    83
lemma finite_ch: "finite (current_shms \<tau>)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    84
apply (induct \<tau>) defer
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    85
apply (case_tac a, auto simp:current_shms.simps init_finite_sets)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    86
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    87
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    88
lemma finite_cm: "finite (current_msgqs \<tau>)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    89
apply (induct \<tau>) defer
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    90
apply (case_tac a, auto simp: init_finite_sets)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    91
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    92
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    93
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    94
lemma finite_option: "finite {x. \<exists> y. f x = Some y} \<Longrightarrow> finite {y. \<exists> x. f x = Some y}"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    95
apply (drule_tac h = f in finite_imageI)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    96
apply (clarsimp simp only:image_def)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    97
apply (rule_tac f = Some in finite_imageD)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    98
apply (rule_tac B = "{y. \<exists>x. (\<exists>y. f x = Some y) \<and> y = f x}" in finite_subset)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
    99
unfolding image_def
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   100
apply auto
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   101
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   102
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   103
lemma finite_ci: "valid \<tau> \<Longrightarrow> finite (current_inode_nums \<tau>)"
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   104
apply (simp add:current_inode_nums_def current_file_inums_def current_sock_inums_def)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   105
apply (rule conjI, drule finite_cf, simp add:current_files_def, erule finite_option) 
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   106
using finite_cn[where \<tau> = \<tau>] 
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   107
apply (simp add:current_sockets_def, drule_tac finite_option, simp)
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   108
done
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   109
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   110
end
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   111
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   112
end
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   113
7d9c0ed02b56 thy files
chunhan
parents:
diff changeset
   114