| author | huffman | 
| Wed, 10 Nov 2010 13:08:42 -0800 | |
| changeset 40498 | 5718fb91d2d8 | 
| parent 40091 | 1ca61fbd8a79 | 
| child 40622 | e40e9e9769f4 | 
| permissions | -rw-r--r-- | 
| 40001 | 1 | (* Title: HOLCF/Fun_Cpo.thy | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 2 | Author: Franz Regensburger | 
| 40001 | 3 | Author: Brian Huffman | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 4 | *) | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 5 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 6 | header {* Class instances for the full function space *}
 | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 7 | |
| 40001 | 8 | theory Fun_Cpo | 
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 9 | imports Adm | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 10 | begin | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 11 | |
| 18291 | 12 | subsection {* Full function space is a partial order *}
 | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 13 | |
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 14 | instantiation "fun" :: (type, below) below | 
| 25758 | 15 | begin | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 16 | |
| 25758 | 17 | definition | 
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 18 | below_fun_def: "(op \<sqsubseteq>) \<equiv> (\<lambda>f g. \<forall>x. f x \<sqsubseteq> g x)" | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 19 | |
| 25758 | 20 | instance .. | 
| 21 | end | |
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 22 | |
| 25758 | 23 | instance "fun" :: (type, po) po | 
| 24 | proof | |
| 25 | fix f :: "'a \<Rightarrow> 'b" | |
| 26 | show "f \<sqsubseteq> f" | |
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 27 | by (simp add: below_fun_def) | 
| 25758 | 28 | next | 
| 29 | fix f g :: "'a \<Rightarrow> 'b" | |
| 30 | assume "f \<sqsubseteq> g" and "g \<sqsubseteq> f" thus "f = g" | |
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39199diff
changeset | 31 | by (simp add: below_fun_def fun_eq_iff below_antisym) | 
| 25758 | 32 | next | 
| 33 | fix f g h :: "'a \<Rightarrow> 'b" | |
| 34 | assume "f \<sqsubseteq> g" and "g \<sqsubseteq> h" thus "f \<sqsubseteq> h" | |
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 35 | unfolding below_fun_def by (fast elim: below_trans) | 
| 25758 | 36 | qed | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 37 | |
| 40002 
c5b5f7a3a3b1
new theorem names: fun_below_iff, fun_belowI, cfun_eq_iff, cfun_eqI, cfun_below_iff, cfun_belowI
 huffman parents: 
40001diff
changeset | 38 | lemma fun_below_iff: "f \<sqsubseteq> g \<longleftrightarrow> (\<forall>x. f x \<sqsubseteq> g x)" | 
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 39 | by (simp add: below_fun_def) | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 40 | |
| 40002 
c5b5f7a3a3b1
new theorem names: fun_below_iff, fun_belowI, cfun_eq_iff, cfun_eqI, cfun_below_iff, cfun_belowI
 huffman parents: 
40001diff
changeset | 41 | lemma fun_belowI: "(\<And>x. f x \<sqsubseteq> g x) \<Longrightarrow> f \<sqsubseteq> g" | 
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 42 | by (simp add: below_fun_def) | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 43 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 44 | lemma fun_belowD: "f \<sqsubseteq> g \<Longrightarrow> f x \<sqsubseteq> g x" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 45 | by (simp add: below_fun_def) | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 46 | |
| 18291 | 47 | subsection {* Full function space is chain complete *}
 | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 48 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 49 | text {* Function application is monotone. *}
 | 
| 25786 | 50 | |
| 51 | lemma monofun_app: "monofun (\<lambda>f. f x)" | |
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 52 | by (rule monofunI, simp add: below_fun_def) | 
| 25786 | 53 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 54 | text {* Properties of chains of functions. *}
 | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 55 | |
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 56 | lemma fun_chain_iff: "chain S \<longleftrightarrow> (\<forall>x. chain (\<lambda>i. S i x))" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 57 | unfolding chain_def fun_below_iff by auto | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 58 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 59 | lemma ch2ch_fun: "chain S \<Longrightarrow> chain (\<lambda>i. S i x)" | 
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 60 | by (simp add: chain_def below_fun_def) | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 61 | |
| 18092 
2c5d5da79a1e
renamed and added ch2ch, cont2cont, mono2mono theorems ending in _fun, _lambda, _LAM
 huffman parents: 
17831diff
changeset | 62 | lemma ch2ch_lambda: "(\<And>x. chain (\<lambda>i. S i x)) \<Longrightarrow> chain S" | 
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 63 | by (simp add: chain_def below_fun_def) | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 64 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 65 | text {* upper bounds of function chains yield upper bound in the po range *}
 | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 66 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 67 | lemma ub2ub_fun: | 
| 26028 | 68 | "range S <| u \<Longrightarrow> range (\<lambda>i. S i x) <| u x" | 
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 69 | by (auto simp add: is_ub_def below_fun_def) | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 70 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 71 | text {* Type @{typ "'a::type => 'b::cpo"} is chain complete *}
 | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 72 | |
| 26028 | 73 | lemma is_lub_lambda: | 
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 74 | "(\<And>x. range (\<lambda>i. Y i x) <<| f x) \<Longrightarrow> range Y <<| f" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 75 | unfolding is_lub_def is_ub_def below_fun_def by simp | 
| 26028 | 76 | |
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 77 | lemma lub_fun: | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 78 | "chain (S::nat \<Rightarrow> 'a::type \<Rightarrow> 'b::cpo) | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 79 | \<Longrightarrow> range S <<| (\<lambda>x. \<Squnion>i. S i x)" | 
| 26028 | 80 | apply (rule is_lub_lambda) | 
| 81 | apply (rule cpo_lubI) | |
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 82 | apply (erule ch2ch_fun) | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 83 | done | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 84 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 85 | lemma thelub_fun: | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 86 | "chain (S::nat \<Rightarrow> 'a::type \<Rightarrow> 'b::cpo) | 
| 27413 | 87 | \<Longrightarrow> (\<Squnion>i. S i) = (\<lambda>x. \<Squnion>i. S i x)" | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 88 | by (rule lub_fun [THEN thelubI]) | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 89 | |
| 20523 
36a59e5d0039
Major update to function package, including new syntax and the (only theoretical)
 krauss parents: 
18291diff
changeset | 90 | instance "fun" :: (type, cpo) cpo | 
| 40006 | 91 | by intro_classes (rule exI, erule lub_fun) | 
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 92 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 93 | subsection {* Chain-finiteness of function space *}
 | 
| 25827 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 94 | |
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 95 | lemma maxinch2maxinch_lambda: | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 96 | "(\<And>x. max_in_chain n (\<lambda>i. S i x)) \<Longrightarrow> max_in_chain n S" | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39199diff
changeset | 97 | unfolding max_in_chain_def fun_eq_iff by simp | 
| 25827 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 98 | |
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 99 | lemma maxinch_mono: | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 100 | "\<lbrakk>max_in_chain i Y; i \<le> j\<rbrakk> \<Longrightarrow> max_in_chain j Y" | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 101 | unfolding max_in_chain_def | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 102 | proof (intro allI impI) | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 103 | fix k | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 104 | assume Y: "\<forall>n\<ge>i. Y i = Y n" | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 105 | assume ij: "i \<le> j" | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 106 | assume jk: "j \<le> k" | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 107 | from ij jk have ik: "i \<le> k" by simp | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 108 | from Y ij have Yij: "Y i = Y j" by simp | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 109 | from Y ik have Yik: "Y i = Y k" by simp | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 110 | from Yij Yik show "Y j = Y k" by auto | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 111 | qed | 
| 
c2adeb1bae5c
new instance proofs for classes finite_po, chfin, flat
 huffman parents: 
25786diff
changeset | 112 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 113 | instance "fun" :: (type, discrete_cpo) discrete_cpo | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 114 | proof | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 115 | fix f g :: "'a \<Rightarrow> 'b" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 116 | show "f \<sqsubseteq> g \<longleftrightarrow> f = g" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 117 | unfolding fun_below_iff fun_eq_iff | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 118 | by simp | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 119 | qed | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 120 | |
| 18291 | 121 | subsection {* Full function space is pointed *}
 | 
| 17831 | 122 | |
| 123 | lemma minimal_fun: "(\<lambda>x. \<bottom>) \<sqsubseteq> f" | |
| 31076 
99fe356cbbc2
rename constant sq_le to below; rename class sq_ord to below; less->below in many lemma names
 huffman parents: 
29138diff
changeset | 124 | by (simp add: below_fun_def) | 
| 17831 | 125 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 126 | instance "fun" :: (type, pcpo) pcpo | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 127 | by default (fast intro: minimal_fun) | 
| 17831 | 128 | |
| 129 | lemma inst_fun_pcpo: "\<bottom> = (\<lambda>x. \<bottom>)" | |
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 130 | by (rule minimal_fun [THEN UU_I, symmetric]) | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 131 | |
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 132 | lemma app_strict [simp]: "\<bottom> x = \<bottom>" | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 133 | by (simp add: inst_fun_pcpo) | 
| 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 134 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 135 | lemma lambda_strict: "(\<lambda>x. \<bottom>) = \<bottom>" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 136 | by (rule UU_I, rule minimal_fun) | 
| 25786 | 137 | |
| 138 | subsection {* Propagation of monotonicity and continuity *}
 | |
| 139 | ||
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 140 | text {* The lub of a chain of monotone functions is monotone. *}
 | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 141 | |
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 142 | lemma adm_monofun: "adm monofun" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 143 | by (rule admI, simp add: thelub_fun fun_chain_iff monofun_def lub_mono) | 
| 25786 | 144 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 145 | text {* The lub of a chain of continuous functions is continuous. *}
 | 
| 25786 | 146 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 147 | lemma adm_cont: "adm cont" | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 148 | by (rule admI, simp add: thelub_fun fun_chain_iff) | 
| 25786 | 149 | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 150 | text {* Function application preserves monotonicity and continuity. *}
 | 
| 25786 | 151 | |
| 152 | lemma mono2mono_fun: "monofun f \<Longrightarrow> monofun (\<lambda>x. f x y)" | |
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 153 | by (simp add: monofun_def fun_below_iff) | 
| 25786 | 154 | |
| 155 | lemma cont2cont_fun: "cont f \<Longrightarrow> cont (\<lambda>x. f x y)" | |
| 35914 | 156 | apply (rule contI2) | 
| 25786 | 157 | apply (erule cont2mono [THEN mono2mono_fun]) | 
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 158 | apply (simp add: cont2contlubE thelub_fun ch2ch_cont) | 
| 25786 | 159 | done | 
| 160 | ||
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 161 | text {*
 | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 162 | Lambda abstraction preserves monotonicity and continuity. | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 163 |   (Note @{text "(\<lambda>x. \<lambda>y. f x y) = f"}.)
 | 
| 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 164 | *} | 
| 25786 | 165 | |
| 26452 
ed657432b8b9
declare cont_lemmas_ext as simp rules individually
 huffman parents: 
26028diff
changeset | 166 | lemma mono2mono_lambda: | 
| 
ed657432b8b9
declare cont_lemmas_ext as simp rules individually
 huffman parents: 
26028diff
changeset | 167 | assumes f: "\<And>y. monofun (\<lambda>x. f x y)" shows "monofun f" | 
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 168 | using f by (simp add: monofun_def fun_below_iff) | 
| 25786 | 169 | |
| 26452 
ed657432b8b9
declare cont_lemmas_ext as simp rules individually
 huffman parents: 
26028diff
changeset | 170 | lemma cont2cont_lambda [simp]: | 
| 
ed657432b8b9
declare cont_lemmas_ext as simp rules individually
 huffman parents: 
26028diff
changeset | 171 | assumes f: "\<And>y. cont (\<lambda>x. f x y)" shows "cont f" | 
| 40011 
b974cf829099
cleaned up Fun_Cpo.thy; deprecated a few theorem names
 huffman parents: 
40006diff
changeset | 172 | by (rule contI, rule is_lub_lambda, rule contE [OF f]) | 
| 25786 | 173 | |
| 174 | text {* What D.A.Schmidt calls continuity of abstraction; never used here *}
 | |
| 175 | ||
| 176 | lemma contlub_lambda: | |
| 177 | "(\<And>x::'a::type. chain (\<lambda>i. S i x::'b::cpo)) | |
| 178 | \<Longrightarrow> (\<lambda>x. \<Squnion>i. S i x) = (\<Squnion>i. (\<lambda>x. S i x))" | |
| 179 | by (simp add: thelub_fun ch2ch_lambda) | |
| 180 | ||
| 16202 
61811f31ce5a
renamed FunCpo theory to Ffun; added theorems ch2ch_fun_rev and app_strict
 huffman parents: diff
changeset | 181 | end |