| author | nipkow | 
| Fri, 17 Aug 2007 19:24:37 +0200 | |
| changeset 24308 | 700e745994c1 | 
| parent 23744 | 7c9e6e2fe249 | 
| child 25207 | d58c14280367 | 
| permissions | -rw-r--r-- | 
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 1 | (* ID: $Id$ | 
| 10213 | 2 | Author: Tobias Nipkow | 
| 3 | Copyright 1992 University of Cambridge | |
| 4 | *) | |
| 5 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 6 | header {*Well-founded Recursion*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 7 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 8 | theory Wellfounded_Recursion | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 9 | imports Transitive_Closure | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 10 | begin | 
| 10213 | 11 | |
| 23744 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 12 | inductive | 
| 22263 | 13 |   wfrec_rel :: "('a * 'a) set => (('a => 'b) => 'a => 'b) => 'a => 'b => bool"
 | 
| 14 |   for R :: "('a * 'a) set"
 | |
| 15 |   and F :: "('a => 'b) => 'a => 'b"
 | |
| 16 | where | |
| 17 | wfrecI: "ALL z. (z, x) : R --> wfrec_rel R F z (g z) ==> | |
| 18 | wfrec_rel R F x (F g x)" | |
| 11328 | 19 | |
| 10213 | 20 | constdefs | 
| 21 |   wf         :: "('a * 'a)set => bool"
 | |
| 22 | "wf(r) == (!P. (!x. (!y. (y,x):r --> P(y)) --> P(x)) --> (!x. P(x)))" | |
| 23 | ||
| 22263 | 24 |   wfP :: "('a => 'a => bool) => bool"
 | 
| 23744 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 25 |   "wfP r == wf {(x, y). r x y}"
 | 
| 22263 | 26 | |
| 10213 | 27 |   acyclic :: "('a*'a)set => bool"
 | 
| 28 | "acyclic r == !x. (x,x) ~: r^+" | |
| 29 | ||
| 30 |   cut        :: "('a => 'b) => ('a * 'a)set => 'a => 'a => 'b"
 | |
| 31 | "cut f r x == (%y. if (y,x):r then f y else arbitrary)" | |
| 32 | ||
| 11328 | 33 |   adm_wf :: "('a * 'a) set => (('a => 'b) => 'a => 'b) => bool"
 | 
| 34 | "adm_wf R F == ALL f g x. | |
| 35 | (ALL z. (z, x) : R --> f z = g z) --> F f x = F g x" | |
| 10213 | 36 | |
| 11328 | 37 |   wfrec :: "('a * 'a) set => (('a => 'b) => 'a => 'b) => 'a => 'b"
 | 
| 22845 | 38 | [code func del]: "wfrec R F == %x. THE y. wfrec_rel R (%f x. F (cut f R x) x) x y" | 
| 22263 | 39 | |
| 40 | abbreviation acyclicP :: "('a => 'a => bool) => bool" where
 | |
| 23744 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 41 |   "acyclicP r == acyclic {(x, y). r x y}"
 | 
| 10213 | 42 | |
| 22390 | 43 | class wellorder = linorder + | 
| 44 |   assumes wf: "wf {(x, y). x \<sqsubset> y}"
 | |
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 45 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 46 | |
| 23744 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 47 | lemma wfP_wf_eq [pred_set_conv]: "wfP (\<lambda>x y. (x, y) \<in> r) = wf r" | 
| 22263 | 48 | by (simp add: wfP_def) | 
| 49 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 50 | lemma wfUNIVI: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 51 | "(!!P x. (ALL x. (ALL y. (y,x) : r --> P(y)) --> P(x)) ==> P(x)) ==> wf(r)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 52 | by (unfold wf_def, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 53 | |
| 22263 | 54 | lemmas wfPUNIVI = wfUNIVI [to_pred] | 
| 55 | ||
| 19766 | 56 | text{*Restriction to domain @{term A} and range @{term B}.  If @{term r} is
 | 
| 57 |     well-founded over their intersection, then @{term "wf r"}*}
 | |
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 58 | lemma wfI: | 
| 19766 | 59 | "[| r \<subseteq> A <*> B; | 
| 60 | !!x P. [|\<forall>x. (\<forall>y. (y,x) : r --> P y) --> P x; x : A; x : B |] ==> P x |] | |
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 61 | ==> wf r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 62 | by (unfold wf_def, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 63 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 64 | lemma wf_induct: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 65 | "[| wf(r); | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 66 | !!x.[| ALL y. (y,x): r --> P(y) |] ==> P(x) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 67 | |] ==> P(a)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 68 | by (unfold wf_def, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 69 | |
| 22263 | 70 | lemmas wfP_induct = wf_induct [to_pred] | 
| 71 | ||
| 18458 | 72 | lemmas wf_induct_rule = wf_induct [rule_format, consumes 1, case_names less, induct set: wf] | 
| 17042 
da5cfaa258f7
moved wf_induct_rule from PreList.thy to Wellfounded_Recursion.thy
 nipkow parents: 
15950diff
changeset | 73 | |
| 22263 | 74 | lemmas wfP_induct_rule = | 
| 75 | wf_induct_rule [to_pred, consumes 1, case_names less, induct set: wfP] | |
| 76 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 77 | lemma wf_not_sym [rule_format]: "wf(r) ==> ALL x. (a,x):r --> (x,a)~:r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 78 | by (erule_tac a=a in wf_induct, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 79 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 80 | (* [| wf r; ~Z ==> (a,x) : r; (x,a) ~: r ==> Z |] ==> Z *) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 81 | lemmas wf_asym = wf_not_sym [elim_format] | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 82 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 83 | lemma wf_not_refl [simp]: "wf(r) ==> (a,a) ~: r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 84 | by (blast elim: wf_asym) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 85 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 86 | (* [| wf r; (a,a) ~: r ==> PROP W |] ==> PROP W *) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 87 | lemmas wf_irrefl = wf_not_refl [elim_format] | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 88 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 89 | text{*transitive closure of a well-founded relation is well-founded! *}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 90 | lemma wf_trancl: "wf(r) ==> wf(r^+)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 91 | apply (subst wf_def, clarify) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 92 | apply (rule allE, assumption) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 93 |   --{*Retains the universal formula for later use!*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 94 | apply (erule mp) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 95 | apply (erule_tac a = x in wf_induct) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 96 | apply (blast elim: tranclE) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 97 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 98 | |
| 22263 | 99 | lemmas wfP_trancl = wf_trancl [to_pred] | 
| 100 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 101 | lemma wf_converse_trancl: "wf (r^-1) ==> wf ((r^+)^-1)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 102 | apply (subst trancl_converse [symmetric]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 103 | apply (erule wf_trancl) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 104 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 105 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 106 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 107 | subsubsection{*Other simple well-foundedness results*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 108 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 109 | |
| 19870 | 110 | text{*Minimal-element characterization of well-foundedness*}
 | 
| 111 | lemma wf_eq_minimal: "wf r = (\<forall>Q x. x\<in>Q --> (\<exists>z\<in>Q. \<forall>y. (y,z)\<in>r --> y\<notin>Q))" | |
| 112 | proof (intro iffI strip) | |
| 113 | fix Q::"'a set" and x | |
| 114 | assume "wf r" and "x \<in> Q" | |
| 115 | thus "\<exists>z\<in>Q. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> Q" | |
| 116 | by (unfold wf_def, | |
| 117 | blast dest: spec [of _ "%x. x\<in>Q \<longrightarrow> (\<exists>z\<in>Q. \<forall>y. (y,z) \<in> r \<longrightarrow> y\<notin>Q)"]) | |
| 118 | next | |
| 22766 | 119 | assume 1: "\<forall>Q x. x \<in> Q \<longrightarrow> (\<exists>z\<in>Q. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> Q)" | 
| 120 | show "wf r" | |
| 121 | proof (rule wfUNIVI) | |
| 122 | fix P :: "'a \<Rightarrow> bool" and x | |
| 123 | assume 2: "\<forall>x. (\<forall>y. (y, x) \<in> r \<longrightarrow> P y) \<longrightarrow> P x" | |
| 124 |     let ?Q = "{x. \<not> P x}"
 | |
| 125 | have "x \<in> ?Q \<longrightarrow> (\<exists>z\<in>?Q. \<forall>y. (y, z) \<in> r \<longrightarrow> y \<notin> ?Q)" | |
| 126 | by (rule 1 [THEN spec, THEN spec]) | |
| 127 | hence "\<not> P x \<longrightarrow> (\<exists>z. \<not> P z \<and> (\<forall>y. (y, z) \<in> r \<longrightarrow> P y))" by simp | |
| 128 | with 2 have "\<not> P x \<longrightarrow> (\<exists>z. \<not> P z \<and> P z)" by fast | |
| 129 | thus "P x" by simp | |
| 130 | qed | |
| 19870 | 131 | qed | 
| 132 | ||
| 23186 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 133 | lemma wfE_min: | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 134 | assumes p:"wf R" "x \<in> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 135 | obtains z where "z \<in> Q" "\<And>y. (y, z) \<in> R \<Longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 136 | using p | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 137 | unfolding wf_eq_minimal | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 138 | by blast | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 139 | |
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 140 | lemma wfI_min: | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 141 | "(\<And>x Q. x \<in> Q \<Longrightarrow> \<exists>z\<in>Q. \<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> Q) | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 142 | \<Longrightarrow> wf R" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 143 | unfolding wf_eq_minimal | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 144 | by blast | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 145 | |
| 22263 | 146 | lemmas wfP_eq_minimal = wf_eq_minimal [to_pred] | 
| 147 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 148 | text{*Well-foundedness of subsets*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 149 | lemma wf_subset: "[| wf(r); p<=r |] ==> wf(p)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 150 | apply (simp (no_asm_use) add: wf_eq_minimal) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 151 | apply fast | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 152 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 153 | |
| 22263 | 154 | lemmas wfP_subset = wf_subset [to_pred] | 
| 155 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 156 | text{*Well-foundedness of the empty relation*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 157 | lemma wf_empty [iff]: "wf({})"
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 158 | by (simp add: wf_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 159 | |
| 23744 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 160 | lemmas wfP_empty [iff] = | 
| 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 161 | wf_empty [to_pred bot_empty_eq2, simplified bot_fun_eq bot_bool_eq] | 
| 22263 | 162 | |
| 19870 | 163 | lemma wf_Int1: "wf r ==> wf (r Int r')" | 
| 164 | by (erule wf_subset, rule Int_lower1) | |
| 165 | ||
| 166 | lemma wf_Int2: "wf r ==> wf (r' Int r)" | |
| 167 | by (erule wf_subset, rule Int_lower2) | |
| 168 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 169 | text{*Well-foundedness of insert*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 170 | lemma wf_insert [iff]: "wf(insert (y,x) r) = (wf(r) & (x,y) ~: r^*)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 171 | apply (rule iffI) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 172 | apply (blast elim: wf_trancl [THEN wf_irrefl] | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 173 | intro: rtrancl_into_trancl1 wf_subset | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 174 | rtrancl_mono [THEN [2] rev_subsetD]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 175 | apply (simp add: wf_eq_minimal, safe) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 176 | apply (rule allE, assumption, erule impE, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 177 | apply (erule bexE) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 178 | apply (rename_tac "a", case_tac "a = x") | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 179 | prefer 2 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 180 | apply blast | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 181 | apply (case_tac "y:Q") | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 182 | prefer 2 apply blast | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 183 | apply (rule_tac x = "{z. z:Q & (z,y) : r^*}" in allE)
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 184 | apply assumption | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 185 | apply (erule_tac V = "ALL Q. (EX x. x : Q) --> ?P Q" in thin_rl) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 186 |   --{*essential for speed*}
 | 
| 15343 | 187 | txt{*Blast with new substOccur fails*}
 | 
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 188 | apply (fast intro: converse_rtrancl_into_rtrancl) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 189 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 190 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 191 | text{*Well-foundedness of image*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 192 | lemma wf_prod_fun_image: "[| wf r; inj f |] ==> wf(prod_fun f f ` r)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 193 | apply (simp only: wf_eq_minimal, clarify) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 194 | apply (case_tac "EX p. f p : Q") | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 195 | apply (erule_tac x = "{p. f p : Q}" in allE)
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 196 | apply (fast dest: inj_onD, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 197 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 198 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 199 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 200 | subsubsection{*Well-Foundedness Results for Unions*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 201 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 202 | text{*Well-foundedness of indexed union with disjoint domains and ranges*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 203 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 204 | lemma wf_UN: "[| ALL i:I. wf(r i); | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 205 |          ALL i:I. ALL j:I. r i ~= r j --> Domain(r i) Int Range(r j) = {}  
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 206 | |] ==> wf(UN i:I. r i)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 207 | apply (simp only: wf_eq_minimal, clarify) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 208 | apply (rename_tac A a, case_tac "EX i:I. EX a:A. EX b:A. (b,a) : r i") | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 209 | prefer 2 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 210 | apply force | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 211 | apply clarify | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 212 | apply (drule bspec, assumption) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 213 | apply (erule_tac x="{a. a:A & (EX b:A. (b,a) : r i) }" in allE)
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 214 | apply (blast elim!: allE) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 215 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 216 | |
| 23744 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 217 | lemmas wfP_SUP = wf_UN [where I=UNIV and r="\<lambda>i. {(x, y). r i x y}",
 | 
| 
7c9e6e2fe249
Adapted to changes in infrastructure for converting between
 berghofe parents: 
23389diff
changeset | 218 | to_pred SUP_UN_eq2 bot_empty_eq, simplified, standard] | 
| 22263 | 219 | |
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 220 | lemma wf_Union: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 221 | "[| ALL r:R. wf r; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 222 |      ALL r:R. ALL s:R. r ~= s --> Domain r Int Range s = {}  
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 223 | |] ==> wf(Union R)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 224 | apply (simp add: Union_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 225 | apply (blast intro: wf_UN) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 226 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 227 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 228 | (*Intuition: we find an (R u S)-min element of a nonempty subset A | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 229 | by case distinction. | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 230 | 1. There is a step a -R-> b with a,b : A. | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 231 |      Pick an R-min element z of the (nonempty) set {a:A | EX b:A. a -R-> b}.
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 232 | By definition, there is z':A s.t. z -R-> z'. Because z is R-min in the | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 233 | subset, z' must be R-min in A. Because z' has an R-predecessor, it cannot | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 234 | have an S-successor and is thus S-min in A as well. | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 235 | 2. There is no such step. | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 236 | Pick an S-min element of A. In this case it must be an R-min | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 237 | element of A as well. | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 238 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 239 | *) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 240 | lemma wf_Un: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 241 |      "[| wf r; wf s; Domain r Int Range s = {} |] ==> wf(r Un s)"
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 242 | apply (simp only: wf_eq_minimal, clarify) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 243 | apply (rename_tac A a) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 244 | apply (case_tac "EX a:A. EX b:A. (b,a) : r") | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 245 | prefer 2 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 246 | apply simp | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 247 | apply (drule_tac x=A in spec)+ | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 248 | apply blast | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 249 | apply (erule_tac x="{a. a:A & (EX b:A. (b,a) : r) }" in allE)+
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 250 | apply (blast elim!: allE) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 251 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 252 | |
| 23186 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 253 | lemma wf_union_merge: | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 254 | "wf (R \<union> S) = wf (R O R \<union> R O S \<union> S)" (is "wf ?A = wf ?B") | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 255 | proof | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 256 | assume "wf ?A" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 257 | with wf_trancl have wfT: "wf (?A^+)" . | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 258 | moreover have "?B \<subseteq> ?A^+" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 259 | by (subst trancl_unfold, subst trancl_unfold) blast | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 260 | ultimately show "wf ?B" by (rule wf_subset) | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 261 | next | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 262 | assume "wf ?B" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 263 | |
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 264 | show "wf ?A" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 265 | proof (rule wfI_min) | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 266 | fix Q :: "'a set" and x | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 267 | assume "x \<in> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 268 | |
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 269 | with `wf ?B` | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 270 | obtain z where "z \<in> Q" and "\<And>y. (y, z) \<in> ?B \<Longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 271 | by (erule wfE_min) | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 272 | hence A1: "\<And>y. (y, z) \<in> R O R \<Longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 273 | and A2: "\<And>y. (y, z) \<in> R O S \<Longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 274 | and A3: "\<And>y. (y, z) \<in> S \<Longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 275 | by auto | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 276 | |
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 277 | show "\<exists>z\<in>Q. \<forall>y. (y, z) \<in> ?A \<longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 278 | proof (cases "\<forall>y. (y, z) \<in> R \<longrightarrow> y \<notin> Q") | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 279 | case True | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 280 | with `z \<in> Q` A3 show ?thesis by blast | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 281 | next | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 282 | case False | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 283 | then obtain z' where "z'\<in>Q" "(z', z) \<in> R" by blast | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 284 | |
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 285 | have "\<forall>y. (y, z') \<in> ?A \<longrightarrow> y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 286 | proof (intro allI impI) | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 287 | fix y assume "(y, z') \<in> ?A" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 288 | thus "y \<notin> Q" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 289 | proof | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 290 | assume "(y, z') \<in> R" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 291 | hence "(y, z) \<in> R O R" using `(z', z) \<in> R` .. | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 292 | with A1 show "y \<notin> Q" . | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 293 | next | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 294 | assume "(y, z') \<in> S" | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 295 | hence "(y, z) \<in> R O S" using `(z', z) \<in> R` .. | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 296 | with A2 show "y \<notin> Q" . | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 297 | qed | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 298 | qed | 
| 23389 | 299 | with `z' \<in> Q` show ?thesis .. | 
| 23186 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 300 | qed | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 301 | qed | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 302 | qed | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 303 | |
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 304 | lemma wf_comp_self: "wf R = wf (R O R)" (* special case *) | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 305 |   by (fact wf_union_merge[where S = "{}", simplified])
 | 
| 
f948708bc100
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
 krauss parents: 
22845diff
changeset | 306 | |
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 307 | subsubsection {*acyclic*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 308 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 309 | lemma acyclicI: "ALL x. (x, x) ~: r^+ ==> acyclic r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 310 | by (simp add: acyclic_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 311 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 312 | lemma wf_acyclic: "wf r ==> acyclic r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 313 | apply (simp add: acyclic_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 314 | apply (blast elim: wf_trancl [THEN wf_irrefl]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 315 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 316 | |
| 22263 | 317 | lemmas wfP_acyclicP = wf_acyclic [to_pred] | 
| 318 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 319 | lemma acyclic_insert [iff]: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 320 | "acyclic(insert (y,x) r) = (acyclic r & (x,y) ~: r^*)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 321 | apply (simp add: acyclic_def trancl_insert) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 322 | apply (blast intro: rtrancl_trans) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 323 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 324 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 325 | lemma acyclic_converse [iff]: "acyclic(r^-1) = acyclic r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 326 | by (simp add: acyclic_def trancl_converse) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 327 | |
| 22263 | 328 | lemmas acyclicP_converse [iff] = acyclic_converse [to_pred] | 
| 329 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 330 | lemma acyclic_impl_antisym_rtrancl: "acyclic r ==> antisym(r^*)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 331 | apply (simp add: acyclic_def antisym_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 332 | apply (blast elim: rtranclE intro: rtrancl_into_trancl1 rtrancl_trancl_trancl) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 333 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 334 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 335 | (* Other direction: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 336 | acyclic = no loops | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 337 | antisym = only self loops | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 338 | Goalw [acyclic_def,antisym_def] "antisym( r^* ) ==> acyclic(r - Id) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 339 | ==> antisym( r^* ) = acyclic(r - Id)"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 340 | *) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 341 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 342 | lemma acyclic_subset: "[| acyclic s; r <= s |] ==> acyclic r" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 343 | apply (simp add: acyclic_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 344 | apply (blast intro: trancl_mono) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 345 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 346 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 347 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 348 | subsection{*Well-Founded Recursion*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 349 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 350 | text{*cut*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 351 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 352 | lemma cuts_eq: "(cut f r x = cut g r x) = (ALL y. (y,x):r --> f(y)=g(y))" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 353 | by (simp add: expand_fun_eq cut_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 354 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 355 | lemma cut_apply: "(x,a):r ==> (cut f r a)(x) = f(x)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 356 | by (simp add: cut_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 357 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 358 | text{*Inductive characterization of wfrec combinator; for details see:  
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 359 | John Harrison, "Inductive definitions: automation and application"*} | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 360 | |
| 22263 | 361 | lemma wfrec_unique: "[| adm_wf R F; wf R |] ==> EX! y. wfrec_rel R F x y" | 
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 362 | apply (simp add: adm_wf_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 363 | apply (erule_tac a=x in wf_induct) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 364 | apply (rule ex1I) | 
| 22263 | 365 | apply (rule_tac g = "%x. THE y. wfrec_rel R F x y" in wfrec_rel.wfrecI) | 
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 366 | apply (fast dest!: theI') | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 367 | apply (erule wfrec_rel.cases, simp) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 368 | apply (erule allE, erule allE, erule allE, erule mp) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 369 | apply (fast intro: the_equality [symmetric]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 370 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 371 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 372 | lemma adm_lemma: "adm_wf R (%f x. F (cut f R x) x)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 373 | apply (simp add: adm_wf_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 374 | apply (intro strip) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 375 | apply (rule cuts_eq [THEN iffD2, THEN subst], assumption) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 376 | apply (rule refl) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 377 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 378 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 379 | lemma wfrec: "wf(r) ==> wfrec r H a = H (cut (wfrec r H) r a) a" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 380 | apply (simp add: wfrec_def) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 381 | apply (rule adm_lemma [THEN wfrec_unique, THEN the1_equality], assumption) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 382 | apply (rule wfrec_rel.wfrecI) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 383 | apply (intro strip) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 384 | apply (erule adm_lemma [THEN wfrec_unique, THEN theI']) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 385 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 386 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 387 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 388 | text{** This form avoids giant explosions in proofs.  NOTE USE OF ==*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 389 | lemma def_wfrec: "[| f==wfrec r H; wf(r) |] ==> f(a) = H (cut f r a) a" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 390 | apply auto | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 391 | apply (blast intro: wfrec) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 392 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 393 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 394 | |
| 17459 | 395 | subsection {* Code generator setup *}
 | 
| 396 | ||
| 397 | consts_code | |
| 17654 
38496187809d
Renamed wf_rec to wfrec in consts_code declaration.
 berghofe parents: 
17459diff
changeset | 398 |   "wfrec"   ("\<module>wfrec?")
 | 
| 17459 | 399 | attach {*
 | 
| 17654 
38496187809d
Renamed wf_rec to wfrec in consts_code declaration.
 berghofe parents: 
17459diff
changeset | 400 | fun wfrec f x = f (wfrec f) x; | 
| 17459 | 401 | *} | 
| 402 | ||
| 403 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 404 | subsection{*Variants for TFL: the Recdef Package*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 405 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 406 | lemma tfl_wf_induct: "ALL R. wf R --> | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 407 | (ALL P. (ALL x. (ALL y. (y,x):R --> P y) --> P x) --> (ALL x. P x))" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 408 | apply clarify | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 409 | apply (rule_tac r = R and P = P and a = x in wf_induct, assumption, blast) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 410 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 411 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 412 | lemma tfl_cut_apply: "ALL f R. (x,a):R --> (cut f R a)(x) = f(x)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 413 | apply clarify | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 414 | apply (rule cut_apply, assumption) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 415 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 416 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 417 | lemma tfl_wfrec: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 418 | "ALL M R f. (f=wfrec R M) --> wf R --> (ALL x. f x = M (cut f R x) x)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 419 | apply clarify | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 420 | apply (erule wfrec) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 421 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 422 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 423 | subsection {*LEAST and wellorderings*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 424 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 425 | text{* See also @{text wf_linord_ex_has_least} and its consequences in
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 426 |  @{text Wellfounded_Relations.ML}*}
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 427 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 428 | lemma wellorder_Least_lemma [rule_format]: | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 429 | "P (k::'a::wellorder) --> P (LEAST x. P(x)) & (LEAST x. P(x)) <= k" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 430 | apply (rule_tac a = k in wf [THEN wf_induct]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 431 | apply (rule impI) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 432 | apply (rule classical) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 433 | apply (rule_tac s = x in Least_equality [THEN ssubst], auto) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 434 | apply (auto simp add: linorder_not_less [symmetric]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 435 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 436 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 437 | lemmas LeastI = wellorder_Least_lemma [THEN conjunct1, standard] | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 438 | lemmas Least_le = wellorder_Least_lemma [THEN conjunct2, standard] | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 439 | |
| 15950 | 440 | -- "The following 3 lemmas are due to Brian Huffman" | 
| 441 | lemma LeastI_ex: "EX x::'a::wellorder. P x ==> P (Least P)" | |
| 442 | apply (erule exE) | |
| 443 | apply (erule LeastI) | |
| 444 | done | |
| 445 | ||
| 446 | lemma LeastI2: | |
| 447 | "[| P (a::'a::wellorder); !!x. P x ==> Q x |] ==> Q (Least P)" | |
| 448 | by (blast intro: LeastI) | |
| 449 | ||
| 450 | lemma LeastI2_ex: | |
| 451 | "[| EX a::'a::wellorder. P a; !!x. P x ==> Q x |] ==> Q (Least P)" | |
| 452 | by (blast intro: LeastI_ex) | |
| 453 | ||
| 15341 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 454 | lemma not_less_Least: "[| k < (LEAST x. P x) |] ==> ~P (k::'a::wellorder)" | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 455 | apply (simp (no_asm_use) add: linorder_not_le [symmetric]) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 456 | apply (erule contrapos_nn) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 457 | apply (erule Least_le) | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 458 | done | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 459 | |
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 460 | ML | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 461 | {*
 | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 462 | val wf_def = thm "wf_def"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 463 | val wfUNIVI = thm "wfUNIVI"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 464 | val wfI = thm "wfI"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 465 | val wf_induct = thm "wf_induct"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 466 | val wf_not_sym = thm "wf_not_sym"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 467 | val wf_asym = thm "wf_asym"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 468 | val wf_not_refl = thm "wf_not_refl"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 469 | val wf_irrefl = thm "wf_irrefl"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 470 | val wf_trancl = thm "wf_trancl"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 471 | val wf_converse_trancl = thm "wf_converse_trancl"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 472 | val wf_eq_minimal = thm "wf_eq_minimal"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 473 | val wf_subset = thm "wf_subset"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 474 | val wf_empty = thm "wf_empty"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 475 | val wf_insert = thm "wf_insert"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 476 | val wf_UN = thm "wf_UN"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 477 | val wf_Union = thm "wf_Union"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 478 | val wf_Un = thm "wf_Un"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 479 | val wf_prod_fun_image = thm "wf_prod_fun_image"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 480 | val acyclicI = thm "acyclicI"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 481 | val wf_acyclic = thm "wf_acyclic"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 482 | val acyclic_insert = thm "acyclic_insert"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 483 | val acyclic_converse = thm "acyclic_converse"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 484 | val acyclic_impl_antisym_rtrancl = thm "acyclic_impl_antisym_rtrancl"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 485 | val acyclic_subset = thm "acyclic_subset"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 486 | val cuts_eq = thm "cuts_eq"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 487 | val cut_apply = thm "cut_apply"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 488 | val wfrec_unique = thm "wfrec_unique"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 489 | val wfrec = thm "wfrec"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 490 | val def_wfrec = thm "def_wfrec"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 491 | val tfl_wf_induct = thm "tfl_wf_induct"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 492 | val tfl_cut_apply = thm "tfl_cut_apply"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 493 | val tfl_wfrec = thm "tfl_wfrec"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 494 | val LeastI = thm "LeastI"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 495 | val Least_le = thm "Least_le"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 496 | val not_less_Least = thm "not_less_Least"; | 
| 
254f6f00b60e
converted to Isar script, simplifying some results
 paulson parents: 
11451diff
changeset | 497 | *} | 
| 11137 | 498 | |
| 10213 | 499 | end |