| author | blanchet | 
| Tue, 18 Feb 2014 23:08:58 +0100 | |
| changeset 55570 | 853b82488fda | 
| parent 46911 | 6d2a2f0e904e | 
| child 57492 | 74bf65a1910a | 
| permissions | -rw-r--r-- | 
| 37936 | 1 | (* Title: HOL/UNITY/Comp/Priority.thy | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 2 | Author: Sidi O Ehmety, Cambridge University Computer Laboratory | 
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 3 | Copyright 2001 University of Cambridge | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 4 | *) | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 5 | |
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 6 | header{*The priority system*}
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 7 | |
| 16417 | 8 | theory Priority imports PriorityAux begin | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 9 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 10 | text{*From Charpentier and Chandy,
 | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 11 | Examples of Program Composition Illustrating the Use of Universal Properties | 
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 12 | In J. Rolim (editor), Parallel and Distributed Processing, | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 13 | Spriner LNCS 1586 (1999), pages 1215-1227.*} | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 14 | |
| 42463 | 15 | type_synonym state = "(vertex*vertex)set" | 
| 16 | type_synonym command = "vertex=>(state*state)set" | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 17 | |
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 18 | consts | 
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 19 | init :: "(vertex*vertex)set" | 
| 15274 | 20 |   --{* the initial state *}
 | 
| 21 | ||
| 22 | text{*Following the definitions given in section 4.4 *}
 | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 23 | |
| 36866 | 24 | definition highest :: "[vertex, (vertex*vertex)set]=>bool" | 
| 25 |   where "highest i r <-> A i r = {}"
 | |
| 15274 | 26 |     --{* i has highest priority in r *}
 | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 27 | |
| 36866 | 28 | definition lowest :: "[vertex, (vertex*vertex)set]=>bool" | 
| 29 |   where "lowest i r <-> R i r = {}"
 | |
| 15274 | 30 |     --{* i has lowest priority in r *}
 | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 31 | |
| 36866 | 32 | definition act :: command | 
| 33 |   where "act i = {(s, s'). s'=reverse i s & highest i s}"
 | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 34 | |
| 36866 | 35 | definition Component :: "vertex=>state program" | 
| 36 |   where "Component i = mk_total_program({init}, {act i}, UNIV)"
 | |
| 15274 | 37 |     --{* All components start with the same initial state *}
 | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 38 | |
| 15274 | 39 | |
| 40 | text{*Some Abbreviations *}
 | |
| 36866 | 41 | definition Highest :: "vertex=>state set" | 
| 42 |   where "Highest i = {s. highest i s}"
 | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 43 | |
| 36866 | 44 | definition Lowest :: "vertex=>state set" | 
| 45 |   where "Lowest i = {s. lowest i s}"
 | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 46 | |
| 36866 | 47 | definition Acyclic :: "state set" | 
| 48 |   where "Acyclic = {s. acyclic s}"
 | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 49 | |
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 50 | |
| 36866 | 51 | definition Maximal :: "state set" | 
| 15274 | 52 |     --{* Every ``above'' set has a maximal vertex*}
 | 
| 36866 | 53 |   where "Maximal = (\<Inter>i. {s. ~highest i s-->(\<exists>j \<in> above i  s. highest j s)})"
 | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 54 | |
| 36866 | 55 | definition Maximal' :: "state set" | 
| 15274 | 56 |     --{* Maximal vertex: equivalent definition*}
 | 
| 36866 | 57 |   where "Maximal' = (\<Inter>i. Highest i Un (\<Union>j. {s. j \<in> above i s} Int Highest j))"
 | 
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 58 | |
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 59 | |
| 36866 | 60 | definition Safety :: "state set" | 
| 61 |   where "Safety = (\<Inter>i. {s. highest i s --> (\<forall>j \<in> neighbors i s. ~highest j s)})"
 | |
| 11194 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 62 | |
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 63 | |
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 64 | (* Composition of a finite set of component; | 
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 65 | the vertex 'UNIV' is finite by assumption *) | 
| 
ea13ff5a26d1
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
 paulson parents: diff
changeset | 66 | |
| 36866 | 67 | definition system :: "state program" | 
| 68 | where "system = (JN i. Component i)" | |
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 69 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 70 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 71 | declare highest_def [simp] lowest_def [simp] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 72 | declare Highest_def [THEN def_set_simp, simp] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 73 | and Lowest_def [THEN def_set_simp, simp] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 74 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 75 | declare Component_def [THEN def_prg_Init, simp] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 76 | declare act_def [THEN def_act_simp, simp] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 77 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 78 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 79 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 80 | subsection{*Component correctness proofs*}
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 81 | |
| 15274 | 82 | text{* neighbors is stable  *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 83 | lemma Component_neighbors_stable: "Component i \<in> stable {s. neighbors k s = n}"
 | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 84 | by (simp add: Component_def, safety, auto) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 85 | |
| 15274 | 86 | text{* property 4 *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 87 | lemma Component_waits_priority: "Component i: {s. ((i,j):s) = b} Int (- Highest i) co {s. ((i,j):s)=b}"
 | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 88 | by (simp add: Component_def, safety) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 89 | |
| 15274 | 90 | text{* property 5: charpentier and Chandy mistakenly express it as
 | 
| 91 | 'transient Highest i'. Consider the case where i has neighbors *} | |
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 92 | lemma Component_yields_priority: | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 93 |  "Component i: {s. neighbors i s \<noteq> {}} Int Highest i  
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 94 | ensures - Highest i" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 95 | apply (simp add: Component_def) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 96 | apply (ensures_tac "act i", blast+) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 97 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 98 | |
| 15274 | 99 | text{* or better *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 100 | lemma Component_yields_priority': "Component i \<in> Highest i ensures Lowest i" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 101 | apply (simp add: Component_def) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 102 | apply (ensures_tac "act i", blast+) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 103 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 104 | |
| 15274 | 105 | text{* property 6: Component doesn't introduce cycle *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 106 | lemma Component_well_behaves: "Component i \<in> Highest i co Highest i Un Lowest i" | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 107 | by (simp add: Component_def, safety, fast) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 108 | |
| 15274 | 109 | text{* property 7: local axiom *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 110 | lemma locality: "Component i \<in> stable {s. \<forall>j k. j\<noteq>i & k\<noteq>i--> ((j,k):s) = b j k}"
 | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 111 | by (simp add: Component_def, safety) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 112 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 113 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 114 | subsection{*System  properties*}
 | 
| 15274 | 115 | text{* property 8: strictly universal *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 116 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 117 | lemma Safety: "system \<in> stable Safety" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 118 | apply (unfold Safety_def) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 119 | apply (rule stable_INT) | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 120 | apply (simp add: system_def, safety, fast) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 121 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 122 | |
| 15274 | 123 | text{* property 13: universal *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 124 | lemma p13: "system \<in> {s. s = q} co {s. s=q} Un {s. \<exists>i. derive i q s}"
 | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 125 | by (simp add: system_def Component_def mk_total_program_def totalize_JN, safety, blast) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 126 | |
| 15274 | 127 | text{* property 14: the 'above set' of a Component that hasn't got 
 | 
| 128 | priority doesn't increase *} | |
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 129 | lemma above_not_increase: | 
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 130 |      "system \<in> -Highest i Int {s. j\<notin>above i s} co {s. j\<notin>above i s}"
 | 
| 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 131 | apply (insert reach_lemma [of concl: j]) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 132 | apply (simp add: system_def Component_def mk_total_program_def totalize_JN, | 
| 16184 
80617b8d33c5
renamed "constrains" to "safety" to avoid keyword clash
 paulson parents: 
15274diff
changeset | 133 | safety) | 
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 134 | apply (simp add: trancl_converse, blast) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 135 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 136 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 137 | lemma above_not_increase': | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 138 |      "system \<in> -Highest i Int {s. above i s = x} co {s. above i s <= x}"
 | 
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 139 | apply (insert above_not_increase [of i]) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 140 | apply (simp add: trancl_converse constrains_def, blast) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 141 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 142 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 143 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 144 | |
| 15274 | 145 | text{* p15: universal property: all Components well behave  *}
 | 
| 46911 | 146 | lemma system_well_behaves: "system \<in> Highest i co Highest i Un Lowest i" | 
| 147 | by (simp add: system_def Component_def mk_total_program_def totalize_JN, safety, auto) | |
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 148 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 149 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 150 | lemma Acyclic_eq: "Acyclic = (\<Inter>i. {s. i\<notin>above i s})"
 | 
| 46911 | 151 | by (auto simp add: Acyclic_def acyclic_def trancl_converse) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 152 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 153 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 154 | lemmas system_co = | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 155 | constrains_Un [OF above_not_increase [rule_format] system_well_behaves] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 156 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 157 | lemma Acyclic_stable: "system \<in> stable Acyclic" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 158 | apply (simp add: stable_def Acyclic_eq) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 159 | apply (auto intro!: constrains_INT system_co [THEN constrains_weaken] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 160 | simp add: image0_r_iff_image0_trancl trancl_converse) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 161 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 162 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 163 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 164 | lemma Acyclic_subset_Maximal: "Acyclic <= Maximal" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 165 | apply (unfold Acyclic_def Maximal_def, clarify) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 166 | apply (drule above_lemma_b, auto) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 167 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 168 | |
| 15274 | 169 | text{* property 17: original one is an invariant *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 170 | lemma Acyclic_Maximal_stable: "system \<in> stable (Acyclic Int Maximal)" | 
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 171 | by (simp add: Acyclic_subset_Maximal [THEN Int_absorb2] Acyclic_stable) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 172 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 173 | |
| 15274 | 174 | text{* property 5: existential property *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 175 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 176 | lemma Highest_leadsTo_Lowest: "system \<in> Highest i leadsTo Lowest i" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 177 | apply (simp add: system_def Component_def mk_total_program_def totalize_JN) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 178 | apply (ensures_tac "act i", auto) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 179 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 180 | |
| 15274 | 181 | text{* a lowest i can never be in any abover set *} 
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 182 | lemma Lowest_above_subset: "Lowest i <= (\<Inter>k. {s. i\<notin>above k s})"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 183 | by (auto simp add: image0_r_iff_image0_trancl trancl_converse) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 184 | |
| 15274 | 185 | text{* property 18: a simpler proof than the original, one which uses psp *}
 | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 186 | lemma Highest_escapes_above: "system \<in> Highest i leadsTo (\<Inter>k. {s. i\<notin>above k s})"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 187 | apply (rule leadsTo_weaken_R) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 188 | apply (rule_tac [2] Lowest_above_subset) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 189 | apply (rule Highest_leadsTo_Lowest) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 190 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 191 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 192 | lemma Highest_escapes_above': | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 193 |      "system \<in> Highest j Int {s. j \<in> above i s} leadsTo {s. j\<notin>above i s}"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 194 | by (blast intro: leadsTo_weaken [OF Highest_escapes_above Int_lower1 INT_lower]) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 195 | |
| 15274 | 196 | subsection{*The main result: above set decreases*}
 | 
| 197 | ||
| 198 | text{* The original proof of the following formula was wrong *}
 | |
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 199 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 200 | lemma Highest_iff_above0: "Highest i = {s. above i s ={}}"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 201 | by (auto simp add: image0_trancl_iff_image0_r) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 202 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 203 | lemmas above_decreases_lemma = | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 204 | psp [THEN leadsTo_weaken, OF Highest_escapes_above' above_not_increase'] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 205 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 206 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 207 | lemma above_decreases: | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 208 |      "system \<in> (\<Union>j. {s. above i s = x} Int {s. j \<in> above i s} Int Highest j)  
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 209 |                leadsTo {s. above i s < x}"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 210 | apply (rule leadsTo_UN) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 211 | apply (rule single_leadsTo_I, clarify) | 
| 45600 
1bbbac9a0cb0
'lemmas' / 'theorems' commands allow 'for' fixes and standardize the result before storing;
 wenzelm parents: 
42463diff
changeset | 212 | apply (rule_tac x = "above i x" in above_decreases_lemma) | 
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 213 | apply (simp_all (no_asm_use) add: Highest_iff_above0) | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 214 | apply blast+ | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 215 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 216 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 217 | (** Just a massage of conditions to have the desired form ***) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 218 | lemma Maximal_eq_Maximal': "Maximal = Maximal'" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 219 | by (unfold Maximal_def Maximal'_def Highest_def, blast) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 220 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 221 | lemma Acyclic_subset: | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 222 |    "x\<noteq>{} ==>  
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 223 |     Acyclic Int {s. above i s = x} <=  
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 224 |     (\<Union>j. {s. above i s = x} Int {s. j \<in> above i s} Int Highest j)"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 225 | apply (rule_tac B = "Maximal' Int {s. above i s = x}" in subset_trans)
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 226 | apply (simp (no_asm) add: Maximal_eq_Maximal' [symmetric]) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 227 | apply (blast intro: Acyclic_subset_Maximal [THEN subsetD]) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 228 | apply (simp (no_asm) del: above_def add: Maximal'_def Highest_iff_above0) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 229 | apply blast | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 230 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 231 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 232 | lemmas above_decreases' = leadsTo_weaken_L [OF above_decreases Acyclic_subset] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 233 | lemmas above_decreases_psp = psp_stable [OF above_decreases' Acyclic_stable] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 234 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 235 | lemma above_decreases_psp': | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 236 | "x\<noteq>{}==> system \<in> Acyclic Int {s. above i s = x} leadsTo 
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 237 |                    Acyclic Int {s. above i s < x}"
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 238 | by (erule above_decreases_psp [THEN leadsTo_weaken], blast, auto) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 239 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 240 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 241 | lemmas finite_psubset_induct = wf_finite_psubset [THEN leadsTo_wf_induct] | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 242 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 243 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 244 | lemma Progress: "system \<in> Acyclic leadsTo Highest i" | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 245 | apply (rule_tac f = "%s. above i s" in finite_psubset_induct) | 
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 246 | apply (simp del: above_def | 
| 14087 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 247 | add: Highest_iff_above0 vimage_def finite_psubset_def, clarify) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 248 | apply (case_tac "m={}")
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 249 | apply (rule Int_lower2 [THEN [2] leadsTo_weaken_L]) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 250 | apply (force simp add: leadsTo_refl) | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 251 | apply (rule_tac A' = "Acyclic Int {x. above i x < m}" in leadsTo_weaken_R)
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 252 | apply (blast intro: above_decreases_psp')+ | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 253 | done | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 254 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 255 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 256 | text{*We have proved all (relevant) theorems given in the paper.  We didn't
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 257 | assume any thing about the relation @{term r}.  It is not necessary that
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 258 | @{term r} be a priority relation as assumed in the original proof.  It
 | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 259 | suffices that we start from a state which is finite and acyclic.*} | 
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 260 | |
| 
cb07c3948668
Conversion of UNITY/Comp/Priority.thy to a linear Isar script
 paulson parents: 
13812diff
changeset | 261 | |
| 14088 
61bd46feb919
converted Counter, Counterc and PriorityAux to Isar scripts (all HOL/UNITY/Comp)
 paulson parents: 
14087diff
changeset | 262 | end |