| author | wenzelm |
| Mon, 06 Mar 2000 21:08:15 +0100 | |
| changeset 8348 | ebbbfdb35c84 |
| parent 8201 | a81d18b0a9b1 |
| child 8551 | 5c22595bc599 |
| permissions | -rw-r--r-- |
| 1461 | 1 |
(* Title: ZF/ex/Limit |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2 |
ID: $Id$ |
| 1461 | 3 |
Author: Sten Agerholm |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
4 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
5 |
The inverse limit construction. |
| 5136 | 6 |
|
7 |
(Proofs tidied up considerably by lcp) |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
8 |
*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
9 |
|
| 2469 | 10 |
val nat_linear_le = [nat_into_Ord,nat_into_Ord] MRS Ord_linear_le; |
11 |
||
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
12 |
(*----------------------------------------------------------------------*) |
| 1461 | 13 |
(* Useful goal commands. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
14 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
15 |
|
| 4152 | 16 |
val brr = fn thl => fn n => by (REPEAT(ares_tac thl n)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
17 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
18 |
(*----------------------------------------------------------------------*) |
| 1461 | 19 |
(* Basic results. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
20 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
21 |
|
| 5136 | 22 |
Goalw [set_def] "x:fst(D) ==> x:set(D)"; |
23 |
by (assume_tac 1); |
|
| 3425 | 24 |
qed "set_I"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
25 |
|
| 5136 | 26 |
Goalw [rel_def] "<x,y>:snd(D) ==> rel(D,x,y)"; |
27 |
by (assume_tac 1); |
|
| 3425 | 28 |
qed "rel_I"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
29 |
|
| 5136 | 30 |
Goalw [rel_def] "rel(D,x,y) ==> <x,y>:snd(D)"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
31 |
by (assume_tac 1); |
| 3425 | 32 |
qed "rel_E"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
33 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
34 |
(*----------------------------------------------------------------------*) |
| 1461 | 35 |
(* I/E/D rules for po and cpo. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
36 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
37 |
|
| 5136 | 38 |
Goalw [po_def] "[|po(D); x:set(D)|] ==> rel(D,x,x)"; |
39 |
by (Blast_tac 1); |
|
| 3425 | 40 |
qed "po_refl"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
41 |
|
| 5136 | 42 |
Goalw [po_def] "[|po(D); rel(D,x,y); rel(D,y,z); x:set(D); \ |
43 |
\ y:set(D); z:set(D)|] ==> rel(D,x,z)"; |
|
44 |
by (Blast_tac 1); |
|
| 3425 | 45 |
qed "po_trans"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
46 |
|
| 5136 | 47 |
Goalw [po_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
48 |
"[|po(D); rel(D,x,y); rel(D,y,x); x:set(D); y:set(D)|] ==> x = y"; |
| 5136 | 49 |
by (Blast_tac 1); |
| 3425 | 50 |
qed "po_antisym"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
51 |
|
| 5136 | 52 |
val prems = Goalw [po_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
53 |
"[| !!x. x:set(D) ==> rel(D,x,x); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
54 |
\ !!x y z. [| rel(D,x,y); rel(D,y,z); x:set(D); y:set(D); z:set(D)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
55 |
\ rel(D,x,z); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
56 |
\ !!x y. [| rel(D,x,y); rel(D,y,x); x:set(D); y:set(D)|] ==> x=y |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
57 |
\ po(D)"; |
| 4152 | 58 |
by Safe_tac; |
| 5136 | 59 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 60 |
qed "poI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
61 |
|
| 5136 | 62 |
val prems = Goalw [cpo_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
63 |
"[| po(D); !!X. chain(D,X) ==> islub(D,X,x(D,X))|] ==> cpo(D)"; |
| 4091 | 64 |
by (safe_tac (claset() addSIs [exI])); |
| 5136 | 65 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 66 |
qed "cpoI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
67 |
|
| 5136 | 68 |
Goalw [cpo_def] "cpo(D) ==> po(D)"; |
69 |
by (Blast_tac 1); |
|
| 3425 | 70 |
qed "cpo_po"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
71 |
|
| 5136 | 72 |
Goal "[|cpo(D); x:set(D)|] ==> rel(D,x,x)"; |
73 |
by (blast_tac (claset() addIs [po_refl, cpo_po]) 1); |
|
| 3425 | 74 |
qed "cpo_refl"; |
| 6158 | 75 |
|
| 3425 | 76 |
Addsimps [cpo_refl]; |
| 5136 | 77 |
AddSIs [cpo_refl]; |
| 6158 | 78 |
AddTCs [cpo_refl]; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
79 |
|
| 5136 | 80 |
Goal "[|cpo(D); rel(D,x,y); rel(D,y,z); x:set(D); \ |
81 |
\ y:set(D); z:set(D)|] ==> rel(D,x,z)"; |
|
82 |
by (blast_tac (claset() addIs [cpo_po, po_trans]) 1); |
|
| 3425 | 83 |
qed "cpo_trans"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
84 |
|
| 5136 | 85 |
Goal "[|cpo(D); rel(D,x,y); rel(D,y,x); x:set(D); y:set(D)|] ==> x = y"; |
86 |
by (blast_tac (claset() addIs [cpo_po, po_antisym]) 1); |
|
| 3425 | 87 |
qed "cpo_antisym"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
88 |
|
| 5136 | 89 |
val [cpo,chain,ex] = Goalw [cpo_def] |
| 2469 | 90 |
"[|cpo(D); chain(D,X); !!x. islub(D,X,x) ==> R|] ==> R"; |
| 1623 | 91 |
by (rtac (chain RS (cpo RS conjunct2 RS spec RS mp) RS exE) 1); |
| 5136 | 92 |
by (etac ex 1); |
| 3425 | 93 |
qed "cpo_islub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
94 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
95 |
(*----------------------------------------------------------------------*) |
| 1461 | 96 |
(* Theorems about isub and islub. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
97 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
98 |
|
| 5136 | 99 |
Goalw [islub_def] "islub(D,X,x) ==> isub(D,X,x)"; |
100 |
by (Asm_simp_tac 1); |
|
| 3425 | 101 |
qed "islub_isub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
102 |
|
| 5136 | 103 |
Goalw [islub_def,isub_def] "islub(D,X,x) ==> x:set(D)"; |
104 |
by (Asm_simp_tac 1); |
|
| 3425 | 105 |
qed "islub_in"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
106 |
|
| 5136 | 107 |
Goalw [islub_def,isub_def] "[|islub(D,X,x); n:nat|] ==> rel(D,X`n,x)"; |
108 |
by (Asm_simp_tac 1); |
|
| 3425 | 109 |
qed "islub_ub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
110 |
|
| 5136 | 111 |
Goalw [islub_def] "[|islub(D,X,x); isub(D,X,y)|] ==> rel(D,x,y)"; |
112 |
by (Blast_tac 1); |
|
| 3425 | 113 |
qed "islub_least"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
114 |
|
| 5136 | 115 |
val prems = Goalw [islub_def] (* islubI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
116 |
"[|isub(D,X,x); !!y. isub(D,X,y) ==> rel(D,x,y)|] ==> islub(D,X,x)"; |
| 4152 | 117 |
by Safe_tac; |
| 1623 | 118 |
by (REPEAT(ares_tac prems 1)); |
| 3425 | 119 |
qed "islubI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
120 |
|
| 5136 | 121 |
val prems = Goalw [isub_def] (* isubI *) |
| 2469 | 122 |
"[|x:set(D); !!n. n:nat ==> rel(D,X`n,x)|] ==> isub(D,X,x)"; |
| 4152 | 123 |
by Safe_tac; |
| 1623 | 124 |
by (REPEAT(ares_tac prems 1)); |
| 3425 | 125 |
qed "isubI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
126 |
|
| 5136 | 127 |
val prems = Goalw [isub_def] (* isubE *) |
128 |
"[|isub(D,X,x); [|x:set(D); !!n. n:nat==>rel(D,X`n,x)|] ==> P \ |
|
129 |
\ |] ==> P"; |
|
130 |
by (asm_simp_tac (simpset() addsimps prems) 1); |
|
| 3425 | 131 |
qed "isubE"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
132 |
|
| 5136 | 133 |
Goalw [isub_def] "isub(D,X,x) ==> x:set(D)"; |
134 |
by (Asm_simp_tac 1); |
|
| 3425 | 135 |
qed "isubD1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
136 |
|
| 5136 | 137 |
Goalw [isub_def] "[|isub(D,X,x); n:nat|]==>rel(D,X`n,x)"; |
138 |
by (Asm_simp_tac 1); |
|
| 3425 | 139 |
qed "isubD2"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
140 |
|
| 5136 | 141 |
Goal "[|islub(D,X,x); islub(D,X,y); cpo(D)|] ==> x = y"; |
142 |
by (blast_tac (claset() addIs [cpo_antisym,islub_least, |
|
143 |
islub_isub,islub_in]) 1); |
|
| 3425 | 144 |
qed "islub_unique"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
145 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
146 |
(*----------------------------------------------------------------------*) |
| 1461 | 147 |
(* lub gives the least upper bound of chains. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
148 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
149 |
|
| 5136 | 150 |
Goalw [lub_def] "[|chain(D,X); cpo(D)|] ==> islub(D,X,lub(D,X))"; |
151 |
by (best_tac (claset() addEs [cpo_islub] addIs [theI, islub_unique]) 1); |
|
| 3425 | 152 |
qed "cpo_lub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
153 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
154 |
(*----------------------------------------------------------------------*) |
| 1461 | 155 |
(* Theorems about chains. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
156 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
157 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
158 |
val chainI = prove_goalw Limit.thy [chain_def] |
| 2469 | 159 |
"!!z.[|X:nat->set(D); !!n. n:nat ==> rel(D,X`n,X`succ(n))|] ==> chain(D,X)" |
160 |
(fn prems => [Asm_simp_tac 1]); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
161 |
|
| 5136 | 162 |
Goalw [chain_def] "chain(D,X) ==> X : nat -> set(D)"; |
163 |
by (Asm_simp_tac 1); |
|
| 3425 | 164 |
qed "chain_fun"; |
| 5136 | 165 |
|
166 |
Goalw [chain_def] "[|chain(D,X); n:nat|] ==> X`n : set(D)"; |
|
167 |
by (blast_tac (claset() addDs [apply_type]) 1); |
|
| 3425 | 168 |
qed "chain_in"; |
| 5136 | 169 |
|
170 |
Goalw [chain_def] "[|chain(D,X); n:nat|] ==> rel(D, X ` n, X ` succ(n))"; |
|
171 |
by (Blast_tac 1); |
|
| 3425 | 172 |
qed "chain_rel"; |
| 5136 | 173 |
|
174 |
Addsimps [chain_in, chain_rel]; |
|
| 6169 | 175 |
AddTCs [chain_fun, chain_in, chain_rel]; |
| 5136 | 176 |
|
177 |
Goal "[|chain(D,X); cpo(D); n:nat; m:nat|] ==> rel(D,X`n,(X`(m #+ n)))"; |
|
| 6070 | 178 |
by (induct_tac "m" 1); |
| 2469 | 179 |
by (ALLGOALS Simp_tac); |
| 6158 | 180 |
by (rtac cpo_trans 1); |
181 |
by Auto_tac; |
|
| 3425 | 182 |
qed "chain_rel_gen_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
183 |
|
| 5136 | 184 |
Goal (* chain_rel_gen *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
185 |
"[|n le m; chain(D,X); cpo(D); n:nat; m:nat|] ==> rel(D,X`n,X`m)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
186 |
by (rtac impE 1); (* The first three steps prepare for the induction proof *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
187 |
by (assume_tac 3); |
| 5136 | 188 |
by (assume_tac 2); |
| 6070 | 189 |
by (induct_tac "m" 1); |
| 4152 | 190 |
by Safe_tac; |
| 5136 | 191 |
by (Asm_full_simp_tac 1); |
192 |
by (rtac cpo_trans 2); |
|
| 6158 | 193 |
by (auto_tac (claset(), |
194 |
simpset() addsimps [le_iff])); |
|
| 3425 | 195 |
qed "chain_rel_gen"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
196 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
197 |
(*----------------------------------------------------------------------*) |
| 1461 | 198 |
(* Theorems about pcpos and bottom. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
199 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
200 |
|
| 5136 | 201 |
val prems = Goalw [pcpo_def] (* pcpoI *) |
| 3840 | 202 |
"[|!!y. y:set(D)==>rel(D,x,y); x:set(D); cpo(D)|]==>pcpo(D)"; |
| 5136 | 203 |
by (auto_tac (claset() addIs prems, simpset())); |
| 3425 | 204 |
qed "pcpoI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
205 |
|
| 5136 | 206 |
Goalw [pcpo_def] "pcpo(D) ==> cpo(D)"; |
207 |
by (etac conjunct1 1); |
|
208 |
qed "pcpo_cpo"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
209 |
|
| 5136 | 210 |
Goalw [pcpo_def] (* pcpo_bot_ex1 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
211 |
"pcpo(D) ==> EX! x. x:set(D) & (ALL y:set(D). rel(D,x,y))"; |
| 5136 | 212 |
by (blast_tac (claset() addIs [cpo_antisym]) 1); |
| 3425 | 213 |
qed "pcpo_bot_ex1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
214 |
|
| 5136 | 215 |
Goalw [bot_def] (* bot_least *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
216 |
"[| pcpo(D); y:set(D)|] ==> rel(D,bot(D),y)"; |
| 5136 | 217 |
by (best_tac (claset() addIs [pcpo_bot_ex1 RS theI2]) 1); |
| 3425 | 218 |
qed "bot_least"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
219 |
|
| 5136 | 220 |
Goalw [bot_def] (* bot_in *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
221 |
"pcpo(D) ==> bot(D):set(D)"; |
| 5136 | 222 |
by (best_tac (claset() addIs [pcpo_bot_ex1 RS theI2]) 1); |
| 3425 | 223 |
qed "bot_in"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
224 |
|
| 6158 | 225 |
AddTCs [pcpo_cpo, bot_least, bot_in]; |
226 |
||
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
227 |
val prems = goal Limit.thy (* bot_unique *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
228 |
"[| pcpo(D); x:set(D); !!y. y:set(D) ==> rel(D,x,y)|] ==> x = bot(D)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
229 |
by (rtac cpo_antisym 1); |
| 1623 | 230 |
brr(pcpo_cpo::bot_in::bot_least::prems) 1; |
| 3425 | 231 |
qed "bot_unique"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
232 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
233 |
(*----------------------------------------------------------------------*) |
| 1461 | 234 |
(* Constant chains and lubs and cpos. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
235 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
236 |
|
| 5136 | 237 |
Goalw [chain_def] "[|x:set(D); cpo(D)|] ==> chain(D,(lam n:nat. x))"; |
238 |
by (asm_simp_tac (simpset() addsimps [lam_type, nat_succI]) 1); |
|
| 3425 | 239 |
qed "chain_const"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
240 |
|
| 5136 | 241 |
Goalw [islub_def,isub_def] |
242 |
"[|x:set(D); cpo(D)|] ==> islub(D,(lam n:nat. x),x)"; |
|
| 3425 | 243 |
by (Asm_simp_tac 1); |
244 |
by (Blast_tac 1); |
|
245 |
qed "islub_const"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
246 |
|
| 5136 | 247 |
Goal "[|x:set(D); cpo(D)|] ==> lub(D,lam n:nat. x) = x"; |
248 |
by (blast_tac (claset() addIs [islub_unique, cpo_lub, |
|
249 |
chain_const, islub_const]) 1); |
|
| 3425 | 250 |
qed "lub_const"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
251 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
252 |
(*----------------------------------------------------------------------*) |
| 1461 | 253 |
(* Taking the suffix of chains has no effect on ub's. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
254 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
255 |
|
| 5136 | 256 |
Goalw [isub_def,suffix_def] (* isub_suffix *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
257 |
"[|chain(D,X); cpo(D); n:nat|] ==> isub(D,suffix(X,n),x) <-> isub(D,X,x)"; |
| 5136 | 258 |
by (Asm_simp_tac 1); |
| 4152 | 259 |
by Safe_tac; |
| 5136 | 260 |
by (blast_tac (claset() addIs [chain_in, add_type]) 2); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
261 |
by (rtac cpo_trans 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
262 |
by (rtac chain_rel_gen_add 2); |
| 5136 | 263 |
by Auto_tac; |
| 3425 | 264 |
qed "isub_suffix"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
265 |
|
| 5136 | 266 |
Goalw [islub_def] (* islub_suffix *) |
267 |
"[|chain(D,X); cpo(D); n:nat|] ==> islub(D,suffix(X,n),x) <-> islub(D,X,x)"; |
|
268 |
by (asm_simp_tac (simpset() addsimps [isub_suffix]) 1); |
|
| 3425 | 269 |
qed "islub_suffix"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
270 |
|
| 5136 | 271 |
Goalw [lub_def] (* lub_suffix *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
272 |
"[|chain(D,X); cpo(D); n:nat|] ==> lub(D,suffix(X,n)) = lub(D,X)"; |
| 5136 | 273 |
by (asm_simp_tac (simpset() addsimps [islub_suffix]) 1); |
| 3425 | 274 |
qed "lub_suffix"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
275 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
276 |
(*----------------------------------------------------------------------*) |
| 1461 | 277 |
(* Dominate and subchain. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
278 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
279 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
280 |
val dominateI = prove_goalw Limit.thy [dominate_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
281 |
"[| !!m. m:nat ==> n(m):nat; !!m. m:nat ==> rel(D,X`m,Y`n(m))|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
282 |
\ dominate(D,X,Y)" |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
283 |
(fn prems => [rtac ballI 1,rtac bexI 1,REPEAT(ares_tac prems 1)]); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
284 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
285 |
val [dom,isub,cpo,X,Y] = goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
286 |
"[|dominate(D,X,Y); isub(D,Y,x); cpo(D); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
287 |
\ X:nat->set(D); Y:nat->set(D)|] ==> isub(D,X,x)"; |
| 1623 | 288 |
by (rewtac isub_def); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
289 |
by (rtac conjI 1); |
| 1623 | 290 |
by (rtac (rewrite_rule[isub_def]isub RS conjunct1) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
291 |
by (rtac ballI 1); |
| 1623 | 292 |
by (rtac (rewrite_rule[dominate_def]dom RS bspec RS bexE) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
293 |
by (assume_tac 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
294 |
by (rtac cpo_trans 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
295 |
by (rtac cpo 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
296 |
by (assume_tac 1); |
| 1623 | 297 |
by (rtac (rewrite_rule[isub_def]isub RS conjunct2 RS bspec) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
298 |
by (assume_tac 1); |
| 1623 | 299 |
by (etac (X RS apply_type) 1); |
300 |
by (etac (Y RS apply_type) 1); |
|
301 |
by (rtac (rewrite_rule[isub_def]isub RS conjunct1) 1); |
|
| 3425 | 302 |
qed "dominate_isub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
303 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
304 |
val [dom,Xlub,Ylub,cpo,X,Y] = goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
305 |
"[|dominate(D,X,Y); islub(D,X,x); islub(D,Y,y); cpo(D); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
306 |
\ X:nat->set(D); Y:nat->set(D)|] ==> rel(D,x,y)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
307 |
val Xub = rewrite_rule[islub_def]Xlub RS conjunct1; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
308 |
val Yub = rewrite_rule[islub_def]Ylub RS conjunct1; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
309 |
val Xub_y = Yub RS (dom RS dominate_isub); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
310 |
val lem = Xub_y RS (rewrite_rule[islub_def]Xlub RS conjunct2 RS spec RS mp); |
| 6046 | 311 |
by (rtac (Y RS (X RS (cpo RS lem))) 1); |
| 3425 | 312 |
qed "dominate_islub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
313 |
|
| 5136 | 314 |
val prems = Goalw [subchain_def] (* subchainE *) |
| 2469 | 315 |
"[|subchain(X,Y); n:nat; !!m. [|m:nat; X`n = Y`(n #+ m)|] ==> Q|] ==> Q"; |
| 1623 | 316 |
by (rtac (hd prems RS bspec RS bexE) 1); |
317 |
by (resolve_tac prems 2); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
318 |
by (assume_tac 3); |
| 1623 | 319 |
by (REPEAT(ares_tac prems 1)); |
| 3425 | 320 |
qed "subchainE"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
321 |
|
| 5136 | 322 |
Goal "[|subchain(Y,X); isub(D,X,x)|] ==> isub(D,Y,x)"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
323 |
by (rtac isubI 1); |
| 5136 | 324 |
by (safe_tac (claset() addSEs [isubE, subchainE])); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
325 |
by (assume_tac 1); |
| 2469 | 326 |
by (Asm_simp_tac 1); |
| 3425 | 327 |
qed "subchain_isub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
328 |
|
| 5268 | 329 |
Goal "[|dominate(D,X,Y); subchain(Y,X); islub(D,X,x); islub(D,Y,y); cpo(D); \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
330 |
\ X:nat->set(D); Y:nat->set(D)|] ==> x = y"; |
| 5136 | 331 |
by (blast_tac (claset() addIs [cpo_antisym, dominate_islub, islub_least, |
332 |
subchain_isub, islub_isub, islub_in]) 1); |
|
| 3425 | 333 |
qed "dominate_islub_eq"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
334 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
335 |
(*----------------------------------------------------------------------*) |
| 1461 | 336 |
(* Matrix. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
337 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
338 |
|
| 5136 | 339 |
Goalw [matrix_def] (* matrix_fun *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
340 |
"matrix(D,M) ==> M : nat -> (nat -> set(D))"; |
| 5136 | 341 |
by (Asm_simp_tac 1); |
| 3425 | 342 |
qed "matrix_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
343 |
|
| 5136 | 344 |
Goal "[|matrix(D,M); n:nat|] ==> M`n : nat -> set(D)"; |
345 |
by (blast_tac (claset() addIs [apply_funtype, matrix_fun]) 1); |
|
| 3425 | 346 |
qed "matrix_in_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
347 |
|
| 5136 | 348 |
Goal "[|matrix(D,M); n:nat; m:nat|] ==> M`n`m : set(D)"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
349 |
by (rtac apply_type 1); |
| 5136 | 350 |
by (REPEAT(ares_tac[matrix_in_fun] 1)); |
| 3425 | 351 |
qed "matrix_in"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
352 |
|
| 5136 | 353 |
Goalw [matrix_def] (* matrix_rel_1_0 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
354 |
"[|matrix(D,M); n:nat; m:nat|] ==> rel(D,M`n`m,M`succ(n)`m)"; |
| 5136 | 355 |
by (Asm_simp_tac 1); |
| 3425 | 356 |
qed "matrix_rel_1_0"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
357 |
|
| 5136 | 358 |
Goalw [matrix_def] (* matrix_rel_0_1 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
359 |
"[|matrix(D,M); n:nat; m:nat|] ==> rel(D,M`n`m,M`n`succ(m))"; |
| 5136 | 360 |
by (Asm_simp_tac 1); |
| 3425 | 361 |
qed "matrix_rel_0_1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
362 |
|
| 5136 | 363 |
Goalw [matrix_def] (* matrix_rel_1_1 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
364 |
"[|matrix(D,M); n:nat; m:nat|] ==> rel(D,M`n`m,M`succ(n)`succ(m))"; |
| 5136 | 365 |
by (Asm_simp_tac 1); |
| 3425 | 366 |
qed "matrix_rel_1_1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
367 |
|
| 5136 | 368 |
Goal "f:X->Y->Z ==> (lam y:Y. lam x:X. f`x`y):Y->X->Z"; |
369 |
by (blast_tac (claset() addIs [lam_type, apply_funtype]) 1); |
|
| 3425 | 370 |
qed "fun_swap"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
371 |
|
| 5136 | 372 |
Goalw [matrix_def] (* matrix_sym_axis *) |
373 |
"matrix(D,M) ==> matrix(D,lam m:nat. lam n:nat. M`n`m)"; |
|
374 |
by (asm_simp_tac (simpset() addsimps [fun_swap]) 1); |
|
| 3425 | 375 |
qed "matrix_sym_axis"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
376 |
|
| 5136 | 377 |
Goalw [chain_def] (* matrix_chain_diag *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
378 |
"matrix(D,M) ==> chain(D,lam n:nat. M`n`n)"; |
| 4152 | 379 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
380 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
381 |
by (rtac matrix_in 1); |
| 1623 | 382 |
by (REPEAT(ares_tac prems 1)); |
| 2469 | 383 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
384 |
by (rtac matrix_rel_1_1 1); |
| 1623 | 385 |
by (REPEAT(ares_tac prems 1)); |
| 3425 | 386 |
qed "matrix_chain_diag"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
387 |
|
| 5136 | 388 |
Goalw [chain_def] (* matrix_chain_left *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
389 |
"[|matrix(D,M); n:nat|] ==> chain(D,M`n)"; |
| 4152 | 390 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
391 |
by (rtac apply_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
392 |
by (rtac matrix_fun 1); |
| 1623 | 393 |
by (REPEAT(ares_tac prems 1)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
394 |
by (rtac matrix_rel_0_1 1); |
| 1623 | 395 |
by (REPEAT(ares_tac prems 1)); |
| 3425 | 396 |
qed "matrix_chain_left"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
397 |
|
| 5136 | 398 |
Goalw [chain_def] (* matrix_chain_right *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
399 |
"[|matrix(D,M); m:nat|] ==> chain(D,lam n:nat. M`n`m)"; |
| 5136 | 400 |
by (auto_tac (claset() addIs [lam_type,matrix_in,matrix_rel_1_0], |
401 |
simpset())); |
|
| 3425 | 402 |
qed "matrix_chain_right"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
403 |
|
| 6169 | 404 |
val xprem::yprem::prems = Goalw [matrix_def] (* matrix_chainI *) |
| 3840 | 405 |
"[|!!x. x:nat==>chain(D,M`x); !!y. y:nat==>chain(D,lam x:nat. M`x`y); \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
406 |
\ M:nat->nat->set(D); cpo(D)|] ==> matrix(D,M)"; |
| 6169 | 407 |
by Safe_tac; |
408 |
by (cut_inst_tac[("y1","m"),("n","n")] (yprem RS chain_rel) 2);
|
|
| 2469 | 409 |
by (Asm_full_simp_tac 4); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
410 |
by (rtac cpo_trans 5); |
| 6169 | 411 |
by (cut_inst_tac[("y1","m"),("n","n")] (yprem RS chain_rel) 6);
|
| 2469 | 412 |
by (Asm_full_simp_tac 8); |
| 6169 | 413 |
by (typecheck_tac (tcset() addTCs (chain_fun RS apply_type):: |
414 |
xprem::yprem::prems)); |
|
| 3425 | 415 |
qed "matrix_chainI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
416 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
417 |
val lemma = prove_goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
418 |
"!!z.[|m : nat; rel(D, (lam n:nat. M`n`n)`m, y)|] ==> rel(D,M`m`m, y)" |
| 2469 | 419 |
(fn prems => [Asm_full_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
420 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
421 |
val lemma2 = prove_goal Limit.thy |
| 3840 | 422 |
"!!z.[|x:nat; m:nat; rel(D,(lam n:nat. M`n`m1)`x,(lam n:nat. M`n`m1)`m)|] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
423 |
\ rel(D,M`x`m1,M`m`m1)" |
| 2469 | 424 |
(fn prems => [Asm_full_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
425 |
|
| 5136 | 426 |
Goalw [isub_def] (* isub_lemma *) |
427 |
"[|isub(D, lam n:nat. M`n`n, y); matrix(D,M); cpo(D)|] ==> \ |
|
428 |
\ isub(D, lam n:nat. lub(D,lam m:nat. M`n`m), y)"; |
|
| 4152 | 429 |
by Safe_tac; |
| 2469 | 430 |
by (Asm_simp_tac 1); |
| 5136 | 431 |
by (forward_tac [matrix_fun RS apply_type] 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
432 |
by (assume_tac 1); |
| 2469 | 433 |
by (Asm_simp_tac 1); |
| 5136 | 434 |
by (rtac (matrix_chain_left RS cpo_lub RS islub_least) 1); |
435 |
by (REPEAT (assume_tac 1)); |
|
| 1623 | 436 |
by (rewtac isub_def); |
| 4152 | 437 |
by Safe_tac; |
| 5136 | 438 |
by (excluded_middle_tac "n le na" 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
439 |
by (rtac cpo_trans 1); |
| 5136 | 440 |
by (assume_tac 1); |
| 1623 | 441 |
by (rtac (not_le_iff_lt RS iffD1 RS leI RS chain_rel_gen) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
442 |
by (assume_tac 3); |
| 5136 | 443 |
by (REPEAT(ares_tac [nat_into_Ord,matrix_chain_left] 1)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
444 |
by (rtac lemma 1); |
| 5136 | 445 |
by (assume_tac 1); |
446 |
by (Blast_tac 1); |
|
447 |
by (REPEAT(ares_tac [matrix_in] 1)); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
448 |
by (rtac cpo_trans 1); |
| 5136 | 449 |
by (assume_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
450 |
by (rtac lemma2 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
451 |
by (rtac lemma 4); |
| 5136 | 452 |
by (Blast_tac 5); |
453 |
by (REPEAT(ares_tac [chain_rel_gen,matrix_chain_right,matrix_in,isubD1] 1)); |
|
| 3425 | 454 |
qed "isub_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
455 |
|
| 5136 | 456 |
Goalw [chain_def] (* matrix_chain_lub *) |
| 3840 | 457 |
"[|matrix(D,M); cpo(D)|] ==> chain(D,lam n:nat. lub(D,lam m:nat. M`n`m))"; |
| 4152 | 458 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
459 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
460 |
by (rtac islub_in 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
461 |
by (rtac cpo_lub 1); |
| 5136 | 462 |
by (assume_tac 2); |
| 2469 | 463 |
by (Asm_simp_tac 2); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
464 |
by (rtac chainI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
465 |
by (rtac lam_type 1); |
| 5136 | 466 |
by (REPEAT(ares_tac [matrix_in] 1)); |
| 2469 | 467 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
468 |
by (rtac matrix_rel_0_1 1); |
| 5136 | 469 |
by (REPEAT(assume_tac 1)); |
| 4091 | 470 |
by (asm_simp_tac (simpset() addsimps |
| 5136 | 471 |
[matrix_chain_left RS chain_fun RS eta]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
472 |
by (rtac dominate_islub 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
473 |
by (rtac cpo_lub 3); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
474 |
by (rtac cpo_lub 2); |
| 1623 | 475 |
by (rewtac dominate_def); |
| 5136 | 476 |
by (REPEAT(ares_tac [matrix_chain_left,nat_succI,chain_fun] 2)); |
477 |
by (blast_tac (claset() addIs [matrix_rel_1_0]) 1); |
|
| 3425 | 478 |
qed "matrix_chain_lub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
479 |
|
| 5136 | 480 |
Goal (* isub_eq *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
481 |
"[|matrix(D,M); cpo(D)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
482 |
\ isub(D,(lam n:nat. lub(D,lam m:nat. M`n`m)),y) <-> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
483 |
\ isub(D,(lam n:nat. M`n`n),y)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
484 |
by (rtac iffI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
485 |
by (rtac dominate_isub 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
486 |
by (assume_tac 2); |
| 1623 | 487 |
by (rewtac dominate_def); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
488 |
by (rtac ballI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
489 |
by (rtac bexI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
490 |
by (assume_tac 2); |
| 2469 | 491 |
by (Asm_simp_tac 1); |
| 4091 | 492 |
by (asm_simp_tac (simpset() addsimps |
| 5136 | 493 |
[matrix_chain_left RS chain_fun RS eta]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
494 |
by (rtac islub_ub 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
495 |
by (rtac cpo_lub 1); |
| 1623 | 496 |
by (REPEAT(ares_tac |
| 5136 | 497 |
[matrix_chain_left,matrix_chain_diag,chain_fun,matrix_chain_lub] 1)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
498 |
by (rtac isub_lemma 1); |
| 5136 | 499 |
by (REPEAT(assume_tac 1)); |
| 3425 | 500 |
qed "isub_eq"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
501 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
502 |
val lemma1 = prove_goalw Limit.thy [lub_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
503 |
"lub(D,(lam n:nat. lub(D,lam m:nat. M`n`m))) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
504 |
\ (THE x. islub(D, (lam n:nat. lub(D,lam m:nat. M`n`m)), x))" |
| 5136 | 505 |
(fn _ => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
506 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
507 |
val lemma2 = prove_goalw Limit.thy [lub_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
508 |
"lub(D,(lam n:nat. M`n`n)) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
509 |
\ (THE x. islub(D, (lam n:nat. M`n`n), x))" |
| 5136 | 510 |
(fn _ => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
511 |
|
| 5136 | 512 |
Goal (* lub_matrix_diag *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
513 |
"[|matrix(D,M); cpo(D)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
514 |
\ lub(D,(lam n:nat. lub(D,lam m:nat. M`n`m))) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
515 |
\ lub(D,(lam n:nat. M`n`n))"; |
| 4091 | 516 |
by (simp_tac (simpset() addsimps [lemma1,lemma2]) 1); |
| 1623 | 517 |
by (rewtac islub_def); |
| 5136 | 518 |
by (asm_simp_tac (simpset() addsimps [isub_eq]) 1); |
| 3425 | 519 |
qed "lub_matrix_diag"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
520 |
|
| 5136 | 521 |
Goal (* lub_matrix_diag_sym *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
522 |
"[|matrix(D,M); cpo(D)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
523 |
\ lub(D,(lam m:nat. lub(D,lam n:nat. M`n`m))) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
524 |
\ lub(D,(lam n:nat. M`n`n))"; |
| 5136 | 525 |
by (dtac (matrix_sym_axis RS lub_matrix_diag) 1); |
526 |
by Auto_tac; |
|
| 3425 | 527 |
qed "lub_matrix_diag_sym"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
528 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
529 |
(*----------------------------------------------------------------------*) |
| 1461 | 530 |
(* I/E/D rules for mono and cont. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
531 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
532 |
|
| 5136 | 533 |
val prems = Goalw [mono_def] (* monoI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
534 |
"[|f:set(D)->set(E); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
535 |
\ !!x y. [|rel(D,x,y); x:set(D); y:set(D)|] ==> rel(E,f`x,f`y)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
536 |
\ f:mono(D,E)"; |
| 5136 | 537 |
by (blast_tac(claset() addSIs prems) 1); |
| 3425 | 538 |
qed "monoI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
539 |
|
| 5136 | 540 |
Goalw [mono_def] "f:mono(D,E) ==> f:set(D)->set(E)"; |
541 |
by (Fast_tac 1); |
|
| 3425 | 542 |
qed "mono_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
543 |
|
| 5136 | 544 |
Goal "[|f:mono(D,E); x:set(D)|] ==> f`x:set(E)"; |
545 |
by (blast_tac(claset() addSIs [mono_fun RS apply_type]) 1); |
|
| 3425 | 546 |
qed "mono_map"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
547 |
|
| 5136 | 548 |
Goalw [mono_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
549 |
"[|f:mono(D,E); rel(D,x,y); x:set(D); y:set(D)|] ==> rel(E,f`x,f`y)"; |
| 5136 | 550 |
by (Blast_tac 1); |
| 3425 | 551 |
qed "mono_mono"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
552 |
|
| 5136 | 553 |
val prems = Goalw [cont_def,mono_def] (* contI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
554 |
"[|f:set(D)->set(E); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
555 |
\ !!x y. [|rel(D,x,y); x:set(D); y:set(D)|] ==> rel(E,f`x,f`y); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
556 |
\ !!X. chain(D,X) ==> f`lub(D,X) = lub(E,lam n:nat. f`(X`n))|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
557 |
\ f:cont(D,E)"; |
| 4091 | 558 |
by (fast_tac(claset() addSIs prems) 1); |
| 3425 | 559 |
qed "contI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
560 |
|
| 5136 | 561 |
Goalw [cont_def] "f:cont(D,E) ==> f:mono(D,E)"; |
562 |
by (Blast_tac 1); |
|
| 3425 | 563 |
qed "cont2mono"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
564 |
|
| 6169 | 565 |
Goalw [cont_def] "f:cont(D,E) ==> f:set(D)->set(E)"; |
| 5136 | 566 |
by (rtac mono_fun 1); |
567 |
by (Blast_tac 1); |
|
| 3425 | 568 |
qed "cont_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
569 |
|
| 5136 | 570 |
Goal "[|f:cont(D,E); x:set(D)|] ==> f`x:set(E)"; |
571 |
by (blast_tac(claset() addSIs [cont_fun RS apply_type]) 1); |
|
| 3425 | 572 |
qed "cont_map"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
573 |
|
| 6169 | 574 |
AddTCs [comp_fun, cont_fun, cont_map]; |
575 |
||
| 5136 | 576 |
Goalw [cont_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
577 |
"[|f:cont(D,E); rel(D,x,y); x:set(D); y:set(D)|] ==> rel(E,f`x,f`y)"; |
| 5136 | 578 |
by (blast_tac(claset() addSIs [mono_mono]) 1); |
| 3425 | 579 |
qed "cont_mono"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
580 |
|
| 5136 | 581 |
Goalw [cont_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
582 |
"[|f:cont(D,E); chain(D,X)|] ==> f`(lub(D,X)) = lub(E,lam n:nat. f`(X`n))"; |
| 5136 | 583 |
by (Blast_tac 1); |
| 3425 | 584 |
qed "cont_lub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
585 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
586 |
(*----------------------------------------------------------------------*) |
| 1461 | 587 |
(* Continuity and chains. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
588 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
589 |
|
| 5136 | 590 |
Goal "[|f:mono(D,E); chain(D,X)|] ==> chain(E,lam n:nat. f`(X`n))"; |
591 |
by (simp_tac (simpset() addsimps [chain_def]) 1); |
|
592 |
by (blast_tac(claset() addIs [lam_type, mono_map, chain_in, |
|
593 |
mono_mono, chain_rel]) 1); |
|
| 3425 | 594 |
qed "mono_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
595 |
|
| 5136 | 596 |
Goal "[|f:cont(D,E); chain(D,X)|] ==> chain(E,lam n:nat. f`(X`n))"; |
597 |
by (blast_tac(claset() addIs [mono_chain, cont2mono]) 1); |
|
| 3425 | 598 |
qed "cont_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
599 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
600 |
(*----------------------------------------------------------------------*) |
| 1461 | 601 |
(* I/E/D rules about (set+rel) cf, the continuous function space. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
602 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
603 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
604 |
(* The following development more difficult with cpo-as-relation approach. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
605 |
|
| 5136 | 606 |
Goalw [set_def,cf_def] "f:set(cf(D,E)) ==> f:cont(D,E)"; |
| 2469 | 607 |
by (Asm_full_simp_tac 1); |
| 3425 | 608 |
qed "cf_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
609 |
|
| 5136 | 610 |
Goalw [set_def,cf_def] (* Non-trivial with relation *) |
611 |
"f:cont(D,E) ==> f:set(cf(D,E))"; |
|
| 2469 | 612 |
by (Asm_full_simp_tac 1); |
| 3425 | 613 |
qed "cont_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
614 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
615 |
(* rel_cf originally an equality. Now stated as two rules. Seemed easiest. |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
616 |
Besides, now complicated by typing assumptions. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
617 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
618 |
val prems = goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
619 |
"[|!!x. x:set(D) ==> rel(E,f`x,g`x); f:cont(D,E); g:cont(D,E)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
620 |
\ rel(cf(D,E),f,g)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
621 |
by (rtac rel_I 1); |
| 4091 | 622 |
by (simp_tac (simpset() addsimps [cf_def]) 1); |
| 4152 | 623 |
by Safe_tac; |
| 5136 | 624 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 625 |
qed "rel_cfI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
626 |
|
| 5136 | 627 |
Goalw [rel_def,cf_def] "[|rel(cf(D,E),f,g); x:set(D)|] ==> rel(E,f`x,g`x)"; |
| 2469 | 628 |
by (Asm_full_simp_tac 1); |
| 3425 | 629 |
qed "rel_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
630 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
631 |
(*----------------------------------------------------------------------*) |
| 1461 | 632 |
(* Theorems about the continuous function space. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
633 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
634 |
|
| 5136 | 635 |
Goal (* chain_cf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
636 |
"[| chain(cf(D,E),X); x:set(D)|] ==> chain(E,lam n:nat. X`n`x)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
637 |
by (rtac chainI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
638 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
639 |
by (rtac apply_type 1); |
| 5136 | 640 |
by (assume_tac 2); |
641 |
by (REPEAT(ares_tac[cont_fun,cf_cont,chain_in] 1)); |
|
| 2469 | 642 |
by (Asm_simp_tac 1); |
| 5136 | 643 |
by (REPEAT(ares_tac[rel_cf,chain_rel] 1)); |
| 3425 | 644 |
qed "chain_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
645 |
|
| 5136 | 646 |
Goal (* matrix_lemma *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
647 |
"[|chain(cf(D,E),X); chain(D,Xa); cpo(D); cpo(E) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
648 |
\ matrix(E,lam x:nat. lam xa:nat. X`x`(Xa`xa))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
649 |
by (rtac matrix_chainI 1); |
| 2469 | 650 |
by (Asm_simp_tac 1); |
651 |
by (Asm_simp_tac 2); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
652 |
by (rtac chainI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
653 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
654 |
by (rtac apply_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
655 |
by (rtac (chain_in RS cf_cont RS cont_fun) 1); |
| 5136 | 656 |
by (REPEAT(assume_tac 1)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
657 |
by (rtac chain_in 1); |
| 5136 | 658 |
by (REPEAT(assume_tac 1)); |
| 2469 | 659 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
660 |
by (rtac cont_mono 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
661 |
by (rtac (chain_in RS cf_cont) 1); |
| 5136 | 662 |
by (REPEAT (assume_tac 1)); |
663 |
brr [chain_rel,chain_in,nat_succI] 1; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
664 |
by (rtac chainI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
665 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
666 |
by (rtac apply_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
667 |
by (rtac (chain_in RS cf_cont RS cont_fun) 1); |
| 5136 | 668 |
by (REPEAT(assume_tac 1)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
669 |
by (rtac chain_in 1); |
| 5136 | 670 |
by (REPEAT(assume_tac 1)); |
| 2469 | 671 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
672 |
by (rtac rel_cf 1); |
| 5136 | 673 |
brr [chain_in,chain_rel] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
674 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
675 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
676 |
by (rtac apply_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
677 |
by (rtac (chain_in RS cf_cont RS cont_fun) 1); |
| 6169 | 678 |
by Auto_tac; |
| 3425 | 679 |
qed "matrix_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
680 |
|
| 5136 | 681 |
Goal (* chain_cf_lub_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
682 |
"[|chain(cf(D,E),X); cpo(D); cpo(E) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
683 |
\ (lam x:set(D). lub(E, lam n:nat. X ` n ` x)) : cont(D, E)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
684 |
by (rtac contI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
685 |
by (rtac lam_type 1); |
| 5136 | 686 |
by (REPEAT(ares_tac[chain_cf RS cpo_lub RS islub_in] 1)); |
| 2469 | 687 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
688 |
by (rtac dominate_islub 1); |
| 5136 | 689 |
by (REPEAT(ares_tac[chain_cf RS cpo_lub] 2)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
690 |
by (rtac dominateI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
691 |
by (assume_tac 1); |
| 2469 | 692 |
by (Asm_simp_tac 1); |
| 5136 | 693 |
by (REPEAT(ares_tac [chain_in RS cf_cont RS cont_mono] 1)); |
694 |
by (REPEAT(ares_tac [chain_cf RS chain_fun] 1)); |
|
| 2034 | 695 |
by (stac beta 1); |
| 5136 | 696 |
by (REPEAT(ares_tac [cpo_lub RS islub_in] 1)); |
697 |
by (asm_simp_tac(simpset() addsimps[chain_in RS cf_cont RS cont_lub]) 1); |
|
698 |
by (forward_tac[matrix_lemma RS lub_matrix_diag]1); |
|
699 |
by (REPEAT (assume_tac 1)); |
|
| 2469 | 700 |
by (Asm_full_simp_tac 1); |
| 4091 | 701 |
by (asm_simp_tac(simpset() addsimps[chain_in RS beta]) 1); |
| 5136 | 702 |
by (dtac (matrix_lemma RS lub_matrix_diag_sym) 1); |
| 6169 | 703 |
by Auto_tac; |
| 3425 | 704 |
qed "chain_cf_lub_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
705 |
|
| 5136 | 706 |
Goal (* islub_cf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
707 |
"[| chain(cf(D,E),X); cpo(D); cpo(E)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
708 |
\ islub(cf(D,E), X, lam x:set(D). lub(E,lam n:nat. X`n`x))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
709 |
by (rtac islubI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
710 |
by (rtac isubI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
711 |
by (rtac (chain_cf_lub_cont RS cont_cf) 1); |
| 5136 | 712 |
by (REPEAT (assume_tac 1)); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
713 |
by (rtac rel_cfI 1); |
| 5136 | 714 |
by (fast_tac (claset() addSDs [chain_cf RS cpo_lub RS islub_ub] |
715 |
addss simpset()) 1); |
|
716 |
by (blast_tac (claset() addIs [cf_cont,chain_in]) 1); |
|
717 |
by (blast_tac (claset() addIs [cont_cf,chain_cf_lub_cont]) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
718 |
by (rtac rel_cfI 1); |
| 2469 | 719 |
by (Asm_simp_tac 1); |
| 5136 | 720 |
by (REPEAT (blast_tac (claset() addIs [chain_cf_lub_cont,isubD1,cf_cont]) 2)); |
721 |
by (best_tac (claset() addIs [chain_cf RS cpo_lub RS islub_least, |
|
722 |
cf_cont RS cont_fun RS apply_type, isubI] |
|
723 |
addEs [isubD2 RS rel_cf, isubD1] |
|
724 |
addss simpset()) 1); |
|
| 3425 | 725 |
qed "islub_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
726 |
|
| 5136 | 727 |
Goal (* cpo_cf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
728 |
"[| cpo(D); cpo(E)|] ==> cpo(cf(D,E))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
729 |
by (rtac (poI RS cpoI) 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
730 |
by (rtac rel_cfI 1); |
| 5136 | 731 |
brr[cpo_refl, cf_cont RS cont_fun RS apply_type, cf_cont] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
732 |
by (rtac rel_cfI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
733 |
by (rtac cpo_trans 1); |
| 5136 | 734 |
by (assume_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
735 |
by (etac rel_cf 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
736 |
by (assume_tac 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
737 |
by (rtac rel_cf 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
738 |
by (assume_tac 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
739 |
brr[cf_cont RS cont_fun RS apply_type,cf_cont]1; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
740 |
by (rtac fun_extension 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
741 |
brr[cf_cont RS cont_fun]1; |
| 5136 | 742 |
by (fast_tac (claset() addIs [islub_cf]) 2); |
743 |
by (blast_tac (claset() addIs [cpo_antisym,rel_cf, |
|
744 |
cf_cont RS cont_fun RS apply_type]) 1); |
|
745 |
||
| 3425 | 746 |
qed "cpo_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
747 |
|
| 6158 | 748 |
AddTCs [cpo_cf]; |
749 |
||
| 5136 | 750 |
Goal "[| chain(cf(D,E),X); cpo(D); cpo(E)|] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
751 |
\ lub(cf(D,E), X) = (lam x:set(D). lub(E,lam n:nat. X`n`x))"; |
| 5136 | 752 |
by (blast_tac (claset() addIs [islub_unique,cpo_lub,islub_cf,cpo_cf]) 1); |
| 3425 | 753 |
qed "lub_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
754 |
|
| 5136 | 755 |
Goal "[|y:set(E); cpo(D); cpo(E)|] ==> (lam x:set(D).y) : cont(D,E)"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
756 |
by (rtac contI 1); |
| 2469 | 757 |
by (Asm_simp_tac 2); |
| 5136 | 758 |
by (blast_tac (claset() addIs [lam_type]) 1); |
759 |
by (asm_simp_tac(simpset() addsimps [chain_in, cpo_lub RS islub_in, |
|
760 |
lub_const]) 1); |
|
| 3425 | 761 |
qed "const_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
762 |
|
| 5136 | 763 |
Goal "[|cpo(D); pcpo(E); y:cont(D,E)|]==>rel(cf(D,E),(lam x:set(D).bot(E)),y)"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
764 |
by (rtac rel_cfI 1); |
| 2469 | 765 |
by (Asm_simp_tac 1); |
| 6169 | 766 |
by (ALLGOALS (type_solver_tac (tcset() addTCs [cont_fun, const_cont]) [])); |
| 3425 | 767 |
qed "cf_least"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
768 |
|
| 5136 | 769 |
Goal (* pcpo_cf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
770 |
"[|cpo(D); pcpo(E)|] ==> pcpo(cf(D,E))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
771 |
by (rtac pcpoI 1); |
| 5136 | 772 |
brr[cf_least, bot_in, const_cont RS cont_cf, cf_cont, cpo_cf, pcpo_cpo] 1; |
| 3425 | 773 |
qed "pcpo_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
774 |
|
| 5136 | 775 |
Goal (* bot_cf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
776 |
"[|cpo(D); pcpo(E)|] ==> bot(cf(D,E)) = (lam x:set(D).bot(E))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
777 |
by (rtac (bot_unique RS sym) 1); |
| 5136 | 778 |
brr[pcpo_cf, cf_least, bot_in RS const_cont RS cont_cf, cf_cont, pcpo_cpo] 1; |
| 3425 | 779 |
qed "bot_cf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
780 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
781 |
(*----------------------------------------------------------------------*) |
| 1461 | 782 |
(* Identity and composition. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
783 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
784 |
|
| 5136 | 785 |
Goal (* id_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
786 |
"cpo(D) ==> id(set(D)):cont(D,D)"; |
| 6169 | 787 |
by (asm_simp_tac(simpset() addsimps[id_type, contI, cpo_lub RS islub_in, |
788 |
chain_fun RS eta]) 1); |
|
| 3425 | 789 |
qed "id_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
790 |
|
| 6153 | 791 |
AddTCs [id_cont]; |
792 |
||
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
793 |
val comp_cont_apply = cont_fun RSN(2,cont_fun RS comp_fun_apply); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
794 |
|
| 5136 | 795 |
Goal (* comp_pres_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
796 |
"[| f:cont(D',E); g:cont(D,D'); cpo(D)|] ==> f O g : cont(D,E)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
797 |
by (rtac contI 1); |
| 2034 | 798 |
by (stac comp_cont_apply 2); |
799 |
by (stac comp_cont_apply 5); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
800 |
by (rtac cont_mono 8); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
801 |
by (rtac cont_mono 9); (* 15 subgoals *) |
| 6169 | 802 |
by Typecheck_tac; (* proves all but the lub case *) |
| 2034 | 803 |
by (stac comp_cont_apply 1); |
804 |
by (stac cont_lub 4); |
|
805 |
by (stac cont_lub 6); |
|
| 5136 | 806 |
by (asm_full_simp_tac(simpset() addsimps [comp_cont_apply,chain_in]) 8); |
807 |
by (auto_tac (claset() addIs [cpo_lub RS islub_in, cont_chain], simpset())); |
|
| 3425 | 808 |
qed "comp_pres_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
809 |
|
| 6153 | 810 |
AddTCs [comp_pres_cont]; |
811 |
||
| 5136 | 812 |
Goal (* comp_mono *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
813 |
"[| f:cont(D',E); g:cont(D,D'); f':cont(D',E); g':cont(D,D'); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
814 |
\ rel(cf(D',E),f,f'); rel(cf(D,D'),g,g'); cpo(D); cpo(E) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
815 |
\ rel(cf(D,E),f O g,f' O g')"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
816 |
by (rtac rel_cfI 1); (* extra proof obl: f O g and f' O g' cont. Extra asm cpo(D). *) |
| 2034 | 817 |
by (stac comp_cont_apply 1); |
818 |
by (stac comp_cont_apply 4); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
819 |
by (rtac cpo_trans 7); |
| 5136 | 820 |
by (REPEAT (ares_tac [rel_cf,cont_mono,cont_map,comp_pres_cont] 1)); |
| 3425 | 821 |
qed "comp_mono"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
822 |
|
| 5136 | 823 |
Goal (* chain_cf_comp *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
824 |
"[| chain(cf(D',E),X); chain(cf(D,D'),Y); cpo(D); cpo(E)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
825 |
\ chain(cf(D,E),lam n:nat. X`n O Y`n)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
826 |
by (rtac chainI 1); |
| 2469 | 827 |
by (Asm_simp_tac 2); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
828 |
by (rtac rel_cfI 2); |
| 2034 | 829 |
by (stac comp_cont_apply 2); |
830 |
by (stac comp_cont_apply 5); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
831 |
by (rtac cpo_trans 8); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
832 |
by (rtac rel_cf 9); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
833 |
by (rtac cont_mono 11); |
| 5136 | 834 |
brr[lam_type, comp_pres_cont, cont_cf, chain_in RS cf_cont, cont_map, chain_rel,rel_cf,nat_succI] 1; |
| 3425 | 835 |
qed "chain_cf_comp"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
836 |
|
| 5136 | 837 |
Goal (* comp_lubs *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
838 |
"[| chain(cf(D',E),X); chain(cf(D,D'),Y); cpo(D); cpo(D'); cpo(E)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
839 |
\ lub(cf(D',E),X) O lub(cf(D,D'),Y) = lub(cf(D,E),lam n:nat. X`n O Y`n)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
840 |
by (rtac fun_extension 1); |
| 2034 | 841 |
by (stac lub_cf 3); |
| 5136 | 842 |
brr[comp_fun, cf_cont RS cont_fun, cpo_lub RS islub_in, cpo_cf, chain_cf_comp] 1; |
843 |
by (asm_simp_tac(simpset() |
|
844 |
addsimps[chain_in RS |
|
845 |
cf_cont RSN(3,chain_in RS |
|
846 |
cf_cont RS comp_cont_apply)]) 1); |
|
| 2034 | 847 |
by (stac comp_cont_apply 1); |
| 5136 | 848 |
brr[cpo_lub RS islub_in RS cf_cont, cpo_cf] 1; |
849 |
by (asm_simp_tac(simpset() addsimps |
|
850 |
[lub_cf,chain_cf, chain_in RS cf_cont RS cont_lub, |
|
851 |
chain_cf RS cpo_lub RS islub_in]) 1); |
|
| 1623 | 852 |
by (cut_inst_tac[("M","lam xa:nat. lam xb:nat. X`xa`(Y`xb`x)")]
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
853 |
lub_matrix_diag 1); |
| 2469 | 854 |
by (Asm_full_simp_tac 3); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
855 |
by (rtac matrix_chainI 1); |
| 2469 | 856 |
by (Asm_simp_tac 1); |
| 5525 | 857 |
by (Asm_simp_tac 2); |
858 |
by (dtac (chain_in RS cf_cont) 1 THEN atac 1); |
|
859 |
by (fast_tac (claset() addDs [chain_cf RSN(2,cont_chain)] |
|
| 5136 | 860 |
addss simpset()) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
861 |
by (rtac chain_cf 1); |
| 5136 | 862 |
by (REPEAT (ares_tac [cont_fun RS apply_type, chain_in RS cf_cont, |
863 |
lam_type] 1)); |
|
| 3425 | 864 |
qed "comp_lubs"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
865 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
866 |
(*----------------------------------------------------------------------*) |
| 1461 | 867 |
(* Theorems about projpair. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
868 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
869 |
|
| 5136 | 870 |
Goalw [projpair_def] (* projpairI *) |
871 |
"[| e:cont(D,E); p:cont(E,D); p O e = id(set(D)); \ |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
872 |
\ rel(cf(E,E))(e O p)(id(set(E)))|] ==> projpair(D,E,e,p)"; |
| 2469 | 873 |
by (Fast_tac 1); |
| 3425 | 874 |
qed "projpairI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
875 |
|
| 5136 | 876 |
val prems = Goalw [projpair_def] (* projpairE *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
877 |
"[| projpair(D,E,e,p); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
878 |
\ [| e:cont(D,E); p:cont(E,D); p O e = id(set(D)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
879 |
\ rel(cf(E,E))(e O p)(id(set(E)))|] ==> Q |] ==> Q"; |
| 1623 | 880 |
by (rtac (hd(tl prems)) 1); |
| 4091 | 881 |
by (REPEAT(asm_simp_tac(simpset() addsimps[hd prems]) 1)); |
| 3425 | 882 |
qed "projpairE"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
883 |
|
| 5136 | 884 |
Goal "projpair(D,E,e,p) ==> e:cont(D,E)"; |
885 |
by (etac projpairE 1); |
|
886 |
by (assume_tac 1); |
|
| 3425 | 887 |
qed "projpair_e_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
888 |
|
| 5136 | 889 |
Goal (* projpair_p_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
890 |
"projpair(D,E,e,p) ==> p:cont(E,D)"; |
| 5136 | 891 |
by (etac projpairE 1); |
892 |
by (assume_tac 1); |
|
| 3425 | 893 |
qed "projpair_p_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
894 |
|
| 5136 | 895 |
Goal "projpair(D,E,e,p) ==> p O e = id(set(D))"; |
896 |
by (etac projpairE 1); |
|
897 |
by (assume_tac 1); |
|
| 3425 | 898 |
qed "projpair_eq"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
899 |
|
| 5136 | 900 |
Goal (* projpair_rel *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
901 |
"projpair(D,E,e,p) ==> rel(cf(E,E))(e O p)(id(set(E)))"; |
| 5136 | 902 |
by (etac projpairE 1); |
903 |
by (assume_tac 1); |
|
| 3425 | 904 |
qed "projpair_rel"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
905 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
906 |
val projpairDs = [projpair_e_cont,projpair_p_cont,projpair_eq,projpair_rel]; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
907 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
908 |
(*----------------------------------------------------------------------*) |
| 1461 | 909 |
(* NB! projpair_e_cont and projpair_p_cont cannot be used repeatedly *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
910 |
(* at the same time since both match a goal of the form f:cont(X,Y).*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
911 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
912 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
913 |
(*----------------------------------------------------------------------*) |
| 1461 | 914 |
(* Uniqueness of embedding projection pairs. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
915 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
916 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
917 |
val id_comp = fun_is_rel RS left_comp_id; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
918 |
val comp_id = fun_is_rel RS right_comp_id; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
919 |
|
| 5136 | 920 |
val prems = goal thy (* lemma1 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
921 |
"[|cpo(D); cpo(E); projpair(D,E,e,p); projpair(D,E,e',p'); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
922 |
\ rel(cf(D,E),e,e')|] ==> rel(cf(E,D),p',p)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
923 |
val [_,_,p1,p2,_] = prems; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
924 |
(* The two theorems proj_e_cont and proj_p_cont are useless unless they |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
925 |
are used manually, one at a time. Therefore the following contl. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
926 |
val contl = [p1 RS projpair_e_cont,p1 RS projpair_p_cont, |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
927 |
p2 RS projpair_e_cont,p2 RS projpair_p_cont]; |
| 1623 | 928 |
by (rtac (p2 RS projpair_p_cont RS cont_fun RS id_comp RS subst) 1); |
929 |
by (rtac (p1 RS projpair_eq RS subst) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
930 |
by (rtac cpo_trans 1); |
| 1623 | 931 |
brr(cpo_cf::prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
932 |
(* The following corresponds to EXISTS_TAC, non-trivial instantiation. *) |
| 1623 | 933 |
by (res_inst_tac[("f","p O (e' O p')")]cont_cf 4);
|
| 2034 | 934 |
by (stac comp_assoc 1); |
| 1623 | 935 |
brr(cpo_refl::cpo_cf::cont_cf::comp_mono::comp_pres_cont::(contl@prems)) 1; |
936 |
by (res_inst_tac[("P","%x. rel(cf(E,D),p O e' O p',x)")]
|
|
937 |
(p1 RS projpair_p_cont RS cont_fun RS comp_id RS subst) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
938 |
by (rtac comp_mono 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
939 |
brr(cpo_refl::cpo_cf::cont_cf::comp_mono::comp_pres_cont::id_cont:: |
| 1623 | 940 |
projpair_rel::(contl@prems)) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
941 |
val lemma1 = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
942 |
|
| 5136 | 943 |
val prems = goal thy (* lemma2 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
944 |
"[|cpo(D); cpo(E); projpair(D,E,e,p); projpair(D,E,e',p'); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
945 |
\ rel(cf(E,D),p',p)|] ==> rel(cf(D,E),e,e')"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
946 |
val [_,_,p1,p2,_] = prems; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
947 |
val contl = [p1 RS projpair_e_cont,p1 RS projpair_p_cont, |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
948 |
p2 RS projpair_e_cont,p2 RS projpair_p_cont]; |
| 1623 | 949 |
by (rtac (p1 RS projpair_e_cont RS cont_fun RS comp_id RS subst) 1); |
950 |
by (rtac (p2 RS projpair_eq RS subst) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
951 |
by (rtac cpo_trans 1); |
| 1623 | 952 |
brr(cpo_cf::prems) 1; |
953 |
by (res_inst_tac[("f","(e O p) O e'")]cont_cf 4);
|
|
| 2034 | 954 |
by (stac comp_assoc 1); |
| 1623 | 955 |
brr((cpo_cf RS cpo_refl)::cont_cf::comp_mono::comp_pres_cont::(contl@prems)) 1; |
956 |
by (res_inst_tac[("P","%x. rel(cf(D,E),(e O p) O e',x)")]
|
|
957 |
(p2 RS projpair_e_cont RS cont_fun RS id_comp RS subst) 1); |
|
| 5136 | 958 |
brr((cpo_cf RS cpo_refl)::cont_cf::comp_mono::id_cont::comp_pres_cont::projpair_rel::(contl@prems)) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
959 |
val lemma2 = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
960 |
|
| 5136 | 961 |
val prems = goal thy (* projpair_unique *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
962 |
"[|cpo(D); cpo(E); projpair(D,E,e,p); projpair(D,E,e',p')|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
963 |
\ (e=e')<->(p=p')"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
964 |
val [_,_,p1,p2] = prems; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
965 |
val contl = [p1 RS projpair_e_cont,p1 RS projpair_p_cont, |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
966 |
p2 RS projpair_e_cont,p2 RS projpair_p_cont]; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
967 |
by (rtac iffI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
968 |
by (rtac cpo_antisym 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
969 |
by (rtac lemma1 2); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
970 |
(* First some existentials are instantiated. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
971 |
by (resolve_tac prems 4); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
972 |
by (resolve_tac prems 4); |
| 2469 | 973 |
by (Asm_simp_tac 4); |
| 5136 | 974 |
brr([cpo_cf,cpo_refl,cont_cf,projpair_e_cont]@prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
975 |
by (rtac lemma1 1); |
| 5136 | 976 |
by (REPEAT (ares_tac prems 1)); |
| 2469 | 977 |
by (Asm_simp_tac 1); |
| 1623 | 978 |
brr(cpo_cf::cpo_refl::cont_cf::(contl @ prems)) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
979 |
by (rtac cpo_antisym 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
980 |
by (rtac lemma2 2); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
981 |
(* First some existentials are instantiated. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
982 |
by (resolve_tac prems 4); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
983 |
by (resolve_tac prems 4); |
| 2469 | 984 |
by (Asm_simp_tac 4); |
| 5136 | 985 |
brr([cpo_cf,cpo_refl,cont_cf,projpair_p_cont]@prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
986 |
by (rtac lemma2 1); |
| 5136 | 987 |
by (REPEAT (ares_tac prems 1)); |
| 2469 | 988 |
by (Asm_simp_tac 1); |
| 1623 | 989 |
brr(cpo_cf::cpo_refl::cont_cf::(contl @ prems)) 1; |
| 3425 | 990 |
qed "projpair_unique"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
991 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
992 |
(* Slightly different, more asms, since THE chooses the unique element. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
993 |
|
| 5136 | 994 |
Goalw [emb_def,Rp_def] (* embRp *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
995 |
"[|emb(D,E,e); cpo(D); cpo(E)|] ==> projpair(D,E,e,Rp(D,E,e))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
996 |
by (rtac theI2 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
997 |
by (assume_tac 2); |
| 5136 | 998 |
by (blast_tac (claset() addIs [projpair_unique RS iffD1]) 1); |
| 3425 | 999 |
qed "embRp"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1000 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1001 |
val embI = prove_goalw Limit.thy [emb_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1002 |
"!!x. projpair(D,E,e,p) ==> emb(D,E,e)" |
| 2469 | 1003 |
(fn prems => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1004 |
|
| 5136 | 1005 |
Goal "[|projpair(D,E,e,p); cpo(D); cpo(E)|] ==> Rp(D,E,e) = p"; |
1006 |
by (blast_tac (claset() addIs [embRp, embI, projpair_unique RS iffD1]) 1); |
|
| 3425 | 1007 |
qed "Rp_unique"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1008 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1009 |
val emb_cont = prove_goalw Limit.thy [emb_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1010 |
"emb(D,E,e) ==> e:cont(D,E)" |
| 1623 | 1011 |
(fn prems => [rtac(hd prems RS exE) 1,rtac projpair_e_cont 1,atac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1012 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1013 |
(* The following three theorems have cpo asms due to THE (uniqueness). *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1014 |
|
| 6153 | 1015 |
bind_thm ("Rp_cont", embRp RS projpair_p_cont);
|
1016 |
bind_thm ("embRp_eq", embRp RS projpair_eq);
|
|
1017 |
bind_thm ("embRp_rel", embRp RS projpair_rel);
|
|
1018 |
||
|
6176
707b6f9859d2
tidied, with left_inverse & right_inverse as default simprules
paulson
parents:
6169
diff
changeset
|
1019 |
AddTCs [emb_cont, Rp_cont]; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1020 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1021 |
val id_apply = prove_goalw Perm.thy [id_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1022 |
"!!z. x:A ==> id(A)`x = x" |
| 2469 | 1023 |
(fn prems => [Asm_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1024 |
|
| 5136 | 1025 |
Goal (* embRp_eq_thm *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1026 |
"[|emb(D,E,e); x:set(D); cpo(D); cpo(E)|] ==> Rp(D,E,e)`(e`x) = x"; |
| 1623 | 1027 |
by (rtac (comp_fun_apply RS subst) 1); |
| 5136 | 1028 |
brr[Rp_cont,emb_cont,cont_fun] 1; |
| 2034 | 1029 |
by (stac embRp_eq 1); |
| 5136 | 1030 |
by (auto_tac (claset() addIs [id_apply], simpset())); |
| 3425 | 1031 |
qed "embRp_eq_thm"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1032 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1033 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1034 |
(*----------------------------------------------------------------------*) |
| 1461 | 1035 |
(* The identity embedding. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1036 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1037 |
|
| 5136 | 1038 |
Goalw [projpair_def] (* projpair_id *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1039 |
"cpo(D) ==> projpair(D,D,id(set(D)),id(set(D)))"; |
| 4152 | 1040 |
by Safe_tac; |
| 5136 | 1041 |
brr[id_cont,id_comp,id_type] 1; |
| 2034 | 1042 |
by (stac id_comp 1); (* Matches almost anything *) |
| 5136 | 1043 |
brr[id_cont,id_type,cpo_refl,cpo_cf,cont_cf] 1; |
| 3425 | 1044 |
qed "projpair_id"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1045 |
|
| 5136 | 1046 |
Goal (* emb_id *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1047 |
"cpo(D) ==> emb(D,D,id(set(D)))"; |
| 5136 | 1048 |
by (auto_tac (claset() addIs [embI,projpair_id], simpset())); |
| 3425 | 1049 |
qed "emb_id"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1050 |
|
| 5136 | 1051 |
Goal (* Rp_id *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1052 |
"cpo(D) ==> Rp(D,D,id(set(D))) = id(set(D))"; |
| 5136 | 1053 |
by (auto_tac (claset() addIs [Rp_unique,projpair_id], simpset())); |
| 3425 | 1054 |
qed "Rp_id"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1055 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1056 |
(*----------------------------------------------------------------------*) |
| 1461 | 1057 |
(* Composition preserves embeddings. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1058 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1059 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1060 |
(* Considerably shorter, only partly due to a simpler comp_assoc. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1061 |
(* Proof in HOL-ST: 70 lines (minus 14 due to comp_assoc complication). *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1062 |
(* Proof in Isa/ZF: 23 lines (compared to 56: 60% reduction). *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1063 |
|
| 5136 | 1064 |
Goalw [projpair_def] (* lemma *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1065 |
"[|emb(D,D',e); emb(D',E,e'); cpo(D); cpo(D'); cpo(E)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1066 |
\ projpair(D,E,e' O e,(Rp(D,D',e)) O (Rp(D',E,e')))"; |
| 4152 | 1067 |
by Safe_tac; |
| 5136 | 1068 |
brr[comp_pres_cont,Rp_cont,emb_cont] 1; |
| 1623 | 1069 |
by (rtac (comp_assoc RS subst) 1); |
1070 |
by (res_inst_tac[("t1","e'")](comp_assoc RS ssubst) 1);
|
|
| 2034 | 1071 |
by (stac embRp_eq 1); (* Matches everything due to subst/ssubst. *) |
| 5136 | 1072 |
by (REPEAT (assume_tac 1)); |
| 2034 | 1073 |
by (stac comp_id 1); |
| 5136 | 1074 |
brr[cont_fun,Rp_cont,embRp_eq] 1; |
| 1623 | 1075 |
by (rtac (comp_assoc RS subst) 1); |
1076 |
by (res_inst_tac[("t1","Rp(D,D',e)")](comp_assoc RS ssubst) 1);
|
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1077 |
by (rtac cpo_trans 1); |
| 5136 | 1078 |
brr[cpo_cf] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1079 |
by (rtac comp_mono 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1080 |
by (rtac cpo_refl 6); |
| 5136 | 1081 |
brr[cont_cf,Rp_cont] 7; |
1082 |
brr[cpo_cf] 6; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1083 |
by (rtac comp_mono 5); |
| 5136 | 1084 |
brr[embRp_rel] 10; |
1085 |
brr[cpo_cf RS cpo_refl, cont_cf,Rp_cont] 9; |
|
| 2034 | 1086 |
by (stac comp_id 10); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1087 |
by (rtac embRp_rel 11); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1088 |
(* There are 16 subgoals at this point. All are proved immediately by: *) |
| 5136 | 1089 |
by (REPEAT (ares_tac [comp_pres_cont,Rp_cont,id_cont, |
1090 |
emb_cont,cont_fun,cont_cf] 1)); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1091 |
val lemma = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1092 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1093 |
(* The use of RS is great in places like the following, both ugly in HOL. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1094 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1095 |
val emb_comp = lemma RS embI; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1096 |
val Rp_comp = lemma RS Rp_unique; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1097 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1098 |
(*----------------------------------------------------------------------*) |
| 1461 | 1099 |
(* Infinite cartesian product. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1100 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1101 |
|
| 5136 | 1102 |
Goalw [set_def,iprod_def] (* iprodI *) |
|
5147
825877190618
More tidying and removal of "\!\!... from Goal commands
paulson
parents:
5136
diff
changeset
|
1103 |
"x:(PROD n:nat. set(DD`n)) ==> x:set(iprod(DD))"; |
| 2469 | 1104 |
by (Asm_full_simp_tac 1); |
| 3425 | 1105 |
qed "iprodI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1106 |
|
| 5136 | 1107 |
Goalw [set_def,iprod_def] (* iprodE *) |
|
5147
825877190618
More tidying and removal of "\!\!... from Goal commands
paulson
parents:
5136
diff
changeset
|
1108 |
"x:set(iprod(DD)) ==> x:(PROD n:nat. set(DD`n))"; |
| 2469 | 1109 |
by (Asm_full_simp_tac 1); |
| 3425 | 1110 |
qed "iprodE"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1111 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1112 |
(* Contains typing conditions in contrast to HOL-ST *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1113 |
|
| 5136 | 1114 |
val prems = Goalw [iprod_def] (* rel_iprodI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1115 |
"[|!!n. n:nat ==> rel(DD`n,f`n,g`n); f:(PROD n:nat. set(DD`n)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1116 |
\ g:(PROD n:nat. set(DD`n))|] ==> rel(iprod(DD),f,g)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1117 |
by (rtac rel_I 1); |
| 2469 | 1118 |
by (Simp_tac 1); |
| 4152 | 1119 |
by Safe_tac; |
| 5136 | 1120 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 1121 |
qed "rel_iprodI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1122 |
|
| 5136 | 1123 |
Goalw [iprod_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1124 |
"[|rel(iprod(DD),f,g); n:nat|] ==> rel(DD`n,f`n,g`n)"; |
| 5136 | 1125 |
by (fast_tac (claset() addDs [rel_E] addss simpset()) 1); |
| 3425 | 1126 |
qed "rel_iprodE"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1127 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1128 |
(* Some special theorems like dProdApIn_cpo and other `_cpo' |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1129 |
probably not needed in Isabelle, wait and see. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1130 |
|
| 5136 | 1131 |
val prems = Goalw [chain_def] (* chain_iprod *) |
| 2469 | 1132 |
"[|chain(iprod(DD),X); !!n. n:nat ==> cpo(DD`n); n:nat|] ==> \ |
| 3840 | 1133 |
\ chain(DD`n,lam m:nat. X`m`n)"; |
| 4152 | 1134 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1135 |
by (rtac lam_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1136 |
by (rtac apply_type 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1137 |
by (rtac iprodE 1); |
| 1623 | 1138 |
by (etac (hd prems RS conjunct1 RS apply_type) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1139 |
by (resolve_tac prems 1); |
| 4091 | 1140 |
by (asm_simp_tac(simpset() addsimps prems) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1141 |
by (rtac rel_iprodE 1); |
| 4091 | 1142 |
by (asm_simp_tac (simpset() addsimps prems) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1143 |
by (resolve_tac prems 1); |
| 3425 | 1144 |
qed "chain_iprod"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1145 |
|
| 5136 | 1146 |
val prems = Goalw [islub_def,isub_def] (* islub_iprod *) |
| 2469 | 1147 |
"[|chain(iprod(DD),X); !!n. n:nat ==> cpo(DD`n)|] ==> \ |
| 3840 | 1148 |
\ islub(iprod(DD),X,lam n:nat. lub(DD`n,lam m:nat. X`m`n))"; |
| 4152 | 1149 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1150 |
by (rtac iprodI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1151 |
by (rtac lam_type 1); |
| 1623 | 1152 |
brr((chain_iprod RS cpo_lub RS islub_in)::prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1153 |
by (rtac rel_iprodI 1); |
| 2469 | 1154 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1155 |
(* Here, HOL resolution is handy, Isabelle resolution bad. *) |
| 1623 | 1156 |
by (res_inst_tac[("P","%t. rel(DD`na,t,lub(DD`na,lam x:nat. X`x`na))"),
|
1157 |
("b1","%n. X`n`na")](beta RS subst) 1);
|
|
1158 |
brr((chain_iprod RS cpo_lub RS islub_ub)::iprodE::chain_in::prems) 1; |
|
1159 |
brr(iprodI::lam_type::(chain_iprod RS cpo_lub RS islub_in)::prems) 1; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1160 |
by (rtac rel_iprodI 1); |
| 2469 | 1161 |
by (Asm_simp_tac 1); |
| 1623 | 1162 |
brr(islub_least::(chain_iprod RS cpo_lub)::prems) 1; |
1163 |
by (rewtac isub_def); |
|
| 4152 | 1164 |
by Safe_tac; |
| 1623 | 1165 |
by (etac (iprodE RS apply_type) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1166 |
by (assume_tac 1); |
| 2469 | 1167 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1168 |
by (dtac bspec 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1169 |
by (etac rel_iprodE 2); |
| 1623 | 1170 |
brr(lam_type::(chain_iprod RS cpo_lub RS islub_in)::iprodE::prems) 1; |
| 3425 | 1171 |
qed "islub_iprod"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1172 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1173 |
val prems = goal Limit.thy (* cpo_iprod *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1174 |
"(!!n. n:nat ==> cpo(DD`n)) ==> cpo(iprod(DD))"; |
| 5136 | 1175 |
brr[cpoI,poI] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1176 |
by (rtac rel_iprodI 1); (* not repeated: want to solve 1 and leave 2 unchanged *) |
| 1623 | 1177 |
brr(cpo_refl::(iprodE RS apply_type)::iprodE::prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1178 |
by (rtac rel_iprodI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1179 |
by (dtac rel_iprodE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1180 |
by (dtac rel_iprodE 2); |
| 1623 | 1181 |
brr(cpo_trans::(iprodE RS apply_type)::iprodE::prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1182 |
by (rtac fun_extension 1); |
| 1623 | 1183 |
brr(cpo_antisym::rel_iprodE::(iprodE RS apply_type)::iprodE::prems) 1; |
1184 |
brr(islub_iprod::prems) 1; |
|
| 3425 | 1185 |
qed "cpo_iprod"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1186 |
|
| 6158 | 1187 |
AddTCs [cpo_iprod]; |
1188 |
||
| 5136 | 1189 |
val prems = Goalw [islub_def,isub_def] (* lub_iprod *) |
| 2469 | 1190 |
"[|chain(iprod(DD),X); !!n. n:nat ==> cpo(DD`n)|] ==> \ |
| 3840 | 1191 |
\ lub(iprod(DD),X) = (lam n:nat. lub(DD`n,lam m:nat. X`m`n))"; |
| 1623 | 1192 |
brr((cpo_lub RS islub_unique)::islub_iprod::cpo_iprod::prems) 1; |
| 3425 | 1193 |
qed "lub_iprod"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1194 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1195 |
(*----------------------------------------------------------------------*) |
| 1461 | 1196 |
(* The notion of subcpo. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1197 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1198 |
|
| 5136 | 1199 |
val prems = Goalw [subcpo_def] (* subcpoI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1200 |
"[|set(D)<=set(E); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1201 |
\ !!x y. [|x:set(D); y:set(D)|] ==> rel(D,x,y)<->rel(E,x,y); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1202 |
\ !!X. chain(D,X) ==> lub(E,X) : set(D)|] ==> subcpo(D,E)"; |
| 4152 | 1203 |
by Safe_tac; |
| 4091 | 1204 |
by (asm_full_simp_tac(simpset() addsimps prems) 2); |
1205 |
by (asm_simp_tac(simpset() addsimps prems) 2); |
|
| 1623 | 1206 |
brr(prems@[subsetD]) 1; |
| 3425 | 1207 |
qed "subcpoI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1208 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1209 |
val subcpo_subset = prove_goalw Limit.thy [subcpo_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1210 |
"!!x. subcpo(D,E) ==> set(D)<=set(E)" |
| 2469 | 1211 |
(fn prems => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1212 |
|
| 5136 | 1213 |
Goalw [subcpo_def] |
1214 |
"[|subcpo(D,E); x:set(D); y:set(D)|] ==> rel(D,x,y)<->rel(E,x,y)"; |
|
1215 |
by (Blast_tac 1); |
|
1216 |
qed "subcpo_rel_eq"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1217 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1218 |
val subcpo_relD1 = subcpo_rel_eq RS iffD1; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1219 |
val subcpo_relD2 = subcpo_rel_eq RS iffD2; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1220 |
|
| 5136 | 1221 |
Goalw [subcpo_def] "[|subcpo(D,E); chain(D,X)|] ==> lub(E,X) : set(D)"; |
1222 |
by (Blast_tac 1); |
|
1223 |
qed "subcpo_lub"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1224 |
|
| 5136 | 1225 |
Goal "[|subcpo(D,E); chain(D,X)|] ==> chain(E,X)"; |
1226 |
by (rtac (Pi_type RS chainI) 1); |
|
1227 |
by (REPEAT |
|
1228 |
(blast_tac (claset() addIs [chain_fun, subcpo_relD1, |
|
1229 |
subcpo_subset RS subsetD, |
|
1230 |
chain_in, chain_rel]) 1)); |
|
| 3425 | 1231 |
qed "chain_subcpo"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1232 |
|
| 5136 | 1233 |
Goal "[|subcpo(D,E); chain(D,X); isub(D,X,x)|] ==> isub(E,X,x)"; |
1234 |
by (blast_tac (claset() addIs [isubI, subcpo_relD1,subcpo_relD1, |
|
1235 |
chain_in, isubD1, isubD2, |
|
1236 |
subcpo_subset RS subsetD, |
|
1237 |
chain_in, chain_rel]) 1); |
|
| 3425 | 1238 |
qed "ub_subcpo"; |
| 1461 | 1239 |
|
| 5136 | 1240 |
Goal "[|subcpo(D,E); cpo(E); chain(D,X)|] ==> islub(D,X,lub(E,X))"; |
1241 |
by (blast_tac (claset() addIs [islubI, isubI, subcpo_lub, |
|
1242 |
subcpo_relD2, chain_in, |
|
1243 |
islub_ub, islub_least, cpo_lub, |
|
1244 |
chain_subcpo, isubD1, ub_subcpo]) 1); |
|
| 3425 | 1245 |
qed "islub_subcpo"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1246 |
|
| 5136 | 1247 |
Goal "[|subcpo(D,E); cpo(E)|] ==> cpo(D)"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1248 |
brr[cpoI,poI]1; |
| 5136 | 1249 |
by (asm_full_simp_tac(simpset() addsimps[subcpo_rel_eq]) 1); |
1250 |
brr[cpo_refl, subcpo_subset RS subsetD] 1; |
|
1251 |
by (rotate_tac ~3 1); |
|
1252 |
by (asm_full_simp_tac(simpset() addsimps[subcpo_rel_eq]) 1); |
|
1253 |
by (blast_tac (claset() addIs [subcpo_subset RS subsetD, cpo_trans]) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1254 |
(* Changing the order of the assumptions, otherwise full_simp doesn't work. *) |
| 5136 | 1255 |
by (rotate_tac ~2 1); |
1256 |
by (asm_full_simp_tac(simpset() addsimps[subcpo_rel_eq]) 1); |
|
1257 |
by (blast_tac (claset() addIs [cpo_antisym, subcpo_subset RS subsetD]) 1); |
|
1258 |
by (fast_tac (claset() addIs [islub_subcpo]) 1); |
|
| 3425 | 1259 |
qed "subcpo_cpo"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1260 |
|
| 5136 | 1261 |
Goal "[|subcpo(D,E); cpo(E); chain(D,X)|] ==> lub(D,X) = lub(E,X)"; |
1262 |
by (blast_tac (claset() addIs [cpo_lub RS islub_unique, |
|
1263 |
islub_subcpo, subcpo_cpo]) 1); |
|
| 3425 | 1264 |
qed "lub_subcpo"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1265 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1266 |
(*----------------------------------------------------------------------*) |
| 1461 | 1267 |
(* Making subcpos using mkcpo. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1268 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1269 |
|
| 5136 | 1270 |
Goalw [set_def,mkcpo_def] "[|x:set(D); P(x)|] ==> x:set(mkcpo(D,P))"; |
1271 |
by Auto_tac; |
|
| 3425 | 1272 |
qed "mkcpoI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1273 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1274 |
(* Old proof where cpos are non-reflexive relations. |
| 1623 | 1275 |
by (rewtac set_def); (* Annoying, cannot just rewrite once. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1276 |
by (rtac CollectI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1277 |
by (rtac domainI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1278 |
by (rtac CollectI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1279 |
(* Now, work on subgoal 2 (and 3) to instantiate unknown. *) |
| 2469 | 1280 |
by (Simp_tac 2); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1281 |
by (rtac conjI 2); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1282 |
by (rtac conjI 3); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1283 |
by (resolve_tac prems 3); |
| 4091 | 1284 |
by (simp_tac(simpset() addsimps [rewrite_rule[set_def](hd prems)]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1285 |
by (resolve_tac prems 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1286 |
by (rtac cpo_refl 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1287 |
by (resolve_tac prems 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1288 |
by (rtac rel_I 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1289 |
by (rtac CollectI 1); |
| 4091 | 1290 |
by (fast_tac(claset() addSIs [rewrite_rule[set_def](hd prems)]) 1); |
| 2469 | 1291 |
by (Simp_tac 1); |
| 5136 | 1292 |
brr[conjI,cpo_refl] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1293 |
*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1294 |
|
| 5136 | 1295 |
Goalw [set_def,mkcpo_def] (* mkcpoD1 *) |
|
5147
825877190618
More tidying and removal of "\!\!... from Goal commands
paulson
parents:
5136
diff
changeset
|
1296 |
"x:set(mkcpo(D,P))==> x:set(D)"; |
| 2469 | 1297 |
by (Asm_full_simp_tac 1); |
| 3425 | 1298 |
qed "mkcpoD1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1299 |
|
| 5136 | 1300 |
Goalw [set_def,mkcpo_def] (* mkcpoD2 *) |
|
5147
825877190618
More tidying and removal of "\!\!... from Goal commands
paulson
parents:
5136
diff
changeset
|
1301 |
"x:set(mkcpo(D,P))==> P(x)"; |
| 2469 | 1302 |
by (Asm_full_simp_tac 1); |
| 3425 | 1303 |
qed "mkcpoD2"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1304 |
|
| 5136 | 1305 |
Goalw [rel_def,mkcpo_def] (* rel_mkcpoE *) |
|
5147
825877190618
More tidying and removal of "\!\!... from Goal commands
paulson
parents:
5136
diff
changeset
|
1306 |
"rel(mkcpo(D,P),x,y) ==> rel(D,x,y)"; |
| 2469 | 1307 |
by (Asm_full_simp_tac 1); |
| 3425 | 1308 |
qed "rel_mkcpoE"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1309 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1310 |
val rel_mkcpo = prove_goalw Limit.thy [mkcpo_def,rel_def,set_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1311 |
"!!z. [|x:set(D); y:set(D)|] ==> rel(mkcpo(D,P),x,y) <-> rel(D,x,y)" |
| 2469 | 1312 |
(fn prems => [Asm_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1313 |
|
| 2469 | 1314 |
(* The HOL proof is simpler, problems due to cpos as purely in upair. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1315 |
(* And chains as set functions. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1316 |
|
| 5136 | 1317 |
Goal (* chain_mkcpo *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1318 |
"chain(mkcpo(D,P),X) ==> chain(D,X)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1319 |
by (rtac chainI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1320 |
(*---begin additional---*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1321 |
by (rtac Pi_type 1); |
| 5136 | 1322 |
brr[chain_fun] 1; |
1323 |
brr[chain_in RS mkcpoD1] 1; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1324 |
(*---end additional---*) |
| 1623 | 1325 |
by (rtac (rel_mkcpo RS iffD1) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1326 |
(*---begin additional---*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1327 |
by (rtac mkcpoD1 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1328 |
by (rtac mkcpoD1 2); |
| 5136 | 1329 |
brr[chain_in,nat_succI] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1330 |
(*---end additional---*) |
| 5136 | 1331 |
by (auto_tac (claset() addIs [chain_rel], simpset())); |
| 3425 | 1332 |
qed "chain_mkcpo"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1333 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1334 |
val prems = goal Limit.thy (* subcpo_mkcpo *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1335 |
"[|!!X. chain(mkcpo(D,P),X) ==> P(lub(D,X)); cpo(D)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1336 |
\ subcpo(mkcpo(D,P),D)"; |
| 1623 | 1337 |
brr(subcpoI::subsetI::prems) 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1338 |
by (rtac rel_mkcpo 2); |
| 1623 | 1339 |
by (REPEAT(etac mkcpoD1 1)); |
1340 |
brr(mkcpoI::(cpo_lub RS islub_in)::chain_mkcpo::prems) 1; |
|
| 3425 | 1341 |
qed "subcpo_mkcpo"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1342 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1343 |
(*----------------------------------------------------------------------*) |
| 1461 | 1344 |
(* Embedding projection chains of cpos. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1345 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1346 |
|
| 5136 | 1347 |
val prems = Goalw [emb_chain_def] (* emb_chainI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1348 |
"[|!!n. n:nat ==> cpo(DD`n); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1349 |
\ !!n. n:nat ==> emb(DD`n,DD`succ(n),ee`n)|] ==> emb_chain(DD,ee)"; |
| 4152 | 1350 |
by Safe_tac; |
| 5136 | 1351 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 1352 |
qed "emb_chainI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1353 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1354 |
val emb_chain_cpo = prove_goalw Limit.thy [emb_chain_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1355 |
"!!x. [|emb_chain(DD,ee); n:nat|] ==> cpo(DD`n)" |
| 2469 | 1356 |
(fn prems => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1357 |
|
| 6153 | 1358 |
AddTCs [emb_chain_cpo]; |
1359 |
||
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1360 |
val emb_chain_emb = prove_goalw Limit.thy [emb_chain_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1361 |
"!!x. [|emb_chain(DD,ee); n:nat|] ==> emb(DD`n,DD`succ(n),ee`n)" |
| 2469 | 1362 |
(fn prems => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1363 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1364 |
(*----------------------------------------------------------------------*) |
| 1461 | 1365 |
(* Dinf, the inverse Limit. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1366 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1367 |
|
| 5136 | 1368 |
val prems = Goalw [Dinf_def] (* DinfI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1369 |
"[|x:(PROD n:nat. set(DD`n)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1370 |
\ !!n. n:nat ==> Rp(DD`n,DD`succ(n),ee`n)`(x`succ(n)) = x`n|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1371 |
\ x:set(Dinf(DD,ee))"; |
| 1623 | 1372 |
brr(mkcpoI::iprodI::ballI::prems) 1; |
| 3425 | 1373 |
qed "DinfI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1374 |
|
| 5136 | 1375 |
Goalw [Dinf_def] "x:set(Dinf(DD,ee)) ==> x:(PROD n:nat. set(DD`n))"; |
1376 |
by (etac (mkcpoD1 RS iprodE) 1); |
|
1377 |
qed "Dinf_prod"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1378 |
|
| 5136 | 1379 |
Goalw [Dinf_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1380 |
"[|x:set(Dinf(DD,ee)); n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1381 |
\ Rp(DD`n,DD`succ(n),ee`n)`(x`succ(n)) = x`n"; |
| 5136 | 1382 |
by (blast_tac (claset() addDs [mkcpoD2]) 1); |
1383 |
qed "Dinf_eq"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1384 |
|
| 5136 | 1385 |
val prems = Goalw [Dinf_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1386 |
"[|!!n. n:nat ==> rel(DD`n,x`n,y`n); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1387 |
\ x:(PROD n:nat. set(DD`n)); y:(PROD n:nat. set(DD`n))|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1388 |
\ rel(Dinf(DD,ee),x,y)"; |
| 1623 | 1389 |
by (rtac (rel_mkcpo RS iffD2) 1); |
1390 |
brr(rel_iprodI::iprodI::prems) 1; |
|
| 3425 | 1391 |
qed "rel_DinfI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1392 |
|
| 5136 | 1393 |
Goalw [Dinf_def] "[|rel(Dinf(DD,ee),x,y); n:nat|] ==> rel(DD`n,x`n,y`n)"; |
1394 |
by (etac (rel_mkcpoE RS rel_iprodE) 1); |
|
1395 |
by (assume_tac 1); |
|
| 3425 | 1396 |
qed "rel_Dinf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1397 |
|
| 5136 | 1398 |
Goalw [Dinf_def] "chain(Dinf(DD,ee),X) ==> chain(iprod(DD),X)"; |
1399 |
by (etac chain_mkcpo 1); |
|
1400 |
qed "chain_Dinf"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1401 |
|
| 5136 | 1402 |
Goalw [Dinf_def] (* subcpo_Dinf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1403 |
"emb_chain(DD,ee) ==> subcpo(Dinf(DD,ee),iprod(DD))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1404 |
by (rtac subcpo_mkcpo 1); |
| 1623 | 1405 |
by (fold_tac [Dinf_def]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1406 |
by (rtac ballI 1); |
| 2034 | 1407 |
by (stac lub_iprod 1); |
| 5136 | 1408 |
brr[chain_Dinf, emb_chain_cpo] 1; |
| 2469 | 1409 |
by (Asm_simp_tac 1); |
| 2034 | 1410 |
by (stac (Rp_cont RS cont_lub) 1); |
| 5136 | 1411 |
brr[emb_chain_cpo,emb_chain_emb,nat_succI,chain_iprod,chain_Dinf] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1412 |
(* Useful simplification, ugly in HOL. *) |
| 5136 | 1413 |
by (asm_simp_tac(simpset() addsimps[Dinf_eq,chain_in]) 1); |
1414 |
by (auto_tac (claset() addIs [cpo_iprod,emb_chain_cpo], simpset())); |
|
| 3425 | 1415 |
qed "subcpo_Dinf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1416 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1417 |
(* Simple example of existential reasoning in Isabelle versus HOL. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1418 |
|
| 5136 | 1419 |
Goal "emb_chain(DD,ee) ==> cpo(Dinf(DD,ee))"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1420 |
by (rtac subcpo_cpo 1); |
| 6163 | 1421 |
by (etac subcpo_Dinf 1); |
| 6158 | 1422 |
by (auto_tac (claset() addIs [cpo_iprod, emb_chain_cpo], simpset())); |
| 3425 | 1423 |
qed "cpo_Dinf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1424 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1425 |
(* Again and again the proofs are much easier to WRITE in Isabelle, but |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1426 |
the proof steps are essentially the same (I think). *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1427 |
|
| 5136 | 1428 |
Goal (* lub_Dinf *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1429 |
"[|chain(Dinf(DD,ee),X); emb_chain(DD,ee)|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1430 |
\ lub(Dinf(DD,ee),X) = (lam n:nat. lub(DD`n,lam m:nat. X`m`n))"; |
| 2034 | 1431 |
by (stac (subcpo_Dinf RS lub_subcpo) 1); |
| 5136 | 1432 |
by (auto_tac (claset() addIs [cpo_iprod,emb_chain_cpo,lub_iprod,chain_Dinf], simpset())); |
| 3425 | 1433 |
qed "lub_Dinf"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1434 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1435 |
(*----------------------------------------------------------------------*) |
| 1461 | 1436 |
(* Generalising embedddings D_m -> D_{m+1} to embeddings D_m -> D_n, *)
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1437 |
(* defined as eps(DD,ee,m,n), via e_less and e_gr. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1438 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1439 |
|
| 5136 | 1440 |
Goalw [e_less_def] (* e_less_eq *) |
1441 |
"m:nat ==> e_less(DD,ee,m,m) = id(set(DD`m))"; |
|
| 4091 | 1442 |
by (asm_simp_tac (simpset() addsimps[diff_self_eq_0]) 1); |
| 3425 | 1443 |
qed "e_less_eq"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1444 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1445 |
(* ARITH_CONV proves the following in HOL. Would like something similar |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1446 |
in Isabelle/ZF. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1447 |
|
| 5136 | 1448 |
Goal "[|n:nat; m:nat|] ==> succ(m#+n)#-m = succ(n)"; |
| 1614 | 1449 |
(*Uses add_succ_right the wrong way round!*) |
| 2469 | 1450 |
by (asm_simp_tac |
| 4091 | 1451 |
(simpset_of Nat.thy addsimps [add_succ_right RS sym, diff_add_inverse]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1452 |
val lemma_succ_sub = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1453 |
|
| 5136 | 1454 |
Goalw [e_less_def] (* e_less_add *) |
1455 |
"[|m:nat; k:nat|] ==> \ |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1456 |
\ e_less(DD,ee,m,succ(m#+k)) = (ee`(m#+k))O(e_less(DD,ee,m,m#+k))"; |
| 4091 | 1457 |
by (asm_simp_tac (simpset() addsimps [lemma_succ_sub,diff_add_inverse]) 1); |
| 3425 | 1458 |
qed "e_less_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1459 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1460 |
(* Again, would like more theorems about arithmetic. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1461 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1462 |
val add1 = prove_goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1463 |
"!!x. n:nat ==> succ(n) = n #+ 1" |
| 6070 | 1464 |
(fn prems => [Asm_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1465 |
|
| 5136 | 1466 |
Goal (* succ_sub1 *) |
|
5514
324e1560a5c9
inserted space in #-1 to prevent confusion with an integer constant
paulson
parents:
5268
diff
changeset
|
1467 |
"x:nat ==> 0 < x --> succ(x #- 1)=x"; |
| 6070 | 1468 |
by (induct_tac "x" 1); |
1469 |
by Auto_tac; |
|
| 3425 | 1470 |
qed "succ_sub1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1471 |
|
| 5136 | 1472 |
Goal (* succ_le_pos *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1473 |
"[|m:nat; k:nat|] ==> succ(m) le m #+ k --> 0 < k"; |
| 6070 | 1474 |
by (induct_tac "m" 1); |
1475 |
by Auto_tac; |
|
| 3425 | 1476 |
qed "succ_le_pos"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1477 |
|
| 5136 | 1478 |
Goal "[|n:nat; m:nat|] ==> m le n --> (EX k:nat. n = m #+ k)"; |
| 6070 | 1479 |
by (induct_tac "m" 1); |
| 4152 | 1480 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1481 |
by (rtac bexI 1); |
| 1623 | 1482 |
by (rtac (add_0 RS sym) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1483 |
by (assume_tac 1); |
| 2469 | 1484 |
by (Asm_full_simp_tac 1); |
1485 |
(* Great, by luck I found le_cs. Such cs's and ss's should be documented. *) |
|
1486 |
by (fast_tac le_cs 1); |
|
1487 |
by (asm_simp_tac |
|
| 4091 | 1488 |
(simpset_of Nat.thy addsimps[add_succ, add_succ_right RS sym]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1489 |
by (rtac bexI 1); |
| 2034 | 1490 |
by (stac (succ_sub1 RS mp) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1491 |
(* Instantiation. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1492 |
by (rtac refl 3); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1493 |
by (assume_tac 1); |
| 1623 | 1494 |
by (rtac (succ_le_pos RS mp) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1495 |
by (assume_tac 3); (* Instantiation *) |
| 5136 | 1496 |
by (ALLGOALS Asm_simp_tac); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1497 |
val lemma_le_exists = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1498 |
|
| 5136 | 1499 |
val prems = goal thy (* le_exists *) |
| 2469 | 1500 |
"[|m le n; !!x. [|n=m#+x; x:nat|] ==> Q; m:nat; n:nat|] ==> Q"; |
| 1623 | 1501 |
by (rtac (lemma_le_exists RS mp RS bexE) 1); |
| 5136 | 1502 |
by (DEPTH_SOLVE (ares_tac prems 1)); |
| 3425 | 1503 |
qed "le_exists"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1504 |
|
| 5136 | 1505 |
Goal (* e_less_le *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1506 |
"[|m le n; m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1507 |
\ e_less(DD,ee,m,succ(n)) = ee`n O e_less(DD,ee,m,n)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1508 |
by (rtac le_exists 1); |
| 5136 | 1509 |
by (assume_tac 1); |
1510 |
by (asm_simp_tac(simpset() addsimps[e_less_add]) 1); |
|
1511 |
by (REPEAT (assume_tac 1)); |
|
| 3425 | 1512 |
qed "e_less_le"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1513 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1514 |
(* All theorems assume variables m and n are natural numbers. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1515 |
|
| 5136 | 1516 |
Goal "m:nat ==> e_less(DD,ee,m,succ(m)) = ee`m O id(set(DD`m))"; |
|
8127
68c6159440f1
new lemmas for Ntree recursor example; more simprules; more lemmas borrowed
paulson
parents:
6176
diff
changeset
|
1517 |
by (asm_simp_tac(simpset() addsimps[e_less_le, e_less_eq]) 1); |
| 3425 | 1518 |
qed "e_less_succ"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1519 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1520 |
val prems = goal Limit.thy (* e_less_succ_emb *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1521 |
"[|!!n. n:nat ==> emb(DD`n,DD`succ(n),ee`n); m:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1522 |
\ e_less(DD,ee,m,succ(m)) = ee`m"; |
| 5529 | 1523 |
by (asm_simp_tac(simpset() addsimps e_less_succ::prems) 1); |
| 2034 | 1524 |
by (stac comp_id 1); |
| 1623 | 1525 |
brr(emb_cont::cont_fun::refl::prems) 1; |
| 3425 | 1526 |
qed "e_less_succ_emb"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1527 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1528 |
(* Compare this proof with the HOL one, here we do type checking. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1529 |
(* In any case the one below was very easy to write. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1530 |
|
| 5136 | 1531 |
Goal "[|emb_chain(DD,ee); m:nat; k:nat|] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1532 |
\ emb(DD`m,DD`(m#+k),e_less(DD,ee,m,m#+k))"; |
| 6070 | 1533 |
by (induct_tac "k" 1); |
1534 |
by (asm_simp_tac(simpset() addsimps[e_less_eq]) 1); |
|
| 5136 | 1535 |
brr[emb_id,emb_chain_cpo] 1; |
| 6070 | 1536 |
by (asm_simp_tac(simpset() addsimps[e_less_add]) 1); |
| 5136 | 1537 |
by (auto_tac (claset() addIs [emb_comp,emb_chain_emb,emb_chain_cpo,add_type], |
1538 |
simpset())); |
|
| 3425 | 1539 |
qed "emb_e_less_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1540 |
|
| 5136 | 1541 |
Goal "[|m le n; emb_chain(DD,ee); m:nat; n:nat|] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1542 |
\ emb(DD`m,DD`n,e_less(DD,ee,m,n))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1543 |
(* same proof as e_less_le *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1544 |
by (rtac le_exists 1); |
| 5136 | 1545 |
by (assume_tac 1); |
1546 |
by (asm_simp_tac(simpset() addsimps[emb_e_less_add]) 1); |
|
1547 |
by (REPEAT (assume_tac 1)); |
|
| 3425 | 1548 |
qed "emb_e_less"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1549 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1550 |
val comp_mono_eq = prove_goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1551 |
"!!z.[|f=f'; g=g'|] ==> f O g = f' O g'" |
| 2469 | 1552 |
(fn prems => [Asm_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1553 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1554 |
(* Typing, typing, typing, three irritating assumptions. Extra theorems |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1555 |
needed in proof, but no real difficulty. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1556 |
(* Note also the object-level implication for induction on k. This |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1557 |
must be removed later to allow the theorems to be used for simp. |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1558 |
Therefore this theorem is only a lemma. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1559 |
|
| 5136 | 1560 |
Goal (* e_less_split_add_lemma *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1561 |
"[| emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1562 |
\ n le k --> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1563 |
\ e_less(DD,ee,m,m#+k) = e_less(DD,ee,m#+n,m#+k) O e_less(DD,ee,m,m#+n)"; |
| 6070 | 1564 |
by (induct_tac "k" 1); |
| 5136 | 1565 |
by (asm_full_simp_tac(simpset() addsimps [e_less_eq, id_type RS id_comp]) 1); |
| 1623 | 1566 |
by (asm_simp_tac(ZF_ss addsimps[le_succ_iff]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1567 |
by (rtac impI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1568 |
by (etac disjE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1569 |
by (etac impE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1570 |
by (assume_tac 1); |
| 5136 | 1571 |
by (asm_simp_tac(ZF_ss addsimps[add_succ_right, e_less_add, add_type,nat_succI]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1572 |
(* Again and again, simplification is a pain. When does it work, when not? *) |
| 2034 | 1573 |
by (stac e_less_le 1); |
| 5136 | 1574 |
brr[add_le_mono,nat_le_refl,add_type,nat_succI] 1; |
| 2034 | 1575 |
by (stac comp_assoc 1); |
| 5136 | 1576 |
brr[comp_mono_eq,refl] 1; |
1577 |
by (asm_simp_tac(ZF_ss addsimps[e_less_eq,add_type,nat_succI]) 1); |
|
| 2034 | 1578 |
by (stac id_comp 1); (* simp cannot unify/inst right, use brr below(?). *) |
| 5136 | 1579 |
by (REPEAT (ares_tac [emb_e_less_add RS emb_cont RS cont_fun, refl, |
1580 |
nat_succI] 1)); |
|
| 3425 | 1581 |
qed "e_less_split_add_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1582 |
|
| 5136 | 1583 |
Goal "[| n le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
1584 |
\ e_less(DD,ee,m,m#+k) = e_less(DD,ee,m#+n,m#+k) O e_less(DD,ee,m,m#+n)"; |
|
1585 |
by (blast_tac (claset() addIs [e_less_split_add_lemma RS mp]) 1); |
|
1586 |
qed "e_less_split_add"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1587 |
|
| 5136 | 1588 |
Goalw [e_gr_def] (* e_gr_eq *) |
1589 |
"m:nat ==> e_gr(DD,ee,m,m) = id(set(DD`m))"; |
|
| 4091 | 1590 |
by (asm_simp_tac (simpset() addsimps[diff_self_eq_0]) 1); |
| 3425 | 1591 |
qed "e_gr_eq"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1592 |
|
| 5136 | 1593 |
Goalw [e_gr_def] (* e_gr_add *) |
1594 |
"[|n:nat; k:nat|] ==> \ |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1595 |
\ e_gr(DD,ee,succ(n#+k),n) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1596 |
\ e_gr(DD,ee,n#+k,n) O Rp(DD`(n#+k),DD`succ(n#+k),ee`(n#+k))"; |
| 4091 | 1597 |
by (asm_simp_tac (simpset() addsimps [lemma_succ_sub,diff_add_inverse]) 1); |
| 3425 | 1598 |
qed "e_gr_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1599 |
|
| 5136 | 1600 |
Goal "[|n le m; m:nat; n:nat|] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1601 |
\ e_gr(DD,ee,succ(m),n) = e_gr(DD,ee,m,n) O Rp(DD`m,DD`succ(m),ee`m)"; |
| 5136 | 1602 |
by (etac le_exists 1); |
1603 |
by (asm_simp_tac(simpset() addsimps[e_gr_add]) 1); |
|
1604 |
by (REPEAT (assume_tac 1)); |
|
| 3425 | 1605 |
qed "e_gr_le"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1606 |
|
| 5136 | 1607 |
Goal "m:nat ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1608 |
\ e_gr(DD,ee,succ(m),m) = id(set(DD`m)) O Rp(DD`m,DD`succ(m),ee`m)"; |
| 5136 | 1609 |
by (asm_simp_tac(simpset() addsimps[e_gr_le,e_gr_eq]) 1); |
| 3425 | 1610 |
qed "e_gr_succ"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1611 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1612 |
(* Cpo asm's due to THE uniqueness. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1613 |
|
| 5136 | 1614 |
Goal "[|emb_chain(DD,ee); m:nat|] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1615 |
\ e_gr(DD,ee,succ(m),m) = Rp(DD`m,DD`succ(m),ee`m)"; |
| 5136 | 1616 |
by (asm_simp_tac(simpset() addsimps[e_gr_succ]) 1); |
1617 |
by (blast_tac (claset() addIs [id_comp, Rp_cont,cont_fun, |
|
1618 |
emb_chain_cpo,emb_chain_emb]) 1); |
|
| 3425 | 1619 |
qed "e_gr_succ_emb"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1620 |
|
| 5136 | 1621 |
Goal (* e_gr_fun_add *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1622 |
"[|emb_chain(DD,ee); n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1623 |
\ e_gr(DD,ee,n#+k,n): set(DD`(n#+k))->set(DD`n)"; |
| 6070 | 1624 |
by (induct_tac "k" 1); |
1625 |
by (asm_simp_tac(simpset() addsimps[e_gr_eq,id_type]) 1); |
|
1626 |
by (asm_simp_tac(simpset() addsimps[e_gr_add]) 1); |
|
| 5136 | 1627 |
brr[comp_fun, Rp_cont, cont_fun, emb_chain_emb, emb_chain_cpo, add_type, nat_succI] 1; |
| 3425 | 1628 |
qed "e_gr_fun_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1629 |
|
| 5136 | 1630 |
Goal (* e_gr_fun *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1631 |
"[|n le m; emb_chain(DD,ee); m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1632 |
\ e_gr(DD,ee,m,n): set(DD`m)->set(DD`n)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1633 |
by (rtac le_exists 1); |
| 5136 | 1634 |
by (assume_tac 1); |
1635 |
by (asm_simp_tac(simpset() addsimps[e_gr_fun_add]) 1); |
|
1636 |
by (REPEAT (assume_tac 1)); |
|
| 3425 | 1637 |
qed "e_gr_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1638 |
|
| 5136 | 1639 |
Goal (* e_gr_split_add_lemma *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1640 |
"[| emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1641 |
\ m le k --> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1642 |
\ e_gr(DD,ee,n#+k,n) = e_gr(DD,ee,n#+m,n) O e_gr(DD,ee,n#+k,n#+m)"; |
| 6070 | 1643 |
by (induct_tac "k" 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1644 |
by (rtac impI 1); |
| 6070 | 1645 |
by (asm_full_simp_tac(simpset() addsimps |
1646 |
[le0_iff, e_gr_eq, id_type RS comp_id]) 1); |
|
| 1623 | 1647 |
by (asm_simp_tac(ZF_ss addsimps[le_succ_iff]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1648 |
by (rtac impI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1649 |
by (etac disjE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1650 |
by (etac impE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1651 |
by (assume_tac 1); |
| 5136 | 1652 |
by (asm_simp_tac(ZF_ss addsimps[add_succ_right, e_gr_add, add_type,nat_succI]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1653 |
(* Again and again, simplification is a pain. When does it work, when not? *) |
| 2034 | 1654 |
by (stac e_gr_le 1); |
| 5136 | 1655 |
brr[add_le_mono,nat_le_refl,add_type,nat_succI] 1; |
| 2034 | 1656 |
by (stac comp_assoc 1); |
| 5136 | 1657 |
brr[comp_mono_eq,refl] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1658 |
(* New direct subgoal *) |
| 5136 | 1659 |
by (asm_simp_tac(ZF_ss addsimps[e_gr_eq,add_type,nat_succI]) 1); |
| 2034 | 1660 |
by (stac comp_id 1); (* simp cannot unify/inst right, use brr below(?). *) |
| 5136 | 1661 |
by (REPEAT (ares_tac [e_gr_fun,add_type,refl,add_le_self,nat_succI] 1)); |
| 3425 | 1662 |
qed "e_gr_split_add_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1663 |
|
| 5136 | 1664 |
Goal "[| m le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
1665 |
\ e_gr(DD,ee,n#+k,n) = e_gr(DD,ee,n#+m,n) O e_gr(DD,ee,n#+k,n#+m)"; |
|
1666 |
by (blast_tac (claset() addIs [e_gr_split_add_lemma RS mp]) 1); |
|
1667 |
qed "e_gr_split_add"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1668 |
|
| 5136 | 1669 |
Goal "[|m le n; emb_chain(DD,ee); m:nat; n:nat|] ==> \ |
1670 |
\ e_less(DD,ee,m,n):cont(DD`m,DD`n)"; |
|
1671 |
by (blast_tac (claset() addIs [emb_cont, emb_e_less]) 1); |
|
1672 |
qed "e_less_cont"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1673 |
|
| 6070 | 1674 |
Goal (* e_gr_cont *) |
1675 |
"[|n le m; emb_chain(DD,ee); m:nat; n:nat|] ==> \ |
|
1676 |
\ e_gr(DD,ee,m,n):cont(DD`m,DD`n)"; |
|
1677 |
by (etac rev_mp 1); |
|
1678 |
by (induct_tac "m" 1); |
|
1679 |
by (asm_full_simp_tac(simpset() addsimps [le0_iff,e_gr_eq,nat_0I]) 1); |
|
| 5136 | 1680 |
brr[impI,id_cont,emb_chain_cpo,nat_0I] 1; |
| 4091 | 1681 |
by (asm_full_simp_tac(simpset() addsimps[le_succ_iff]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1682 |
by (etac disjE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1683 |
by (etac impE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1684 |
by (assume_tac 1); |
| 5136 | 1685 |
by (asm_simp_tac(simpset() addsimps[e_gr_le]) 1); |
1686 |
brr[comp_pres_cont,Rp_cont,emb_chain_cpo,emb_chain_emb,nat_succI] 1; |
|
1687 |
by (asm_simp_tac(simpset() addsimps[e_gr_eq,nat_succI]) 1); |
|
1688 |
by (auto_tac (claset() addIs [id_cont,emb_chain_cpo], simpset())); |
|
| 3425 | 1689 |
qed "e_gr_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1690 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1691 |
(* Considerably shorter.... 57 against 26 *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1692 |
|
| 5136 | 1693 |
Goal (* e_less_e_gr_split_add *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1694 |
"[|n le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1695 |
\ e_less(DD,ee,m,m#+n) = e_gr(DD,ee,m#+k,m#+n) O e_less(DD,ee,m,m#+k)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1696 |
(* Use mp to prepare for induction. *) |
| 6070 | 1697 |
by (etac rev_mp 1); |
1698 |
by (induct_tac "k" 1); |
|
1699 |
by (asm_full_simp_tac(simpset() addsimps |
|
1700 |
[e_gr_eq, e_less_eq, id_type RS id_comp]) 1); |
|
1701 |
by (simp_tac(ZF_ss addsimps[le_succ_iff]) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1702 |
by (rtac impI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1703 |
by (etac disjE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1704 |
by (etac impE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1705 |
by (assume_tac 1); |
| 5136 | 1706 |
by (asm_simp_tac(ZF_ss addsimps[add_succ_right, e_gr_le, e_less_le, add_le_self,nat_le_refl,add_le_mono,add_type]) 1); |
| 2034 | 1707 |
by (stac comp_assoc 1); |
| 1623 | 1708 |
by (res_inst_tac[("s1","ee`(m#+x)")](comp_assoc RS subst) 1);
|
| 2034 | 1709 |
by (stac embRp_eq 1); |
| 5136 | 1710 |
brr[emb_chain_emb,add_type,emb_chain_cpo,nat_succI] 1; |
| 2034 | 1711 |
by (stac id_comp 1); |
| 5136 | 1712 |
brr[e_less_cont RS cont_fun, add_type,add_le_self,refl] 1; |
1713 |
by (asm_full_simp_tac(ZF_ss addsimps[e_gr_eq,nat_succI,add_type]) 1); |
|
| 2034 | 1714 |
by (stac id_comp 1); |
| 5136 | 1715 |
by (REPEAT (ares_tac [e_less_cont RS cont_fun, add_type, |
1716 |
nat_succI,add_le_self,refl] 1)); |
|
| 3425 | 1717 |
qed "e_less_e_gr_split_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1718 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1719 |
(* Again considerably shorter, and easy to obtain from the previous thm. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1720 |
|
| 5136 | 1721 |
Goal (* e_gr_e_less_split_add *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1722 |
"[|m le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1723 |
\ e_gr(DD,ee,n#+m,n) = e_gr(DD,ee,n#+k,n) O e_less(DD,ee,n#+m,n#+k)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1724 |
(* Use mp to prepare for induction. *) |
| 6070 | 1725 |
by (etac rev_mp 1); |
1726 |
by (induct_tac "k" 1); |
|
| 4091 | 1727 |
by (asm_full_simp_tac(simpset() addsimps |
| 6070 | 1728 |
[e_gr_eq, e_less_eq, id_type RS id_comp]) 1); |
| 1623 | 1729 |
by (simp_tac(ZF_ss addsimps[le_succ_iff]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1730 |
by (rtac impI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1731 |
by (etac disjE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1732 |
by (etac impE 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1733 |
by (assume_tac 1); |
| 5136 | 1734 |
by (asm_simp_tac(ZF_ss addsimps[add_succ_right, e_gr_le, e_less_le, add_le_self,nat_le_refl,add_le_mono,add_type]) 1); |
| 2034 | 1735 |
by (stac comp_assoc 1); |
| 1623 | 1736 |
by (res_inst_tac[("s1","ee`(n#+x)")](comp_assoc RS subst) 1);
|
| 2034 | 1737 |
by (stac embRp_eq 1); |
| 5136 | 1738 |
brr[emb_chain_emb,add_type,emb_chain_cpo,nat_succI] 1; |
| 2034 | 1739 |
by (stac id_comp 1); |
| 5136 | 1740 |
brr[e_less_cont RS cont_fun, add_type, add_le_mono, nat_le_refl, refl] 1; |
1741 |
by (asm_full_simp_tac(ZF_ss addsimps[e_less_eq,nat_succI,add_type]) 1); |
|
| 2034 | 1742 |
by (stac comp_id 1); |
| 5136 | 1743 |
by (REPEAT (ares_tac [e_gr_cont RS cont_fun, add_type,nat_succI,add_le_self, |
1744 |
refl] 1)); |
|
| 3425 | 1745 |
qed "e_gr_e_less_split_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1746 |
|
| 2469 | 1747 |
|
| 5136 | 1748 |
Goalw [eps_def] (* emb_eps *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1749 |
"[|m le n; emb_chain(DD,ee); m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1750 |
\ emb(DD`m,DD`n,eps(DD,ee,m,n))"; |
| 5136 | 1751 |
by (asm_simp_tac(simpset()) 1); |
1752 |
brr[emb_e_less] 1; |
|
| 3425 | 1753 |
qed "emb_eps"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1754 |
|
| 5136 | 1755 |
Goalw [eps_def] (* eps_fun *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1756 |
"[|emb_chain(DD,ee); m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1757 |
\ eps(DD,ee,m,n): set(DD`m)->set(DD`n)"; |
|
5116
8eb343ab5748
Renamed expand_if to split_if and setloop split_tac to addsplits,
paulson
parents:
5068
diff
changeset
|
1758 |
by (rtac (split_if RS iffD2) 1); |
| 4152 | 1759 |
by Safe_tac; |
| 5136 | 1760 |
brr[e_less_cont RS cont_fun] 1; |
1761 |
by (auto_tac (claset() addIs [not_le_iff_lt RS iffD1 RS leI, e_gr_fun,nat_into_Ord], simpset())); |
|
| 3425 | 1762 |
qed "eps_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1763 |
|
| 5136 | 1764 |
Goalw [eps_def] "n:nat ==> eps(DD,ee,n,n) = id(set(DD`n))"; |
1765 |
by (asm_simp_tac(simpset() addsimps [e_less_eq]) 1); |
|
1766 |
qed "eps_id"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1767 |
|
| 5136 | 1768 |
Goalw [eps_def] |
1769 |
"[|m:nat; n:nat|] ==> eps(DD,ee,m,m#+n) = e_less(DD,ee,m,m#+n)"; |
|
1770 |
by (asm_simp_tac(simpset() addsimps [add_le_self]) 1); |
|
1771 |
qed "eps_e_less_add"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1772 |
|
| 5136 | 1773 |
Goalw [eps_def] |
1774 |
"[|m le n; m:nat; n:nat|] ==> eps(DD,ee,m,n) = e_less(DD,ee,m,n)"; |
|
1775 |
by (Asm_simp_tac 1); |
|
1776 |
qed "eps_e_less"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1777 |
|
| 5136 | 1778 |
Goalw [eps_def] (* eps_e_gr_add *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1779 |
"[|n:nat; k:nat|] ==> eps(DD,ee,n#+k,n) = e_gr(DD,ee,n#+k,n)"; |
|
5116
8eb343ab5748
Renamed expand_if to split_if and setloop split_tac to addsplits,
paulson
parents:
5068
diff
changeset
|
1780 |
by (rtac (split_if RS iffD2) 1); |
| 4152 | 1781 |
by Safe_tac; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1782 |
by (etac leE 1); |
| 5136 | 1783 |
by (asm_simp_tac(simpset() addsimps[e_less_eq,e_gr_eq]) 2); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1784 |
(* Must control rewriting by instantiating a variable. *) |
| 4091 | 1785 |
by (asm_full_simp_tac(simpset() addsimps |
| 5136 | 1786 |
[read_instantiate [("i1","n")] (nat_into_Ord RS not_le_iff_lt RS iff_sym),
|
1787 |
add_le_self]) 1); |
|
| 3425 | 1788 |
qed "eps_e_gr_add"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1789 |
|
| 5136 | 1790 |
Goal (* eps_e_gr *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1791 |
"[|n le m; m:nat; n:nat|] ==> eps(DD,ee,m,n) = e_gr(DD,ee,m,n)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1792 |
by (rtac le_exists 1); |
| 5136 | 1793 |
by (assume_tac 1); |
1794 |
by (asm_simp_tac(simpset() addsimps[eps_e_gr_add]) 1); |
|
1795 |
by (REPEAT (assume_tac 1)); |
|
| 3425 | 1796 |
qed "eps_e_gr"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1797 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1798 |
val prems = goal Limit.thy (* eps_succ_ee *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1799 |
"[|!!n. n:nat ==> emb(DD`n,DD`succ(n),ee`n); m:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1800 |
\ eps(DD,ee,m,succ(m)) = ee`m"; |
| 5529 | 1801 |
by (asm_simp_tac(simpset() addsimps eps_e_less::le_succ_iff::e_less_succ_emb:: |
1802 |
prems) 1); |
|
| 3425 | 1803 |
qed "eps_succ_ee"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1804 |
|
| 5136 | 1805 |
Goal (* eps_succ_Rp *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1806 |
"[|emb_chain(DD,ee); m:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1807 |
\ eps(DD,ee,succ(m),m) = Rp(DD`m,DD`succ(m),ee`m)"; |
| 5529 | 1808 |
by (asm_simp_tac(simpset() addsimps eps_e_gr::le_succ_iff::e_gr_succ_emb:: |
1809 |
prems) 1); |
|
| 3425 | 1810 |
qed "eps_succ_Rp"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1811 |
|
| 5136 | 1812 |
Goal (* eps_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1813 |
"[|emb_chain(DD,ee); m:nat; n:nat|] ==> eps(DD,ee,m,n): cont(DD`m,DD`n)"; |
| 5136 | 1814 |
by (res_inst_tac [("i","m"),("j","n")] nat_linear_le 1);
|
1815 |
by (ALLGOALS (asm_simp_tac(simpset() addsimps [eps_e_less,e_less_cont, |
|
1816 |
eps_e_gr,e_gr_cont]))); |
|
| 3425 | 1817 |
qed "eps_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1818 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1819 |
(* Theorems about splitting. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1820 |
|
| 5136 | 1821 |
Goal (* eps_split_add_left *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1822 |
"[|n le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1823 |
\ eps(DD,ee,m,m#+k) = eps(DD,ee,m#+n,m#+k) O eps(DD,ee,m,m#+n)"; |
| 4091 | 1824 |
by (asm_simp_tac(simpset() addsimps |
| 5136 | 1825 |
[eps_e_less,add_le_self,add_le_mono]) 1); |
1826 |
by (auto_tac (claset() addIs [e_less_split_add], simpset())); |
|
| 3425 | 1827 |
qed "eps_split_add_left"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1828 |
|
| 5136 | 1829 |
Goal (* eps_split_add_left_rev *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1830 |
"[|n le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1831 |
\ eps(DD,ee,m,m#+n) = eps(DD,ee,m#+k,m#+n) O eps(DD,ee,m,m#+k)"; |
| 4091 | 1832 |
by (asm_simp_tac(simpset() addsimps |
| 5136 | 1833 |
[eps_e_less_add,eps_e_gr,add_le_self,add_le_mono]) 1); |
1834 |
by (auto_tac (claset() addIs [e_less_e_gr_split_add], simpset())); |
|
| 3425 | 1835 |
qed "eps_split_add_left_rev"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1836 |
|
| 5136 | 1837 |
Goal (* eps_split_add_right *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1838 |
"[|m le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1839 |
\ eps(DD,ee,n#+k,n) = eps(DD,ee,n#+m,n) O eps(DD,ee,n#+k,n#+m)"; |
| 4091 | 1840 |
by (asm_simp_tac(simpset() addsimps |
| 5136 | 1841 |
[eps_e_gr,add_le_self,add_le_mono]) 1); |
1842 |
by (auto_tac (claset() addIs [e_gr_split_add], simpset())); |
|
| 3425 | 1843 |
qed "eps_split_add_right"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1844 |
|
| 5136 | 1845 |
Goal (* eps_split_add_right_rev *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1846 |
"[|m le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1847 |
\ eps(DD,ee,n#+m,n) = eps(DD,ee,n#+k,n) O eps(DD,ee,n#+m,n#+k)"; |
| 4091 | 1848 |
by (asm_simp_tac(simpset() addsimps |
| 5136 | 1849 |
[eps_e_gr_add,eps_e_less,add_le_self,add_le_mono]) 1); |
1850 |
by (auto_tac (claset() addIs [e_gr_e_less_split_add], simpset())); |
|
| 3425 | 1851 |
qed "eps_split_add_right_rev"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1852 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1853 |
(* Arithmetic, little support in Isabelle/ZF. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1854 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1855 |
val prems = goal Limit.thy (* le_exists_lemma *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1856 |
"[|n le k; k le m; \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1857 |
\ !!p q. [|p le q; k=n#+p; m=n#+q; p:nat; q:nat|] ==> R; \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1858 |
\ m:nat; n:nat; k:nat|]==>R"; |
| 1623 | 1859 |
by (rtac (hd prems RS le_exists) 1); |
1860 |
by (rtac (le_exists) 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1861 |
by (rtac le_trans 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1862 |
(* Careful *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1863 |
by (resolve_tac prems 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1864 |
by (resolve_tac prems 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1865 |
by (resolve_tac prems 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1866 |
by (assume_tac 2); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1867 |
by (assume_tac 2); |
| 1623 | 1868 |
by (cut_facts_tac[hd prems,hd(tl prems)]1); |
| 2469 | 1869 |
by (Asm_full_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1870 |
by (etac add_le_elim1 1); |
| 5136 | 1871 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 1872 |
qed "le_exists_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1873 |
|
| 5136 | 1874 |
Goal (* eps_split_left_le *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1875 |
"[|m le k; k le n; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1876 |
\ eps(DD,ee,m,n) = eps(DD,ee,k,n) O eps(DD,ee,m,k)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1877 |
by (rtac le_exists_lemma 1); |
| 5136 | 1878 |
by (REPEAT (assume_tac 1)); |
| 2469 | 1879 |
by (Asm_simp_tac 1); |
| 5136 | 1880 |
by (auto_tac (claset() addIs [eps_split_add_left], simpset())); |
| 3425 | 1881 |
qed "eps_split_left_le"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1882 |
|
| 5136 | 1883 |
Goal (* eps_split_left_le_rev *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1884 |
"[|m le n; n le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1885 |
\ eps(DD,ee,m,n) = eps(DD,ee,k,n) O eps(DD,ee,m,k)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1886 |
by (rtac le_exists_lemma 1); |
| 5136 | 1887 |
by (REPEAT (assume_tac 1)); |
| 2469 | 1888 |
by (Asm_simp_tac 1); |
| 5136 | 1889 |
by (auto_tac (claset() addIs [eps_split_add_left_rev], simpset())); |
| 3425 | 1890 |
qed "eps_split_left_le_rev"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1891 |
|
| 5136 | 1892 |
Goal (* eps_split_right_le *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1893 |
"[|n le k; k le m; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1894 |
\ eps(DD,ee,m,n) = eps(DD,ee,k,n) O eps(DD,ee,m,k)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1895 |
by (rtac le_exists_lemma 1); |
| 5136 | 1896 |
by (REPEAT (assume_tac 1)); |
| 2469 | 1897 |
by (Asm_simp_tac 1); |
| 5136 | 1898 |
by (auto_tac (claset() addIs [eps_split_add_right], simpset())); |
| 3425 | 1899 |
qed "eps_split_right_le"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1900 |
|
| 5136 | 1901 |
Goal (* eps_split_right_le_rev *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1902 |
"[|n le m; m le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1903 |
\ eps(DD,ee,m,n) = eps(DD,ee,k,n) O eps(DD,ee,m,k)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1904 |
by (rtac le_exists_lemma 1); |
| 5136 | 1905 |
by (REPEAT (assume_tac 1)); |
| 2469 | 1906 |
by (Asm_simp_tac 1); |
| 5136 | 1907 |
by (auto_tac (claset() addIs [eps_split_add_right_rev], simpset())); |
| 3425 | 1908 |
qed "eps_split_right_le_rev"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1909 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1910 |
(* The desired two theorems about `splitting'. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1911 |
|
| 5136 | 1912 |
Goal (* eps_split_left *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1913 |
"[|m le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1914 |
\ eps(DD,ee,m,n) = eps(DD,ee,k,n) O eps(DD,ee,m,k)"; |
| 2469 | 1915 |
by (rtac nat_linear_le 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1916 |
by (rtac eps_split_right_le_rev 4); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1917 |
by (assume_tac 4); |
| 2469 | 1918 |
by (rtac nat_linear_le 3); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1919 |
by (rtac eps_split_left_le 5); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1920 |
by (assume_tac 6); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1921 |
by (rtac eps_split_left_le_rev 10); |
| 5136 | 1922 |
by (REPEAT (assume_tac 1)); (* 20 trivial subgoals *) |
| 3425 | 1923 |
qed "eps_split_left"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1924 |
|
| 5136 | 1925 |
Goal (* eps_split_right *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1926 |
"[|n le k; emb_chain(DD,ee); m:nat; n:nat; k:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1927 |
\ eps(DD,ee,m,n) = eps(DD,ee,k,n) O eps(DD,ee,m,k)"; |
| 2469 | 1928 |
by (rtac nat_linear_le 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1929 |
by (rtac eps_split_left_le_rev 3); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1930 |
by (assume_tac 3); |
| 2469 | 1931 |
by (rtac nat_linear_le 8); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1932 |
by (rtac eps_split_right_le 10); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1933 |
by (assume_tac 11); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1934 |
by (rtac eps_split_right_le_rev 15); |
| 5136 | 1935 |
by (REPEAT (assume_tac 1)); (* 20 trivial subgoals *) |
| 3425 | 1936 |
qed "eps_split_right"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1937 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1938 |
(*----------------------------------------------------------------------*) |
| 1461 | 1939 |
(* That was eps: D_m -> D_n, NEXT rho_emb: D_n -> Dinf. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1940 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1941 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1942 |
(* Considerably shorter. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1943 |
|
| 5136 | 1944 |
Goalw [rho_emb_def] (* rho_emb_fun *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1945 |
"[|emb_chain(DD,ee); n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1946 |
\ rho_emb(DD,ee,n): set(DD`n) -> set(Dinf(DD,ee))"; |
| 5136 | 1947 |
brr[lam_type, DinfI, eps_cont RS cont_fun RS apply_type] 1; |
| 2469 | 1948 |
by (Asm_simp_tac 1); |
| 5136 | 1949 |
by (res_inst_tac [("i","succ(na)"),("j","n")] nat_linear_le 1);
|
1950 |
by (Blast_tac 1); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1951 |
by (assume_tac 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1952 |
(* The easiest would be to apply add1 everywhere also in the assumptions, |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1953 |
but since x le y is x<succ(y) simplification does too much with this thm. *) |
| 2034 | 1954 |
by (stac eps_split_right_le 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1955 |
by (assume_tac 2); |
| 6153 | 1956 |
by (asm_simp_tac(FOL_ss addsimps [add1]) 1); |
| 5136 | 1957 |
brr[add_le_self,nat_0I,nat_succI] 1; |
1958 |
by (asm_simp_tac(simpset() addsimps[eps_succ_Rp]) 1); |
|
| 2034 | 1959 |
by (stac comp_fun_apply 1); |
| 5136 | 1960 |
brr[eps_fun, nat_succI, Rp_cont RS cont_fun, emb_chain_emb, emb_chain_cpo,refl] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1961 |
(* Now the second part of the proof. Slightly different than HOL. *) |
| 5136 | 1962 |
by (asm_simp_tac(simpset() addsimps[eps_e_less,nat_succI]) 1); |
| 1623 | 1963 |
by (etac (le_iff RS iffD1 RS disjE) 1); |
| 5136 | 1964 |
by (asm_simp_tac(simpset() addsimps[e_less_le]) 1); |
| 2034 | 1965 |
by (stac comp_fun_apply 1); |
| 5136 | 1966 |
brr[e_less_cont,cont_fun,emb_chain_emb,emb_cont] 1; |
| 2034 | 1967 |
by (stac embRp_eq_thm 1); |
| 5136 | 1968 |
brr[emb_chain_emb, e_less_cont RS cont_fun RS apply_type, emb_chain_cpo, nat_succI] 1; |
1969 |
by (asm_simp_tac(simpset() addsimps[eps_e_less]) 1); |
|
1970 |
by (dtac asm_rl 1); |
|
1971 |
by (asm_full_simp_tac(simpset() addsimps[eps_succ_Rp, e_less_eq, id_apply, nat_succI]) 1); |
|
| 3425 | 1972 |
qed "rho_emb_fun"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1973 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1974 |
val rho_emb_apply1 = prove_goalw Limit.thy [rho_emb_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1975 |
"!!z. x:set(DD`n) ==> rho_emb(DD,ee,n)`x = (lam m:nat. eps(DD,ee,n,m)`x)" |
| 2469 | 1976 |
(fn prems => [Asm_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1977 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1978 |
val rho_emb_apply2 = prove_goalw Limit.thy [rho_emb_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1979 |
"!!z. [|x:set(DD`n); m:nat|] ==> rho_emb(DD,ee,n)`x`m = eps(DD,ee,n,m)`x" |
| 2469 | 1980 |
(fn prems => [Asm_simp_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1981 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1982 |
val rho_emb_id = prove_goal Limit.thy |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1983 |
"!!z. [| x:set(DD`n); n:nat|] ==> rho_emb(DD,ee,n)`x`n = x" |
| 6169 | 1984 |
(fn prems => [asm_simp_tac(simpset() addsimps[rho_emb_apply2,eps_id]) 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1985 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1986 |
(* Shorter proof, 23 against 62. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1987 |
|
| 5136 | 1988 |
Goal (* rho_emb_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1989 |
"[|emb_chain(DD,ee); n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1990 |
\ rho_emb(DD,ee,n): cont(DD`n,Dinf(DD,ee))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1991 |
by (rtac contI 1); |
| 5136 | 1992 |
brr[rho_emb_fun] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1993 |
by (rtac rel_DinfI 1); |
| 1623 | 1994 |
by (SELECT_GOAL(rewtac rho_emb_def) 1); |
| 2469 | 1995 |
by (Asm_simp_tac 1); |
| 5136 | 1996 |
brr[eps_cont RS cont_mono, Dinf_prod,apply_type,rho_emb_fun] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1997 |
(* Continuity, different order, slightly different proofs. *) |
| 2034 | 1998 |
by (stac lub_Dinf 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
1999 |
by (rtac chainI 1); |
| 5136 | 2000 |
brr[lam_type, rho_emb_fun RS apply_type, chain_in] 1; |
| 2469 | 2001 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2002 |
by (rtac rel_DinfI 1); |
| 5136 | 2003 |
by (asm_simp_tac(simpset() addsimps [rho_emb_apply2,chain_in]) 1); |
2004 |
brr[eps_cont RS cont_mono, chain_rel, Dinf_prod, rho_emb_fun RS apply_type, chain_in,nat_succI] 1; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2005 |
(* Now, back to the result of applying lub_Dinf *) |
| 5136 | 2006 |
by (asm_simp_tac(simpset() addsimps [rho_emb_apply2,chain_in]) 1); |
| 2034 | 2007 |
by (stac rho_emb_apply1 1); |
| 5136 | 2008 |
brr[cpo_lub RS islub_in, emb_chain_cpo] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2009 |
by (rtac fun_extension 1); |
| 5136 | 2010 |
brr[lam_type, eps_cont RS cont_fun RS apply_type, cpo_lub RS islub_in, emb_chain_cpo] 1; |
2011 |
brr[cont_chain,eps_cont,emb_chain_cpo] 1; |
|
| 2469 | 2012 |
by (Asm_simp_tac 1); |
| 5136 | 2013 |
by (asm_simp_tac(simpset() addsimps[eps_cont RS cont_lub]) 1); |
| 3425 | 2014 |
qed "rho_emb_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2015 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2016 |
(* 32 vs 61, using safe_tac with imp in asm would be unfortunate (5steps) *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2017 |
|
| 5136 | 2018 |
Goal (* lemma1 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2019 |
"[|m le n; emb_chain(DD,ee); x:set(Dinf(DD,ee)); m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2020 |
\ rel(DD`n,e_less(DD,ee,m,n)`(x`m),x`n)"; |
| 5136 | 2021 |
by (etac rev_mp 1); (* For induction proof *) |
| 6070 | 2022 |
by (induct_tac "n" 1); |
2023 |
by (rtac impI 1); |
|
2024 |
by (asm_full_simp_tac (simpset() addsimps [e_less_eq]) 1); |
|
| 6169 | 2025 |
by (stac id_conv 1); |
| 5136 | 2026 |
brr[apply_type,Dinf_prod,cpo_refl,emb_chain_cpo,nat_0I] 1; |
| 4091 | 2027 |
by (asm_full_simp_tac (simpset() addsimps [le_succ_iff]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2028 |
by (rtac impI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2029 |
by (etac disjE 1); |
| 1623 | 2030 |
by (dtac mp 1 THEN atac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2031 |
by (rtac cpo_trans 1); |
| 2034 | 2032 |
by (stac e_less_le 2); |
| 5136 | 2033 |
brr[emb_chain_cpo,nat_succI] 1; |
| 2034 | 2034 |
by (stac comp_fun_apply 1); |
| 5136 | 2035 |
brr[emb_chain_emb RS emb_cont, e_less_cont, cont_fun, apply_type, Dinf_prod] 1; |
| 1623 | 2036 |
by (res_inst_tac[("y","x`xa")](emb_chain_emb RS emb_cont RS cont_mono) 1);
|
| 5136 | 2037 |
brr[e_less_cont RS cont_fun, apply_type,Dinf_prod] 1; |
| 1623 | 2038 |
by (res_inst_tac[("x1","x"),("n1","xa")](Dinf_eq RS subst) 1);
|
2039 |
by (rtac (comp_fun_apply RS subst) 3); |
|
2040 |
by (res_inst_tac |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2041 |
[("P",
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2042 |
"%z. rel(DD ` succ(xa), \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2043 |
\ (ee ` xa O Rp(?DD46(xa) ` xa,?DD46(xa) ` succ(xa),?ee46(xa) ` xa)) ` \ |
| 6169 | 2044 |
\ (x ` succ(xa)),z)")](id_conv RS subst) 6); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2045 |
by (rtac rel_cf 7); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2046 |
(* Dinf and cont_fun doesn't go well together, both Pi(_,%x._). *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2047 |
(* brr solves 11 of 12 subgoals *) |
| 5136 | 2048 |
brr[Dinf_prod RS apply_type, cont_fun, Rp_cont, e_less_cont, emb_cont, emb_chain_emb, emb_chain_cpo, apply_type, embRp_rel, disjI1 RS (le_succ_iff RS iffD2), nat_succI] 1; |
2049 |
by (asm_full_simp_tac (simpset() addsimps [e_less_eq]) 1); |
|
| 6169 | 2050 |
by (stac id_conv 1); |
| 5136 | 2051 |
by (auto_tac (claset() addIs [apply_type,Dinf_prod,emb_chain_cpo], simpset())); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2052 |
val lemma1 = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2053 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2054 |
(* 18 vs 40 *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2055 |
|
| 5136 | 2056 |
Goal (* lemma2 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2057 |
"[|n le m; emb_chain(DD,ee); x:set(Dinf(DD,ee)); m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2058 |
\ rel(DD`n,e_gr(DD,ee,m,n)`(x`m),x`n)"; |
| 5136 | 2059 |
by (etac rev_mp 1); (* For induction proof *) |
| 6070 | 2060 |
by (induct_tac "m" 1); |
2061 |
by (rtac impI 1); |
|
2062 |
by (asm_full_simp_tac (simpset() addsimps [e_gr_eq]) 1); |
|
| 6169 | 2063 |
by (stac id_conv 1); |
| 5136 | 2064 |
brr[apply_type,Dinf_prod,cpo_refl,emb_chain_cpo,nat_0I] 1; |
| 4091 | 2065 |
by (asm_full_simp_tac (simpset() addsimps [le_succ_iff]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2066 |
by (rtac impI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2067 |
by (etac disjE 1); |
| 1623 | 2068 |
by (dtac mp 1 THEN atac 1); |
| 2034 | 2069 |
by (stac e_gr_le 1); |
2070 |
by (stac comp_fun_apply 4); |
|
2071 |
by (stac Dinf_eq 7); |
|
| 5136 | 2072 |
brr[emb_chain_emb, emb_chain_cpo, Rp_cont, e_gr_cont, cont_fun, emb_cont, apply_type,Dinf_prod,nat_succI] 1; |
2073 |
by (asm_full_simp_tac (simpset() addsimps [e_gr_eq]) 1); |
|
| 6169 | 2074 |
by (stac id_conv 1); |
| 5136 | 2075 |
by (auto_tac (claset() addIs [apply_type,Dinf_prod,emb_chain_cpo], simpset())); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2076 |
val lemma2 = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2077 |
|
| 5136 | 2078 |
Goalw [eps_def] (* eps1 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2079 |
"[|emb_chain(DD,ee); x:set(Dinf(DD,ee)); m:nat; n:nat|] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2080 |
\ rel(DD`n,eps(DD,ee,m,n)`(x`m),x`n)"; |
|
5116
8eb343ab5748
Renamed expand_if to split_if and setloop split_tac to addsplits,
paulson
parents:
5068
diff
changeset
|
2081 |
by (split_tac [split_if] 1); |
| 5136 | 2082 |
brr[conjI, impI, lemma1, not_le_iff_lt RS iffD1 RS leI RS lemma2, nat_into_Ord] 1; |
| 3425 | 2083 |
qed "eps1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2084 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2085 |
(* The following theorem is needed/useful due to type check for rel_cfI, |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2086 |
but also elsewhere. |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2087 |
Look for occurences of rel_cfI, rel_DinfI, etc to evaluate the problem. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2088 |
|
| 5136 | 2089 |
Goal (* lam_Dinf_cont *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2090 |
"[| emb_chain(DD,ee); n:nat |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2091 |
\ (lam x:set(Dinf(DD,ee)). x`n) : cont(Dinf(DD,ee),DD`n)"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2092 |
by (rtac contI 1); |
| 5136 | 2093 |
brr[lam_type,apply_type,Dinf_prod] 1; |
| 2469 | 2094 |
by (Asm_simp_tac 1); |
| 5136 | 2095 |
brr[rel_Dinf] 1; |
| 2034 | 2096 |
by (stac beta 1); |
| 5136 | 2097 |
by (auto_tac (claset() addIs [cpo_Dinf,islub_in,cpo_lub], simpset())); |
2098 |
by (asm_simp_tac(simpset() addsimps[chain_in,lub_Dinf]) 1); |
|
| 3425 | 2099 |
qed "lam_Dinf_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2100 |
|
| 5136 | 2101 |
Goalw [rho_proj_def] (* rho_projpair *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2102 |
"[| emb_chain(DD,ee); n:nat |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2103 |
\ projpair(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n),rho_proj(DD,ee,n))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2104 |
by (rtac projpairI 1); |
| 5136 | 2105 |
brr[rho_emb_cont] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2106 |
(* lemma used, introduced because same fact needed below due to rel_cfI. *) |
| 5136 | 2107 |
brr[lam_Dinf_cont] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2108 |
(*-----------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2109 |
(* This part is 7 lines, but 30 in HOL (75% reduction!) *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2110 |
by (rtac fun_extension 1); |
| 6169 | 2111 |
by (stac id_conv 3); |
| 2034 | 2112 |
by (stac comp_fun_apply 4); |
2113 |
by (stac beta 7); |
|
2114 |
by (stac rho_emb_id 8); |
|
| 5136 | 2115 |
brr[comp_fun, id_type, lam_type, rho_emb_fun, Dinf_prod RS apply_type, apply_type,refl] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2116 |
(*^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2117 |
by (rtac rel_cfI 1); (* ------------------>>>Yields type cond, not in HOL *) |
| 6169 | 2118 |
by (stac id_conv 1); |
| 2034 | 2119 |
by (stac comp_fun_apply 2); |
2120 |
by (stac beta 5); |
|
2121 |
by (stac rho_emb_apply1 6); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2122 |
by (rtac rel_DinfI 7); (* ------------------>>>Yields type cond, not in HOL *) |
| 2034 | 2123 |
by (stac beta 7); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2124 |
brr(eps1::lam_type::rho_emb_fun::eps_fun:: (* Dinf_prod bad with lam_type *) |
| 5136 | 2125 |
[Dinf_prod RS apply_type, refl]) 1; |
2126 |
brr[apply_type, eps_fun, Dinf_prod, comp_pres_cont, rho_emb_cont, lam_Dinf_cont,id_cont,cpo_Dinf,emb_chain_cpo] 1; |
|
| 3425 | 2127 |
qed "rho_projpair"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2128 |
|
| 5136 | 2129 |
Goalw [emb_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2130 |
"[| emb_chain(DD,ee); n:nat |] ==> emb(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n))"; |
| 5136 | 2131 |
by (auto_tac (claset() addIs [exI,rho_projpair], simpset())); |
| 3425 | 2132 |
qed "emb_rho_emb"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2133 |
|
| 5268 | 2134 |
Goal "[| emb_chain(DD,ee); n:nat |] ==> \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2135 |
\ rho_proj(DD,ee,n) : cont(Dinf(DD,ee),DD`n)"; |
| 5136 | 2136 |
by (auto_tac (claset() addIs [rho_projpair,projpair_p_cont], simpset())); |
| 3425 | 2137 |
qed "rho_proj_cont"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2138 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2139 |
(*----------------------------------------------------------------------*) |
| 1461 | 2140 |
(* Commutivity and universality. *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2141 |
(*----------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2142 |
|
| 5136 | 2143 |
val prems = Goalw [commute_def] (* commuteI *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2144 |
"[| !!n. n:nat ==> emb(DD`n,E,r(n)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2145 |
\ !!m n. [|m le n; m:nat; n:nat|] ==> r(n) O eps(DD,ee,m,n) = r(m) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2146 |
\ commute(DD,ee,E,r)"; |
| 4152 | 2147 |
by Safe_tac; |
| 5136 | 2148 |
by (REPEAT (ares_tac prems 1)); |
| 3425 | 2149 |
qed "commuteI"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2150 |
|
| 5136 | 2151 |
Goalw [commute_def] (* commute_emb *) |
2152 |
"[| commute(DD,ee,E,r); n:nat |] ==> emb(DD`n,E,r(n))"; |
|
| 2469 | 2153 |
by (Fast_tac 1); |
| 3425 | 2154 |
qed "commute_emb"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2155 |
|
|
6176
707b6f9859d2
tidied, with left_inverse & right_inverse as default simprules
paulson
parents:
6169
diff
changeset
|
2156 |
AddTCs [commute_emb]; |
|
707b6f9859d2
tidied, with left_inverse & right_inverse as default simprules
paulson
parents:
6169
diff
changeset
|
2157 |
|
| 5136 | 2158 |
Goalw [commute_def] (* commute_eq *) |
2159 |
"[| commute(DD,ee,E,r); m le n; m:nat; n:nat |] ==> \ |
|
2160 |
\ r(n) O eps(DD,ee,m,n) = r(m) "; |
|
2161 |
by (Blast_tac 1); |
|
| 3425 | 2162 |
qed "commute_eq"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2163 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2164 |
(* Shorter proof: 11 vs 46 lines. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2165 |
|
| 5136 | 2166 |
Goal (* rho_emb_commute *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2167 |
"emb_chain(DD,ee) ==> commute(DD,ee,Dinf(DD,ee),rho_emb(DD,ee))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2168 |
by (rtac commuteI 1); |
| 5136 | 2169 |
brr[emb_rho_emb] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2170 |
by (rtac fun_extension 1); (* Manual instantiation in HOL. *) |
| 2034 | 2171 |
by (stac comp_fun_apply 3); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2172 |
by (rtac fun_extension 6); (* Next, clean up and instantiate unknowns *) |
| 5136 | 2173 |
brr[comp_fun,rho_emb_fun,eps_fun,Dinf_prod,apply_type] 1; |
| 1623 | 2174 |
by (asm_simp_tac |
| 5136 | 2175 |
(simpset() addsimps[rho_emb_apply2, eps_fun RS apply_type]) 1); |
| 1623 | 2176 |
by (rtac (comp_fun_apply RS subst) 1); |
2177 |
by (rtac (eps_split_left RS subst) 4); |
|
| 5136 | 2178 |
by (auto_tac (claset() addIs [eps_fun], simpset())); |
| 3425 | 2179 |
qed "rho_emb_commute"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2180 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2181 |
val le_succ = prove_goal Arith.thy "n:nat ==> n le succ(n)" |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2182 |
(fn prems => |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2183 |
[REPEAT (ares_tac |
| 1623 | 2184 |
((disjI1 RS(le_succ_iff RS iffD2))::le_refl::nat_into_Ord::prems) 1)]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2185 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2186 |
(* Shorter proof: 21 vs 83 (106 - 23, due to OAssoc complication) *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2187 |
|
| 5136 | 2188 |
Goal (* commute_chain *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2189 |
"[| commute(DD,ee,E,r); emb_chain(DD,ee); cpo(E) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2190 |
\ chain(cf(E,E),lam n:nat. r(n) O Rp(DD`n,E,r(n)))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2191 |
by (rtac chainI 1); |
| 5136 | 2192 |
by (blast_tac (claset() addIs [lam_type, cont_cf, comp_pres_cont, commute_emb, Rp_cont, emb_cont, emb_chain_cpo]) 1); |
| 2469 | 2193 |
by (Asm_simp_tac 1); |
| 1623 | 2194 |
by (res_inst_tac[("r1","r"),("m1","n")](commute_eq RS subst) 1);
|
| 5136 | 2195 |
brr[le_succ,nat_succI] 1; |
| 2034 | 2196 |
by (stac Rp_comp 1); |
| 5136 | 2197 |
brr[emb_eps,commute_emb,emb_chain_cpo,le_succ,nat_succI] 1; |
| 1623 | 2198 |
by (rtac (comp_assoc RS subst) 1); (* Remember that comp_assoc is simpler in Isa *) |
2199 |
by (res_inst_tac[("r1","r(succ(n))")](comp_assoc RS ssubst) 1);
|
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2200 |
by (rtac comp_mono 1); |
| 5136 | 2201 |
by (REPEAT |
2202 |
(blast_tac (claset() addIs [comp_pres_cont, eps_cont, emb_eps, |
|
2203 |
commute_emb, Rp_cont, emb_cont, |
|
2204 |
emb_chain_cpo,le_succ]) 1)); |
|
| 1623 | 2205 |
by (res_inst_tac[("b","r(succ(n))")](comp_id RS subst) 1); (* 1 subst too much *)
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2206 |
by (rtac comp_mono 2); |
| 5136 | 2207 |
by (REPEAT |
2208 |
(blast_tac (claset() addIs [comp_pres_cont, eps_cont, emb_eps, emb_id, |
|
2209 |
commute_emb, Rp_cont, emb_cont, cont_fun, |
|
2210 |
emb_chain_cpo,le_succ]) 1)); |
|
2211 |
by (stac comp_id 1); (* Undoes "1 subst too much", typing next anyway *) |
|
2212 |
by (REPEAT |
|
2213 |
(blast_tac (claset() addIs [cont_fun, Rp_cont, emb_cont, commute_emb, |
|
2214 |
cont_cf, cpo_cf, emb_chain_cpo, |
|
2215 |
embRp_rel,emb_eps,le_succ]) 1)); |
|
| 3425 | 2216 |
qed "commute_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2217 |
|
| 5136 | 2218 |
Goal (* rho_emb_chain *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2219 |
"emb_chain(DD,ee) ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2220 |
\ chain(cf(Dinf(DD,ee),Dinf(DD,ee)), \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2221 |
\ lam n:nat. rho_emb(DD,ee,n) O Rp(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n)))"; |
| 5136 | 2222 |
by (auto_tac (claset() addIs [commute_chain,rho_emb_commute,cpo_Dinf], simpset())); |
| 3425 | 2223 |
qed "rho_emb_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2224 |
|
| 5136 | 2225 |
Goal "[| emb_chain(DD,ee); x:set(Dinf(DD,ee)) |] ==> \ |
2226 |
\ chain(Dinf(DD,ee), \ |
|
2227 |
\ lam n:nat. \ |
|
2228 |
\ (rho_emb(DD,ee,n) O Rp(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n)))`x)"; |
|
2229 |
by (dtac (rho_emb_chain RS chain_cf) 1); |
|
2230 |
by (assume_tac 1); |
|
| 2469 | 2231 |
by (Asm_full_simp_tac 1); |
| 3425 | 2232 |
qed "rho_emb_chain_apply1"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2233 |
|
| 5136 | 2234 |
Goal "[| chain(iprod(DD),X); emb_chain(DD,ee); n:nat |] ==> \ |
2235 |
\ chain(DD`n,lam m:nat. X `m `n)"; |
|
2236 |
by (auto_tac (claset() addIs [chain_iprod,emb_chain_cpo], simpset())); |
|
| 3425 | 2237 |
qed "chain_iprod_emb_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2238 |
|
| 5136 | 2239 |
Goal (* rho_emb_chain_apply2 *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2240 |
"[| emb_chain(DD,ee); x:set(Dinf(DD,ee)); n:nat |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2241 |
\ chain \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2242 |
\ (DD`n, \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2243 |
\ lam xa:nat. \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2244 |
\ (rho_emb(DD, ee, xa) O Rp(DD ` xa, Dinf(DD, ee),rho_emb(DD, ee, xa))) ` \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2245 |
\ x ` n)"; |
| 5136 | 2246 |
by (forward_tac [rho_emb_chain_apply1 RS chain_Dinf RS chain_iprod_emb_chain] 1); |
2247 |
by Auto_tac; |
|
| 3425 | 2248 |
qed "rho_emb_chain_apply2"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2249 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2250 |
(* Shorter proof: 32 vs 72 (roughly), Isabelle proof has lemmas. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2251 |
|
| 5136 | 2252 |
Goal (* rho_emb_lub *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2253 |
"emb_chain(DD,ee) ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2254 |
\ lub(cf(Dinf(DD,ee),Dinf(DD,ee)), \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2255 |
\ lam n:nat. rho_emb(DD,ee,n) O Rp(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n))) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2256 |
\ id(set(Dinf(DD,ee)))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2257 |
by (rtac cpo_antisym 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2258 |
by (rtac cpo_cf 1); (* Instantiate variable, continued below (would loop otherwise) *) |
| 5136 | 2259 |
brr[cpo_Dinf] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2260 |
by (rtac islub_least 1); |
| 5136 | 2261 |
brr[cpo_lub,rho_emb_chain,cpo_cf,cpo_Dinf,isubI,cont_cf,id_cont] 1; |
| 2469 | 2262 |
by (Asm_simp_tac 1); |
| 5136 | 2263 |
brr[embRp_rel,emb_rho_emb,emb_chain_cpo,cpo_Dinf] 1; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2264 |
by (rtac rel_cfI 1); |
| 6169 | 2265 |
by (asm_simp_tac (simpset() addsimps[lub_cf,rho_emb_chain,cpo_Dinf]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2266 |
by (rtac rel_DinfI 1); (* Addtional assumptions *) |
| 2034 | 2267 |
by (stac lub_Dinf 1); |
| 5136 | 2268 |
brr[rho_emb_chain_apply1] 1; |
2269 |
brr[Dinf_prod, cpo_lub RS islub_in, id_cont, cpo_Dinf, cpo_cf, cf_cont, rho_emb_chain, rho_emb_chain_apply1, id_cont RS cont_cf] 2; |
|
| 2469 | 2270 |
by (Asm_simp_tac 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2271 |
by (rtac dominate_islub 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2272 |
by (rtac cpo_lub 3); |
| 5136 | 2273 |
brr[rho_emb_chain_apply2,emb_chain_cpo] 3; |
| 1623 | 2274 |
by (res_inst_tac[("x1","x`n")](chain_const RS chain_fun) 3);
|
| 5136 | 2275 |
brr[islub_const, apply_type, Dinf_prod, emb_chain_cpo, chain_fun, rho_emb_chain_apply2] 2; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2276 |
by (rtac dominateI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2277 |
by (assume_tac 1); |
| 2469 | 2278 |
by (Asm_simp_tac 1); |
| 2034 | 2279 |
by (stac comp_fun_apply 1); |
| 5136 | 2280 |
brr[cont_fun,Rp_cont,emb_cont,emb_rho_emb,cpo_Dinf,emb_chain_cpo] 1; |
| 2034 | 2281 |
by (stac ((rho_projpair RS Rp_unique)) 1); |
| 1623 | 2282 |
by (SELECT_GOAL(rewtac rho_proj_def) 5); |
| 2469 | 2283 |
by (Asm_simp_tac 5); |
| 2034 | 2284 |
by (stac rho_emb_id 5); |
| 5136 | 2285 |
by (auto_tac (claset() addIs [cpo_Dinf,apply_type,Dinf_prod,emb_chain_cpo], |
2286 |
simpset())); |
|
| 3425 | 2287 |
qed "rho_emb_lub"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2288 |
|
| 5136 | 2289 |
Goal (* theta_chain, almost same prf as commute_chain *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2290 |
"[| commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2291 |
\ emb_chain(DD,ee); cpo(E); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2292 |
\ chain(cf(E,G),lam n:nat. f(n) O Rp(DD`n,E,r(n)))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2293 |
by (rtac chainI 1); |
| 5136 | 2294 |
by (blast_tac (claset() addIs [lam_type, cont_cf, comp_pres_cont, commute_emb, Rp_cont,emb_cont,emb_chain_cpo]) 1); |
| 2469 | 2295 |
by (Asm_simp_tac 1); |
| 1623 | 2296 |
by (res_inst_tac[("r1","r"),("m1","n")](commute_eq RS subst) 1);
|
2297 |
by (res_inst_tac[("r1","f"),("m1","n")](commute_eq RS subst) 5);
|
|
| 5136 | 2298 |
brr[le_succ,nat_succI] 1; |
| 2034 | 2299 |
by (stac Rp_comp 1); |
| 5136 | 2300 |
brr[emb_eps,commute_emb,emb_chain_cpo,le_succ,nat_succI] 1; |
| 1623 | 2301 |
by (rtac (comp_assoc RS subst) 1); (* Remember that comp_assoc is simpler in Isa *) |
2302 |
by (res_inst_tac[("r1","f(succ(n))")](comp_assoc RS ssubst) 1);
|
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2303 |
by (rtac comp_mono 1); |
| 5136 | 2304 |
by (REPEAT (blast_tac (claset() addIs [comp_pres_cont, eps_cont, emb_eps, commute_emb, Rp_cont, emb_cont,emb_chain_cpo,le_succ]) 1)); |
| 1623 | 2305 |
by (res_inst_tac[("b","f(succ(n))")](comp_id RS subst) 1); (* 1 subst too much *)
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2306 |
by (rtac comp_mono 2); |
| 5136 | 2307 |
by (REPEAT (blast_tac (claset() addIs[comp_pres_cont, eps_cont, emb_eps, emb_id, commute_emb, Rp_cont, emb_cont,cont_fun,emb_chain_cpo,le_succ]) 1)); |
2308 |
by (stac comp_id 1); (* Undoes "1 subst too much", typing next anyway *) |
|
2309 |
by (REPEAT |
|
2310 |
(blast_tac (claset() addIs[cont_fun, Rp_cont, emb_cont, commute_emb, |
|
2311 |
cont_cf, cpo_cf,emb_chain_cpo, |
|
2312 |
embRp_rel,emb_eps,le_succ]) 1)); |
|
| 3425 | 2313 |
qed "theta_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2314 |
|
| 5136 | 2315 |
Goal (* theta_proj_chain, same prf as theta_chain *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2316 |
"[| commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2317 |
\ emb_chain(DD,ee); cpo(E); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2318 |
\ chain(cf(G,E),lam n:nat. r(n) O Rp(DD`n,G,f(n)))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2319 |
by (rtac chainI 1); |
| 5136 | 2320 |
by (blast_tac (claset() addIs [lam_type, cont_cf, comp_pres_cont, commute_emb, Rp_cont,emb_cont,emb_chain_cpo]) 1); |
| 2469 | 2321 |
by (Asm_simp_tac 1); |
| 1623 | 2322 |
by (res_inst_tac[("r1","r"),("m1","n")](commute_eq RS subst) 1);
|
2323 |
by (res_inst_tac[("r1","f"),("m1","n")](commute_eq RS subst) 5);
|
|
| 5136 | 2324 |
brr[le_succ,nat_succI] 1; |
| 2034 | 2325 |
by (stac Rp_comp 1); |
| 5136 | 2326 |
brr[emb_eps,commute_emb,emb_chain_cpo,le_succ,nat_succI] 1; |
| 1623 | 2327 |
by (rtac (comp_assoc RS subst) 1); (* Remember that comp_assoc is simpler in Isa *) |
2328 |
by (res_inst_tac[("r1","r(succ(n))")](comp_assoc RS ssubst) 1);
|
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2329 |
by (rtac comp_mono 1); |
| 5136 | 2330 |
by (REPEAT (blast_tac (claset() addIs [comp_pres_cont, eps_cont, emb_eps, commute_emb, Rp_cont, emb_cont,emb_chain_cpo,le_succ]) 1)); |
| 1623 | 2331 |
by (res_inst_tac[("b","r(succ(n))")](comp_id RS subst) 1); (* 1 subst too much *)
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2332 |
by (rtac comp_mono 2); |
| 5136 | 2333 |
by (REPEAT (blast_tac (claset() addIs[comp_pres_cont, eps_cont, emb_eps, emb_id, commute_emb, Rp_cont, emb_cont,cont_fun,emb_chain_cpo,le_succ]) 1)); |
2334 |
by (stac comp_id 1); (* Undoes "1 subst too much", typing next anyway *) |
|
2335 |
by (REPEAT |
|
2336 |
(blast_tac (claset() addIs[cont_fun, Rp_cont, emb_cont, commute_emb, |
|
2337 |
cont_cf, cpo_cf,emb_chain_cpo,embRp_rel, |
|
2338 |
emb_eps,le_succ]) 1)); |
|
| 3425 | 2339 |
qed "theta_proj_chain"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2340 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2341 |
(* Simplification with comp_assoc is possible inside a lam-abstraction, |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2342 |
because it does not have assumptions. If it had, as the HOL-ST theorem |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2343 |
too strongly has, we would be in deep trouble due to the lack of proper |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2344 |
conditional rewriting (a HOL contrib provides something that works). *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2345 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2346 |
(* Controlled simplification inside lambda: introduce lemmas *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2347 |
|
| 5136 | 2348 |
Goal "[| commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2349 |
\ emb_chain(DD,ee); cpo(E); cpo(G); x:nat |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2350 |
\ r(x) O Rp(DD ` x, G, f(x)) O f(x) O Rp(DD ` x, E, r(x)) = \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2351 |
\ r(x) O Rp(DD ` x, E, r(x))"; |
| 1623 | 2352 |
by (res_inst_tac[("s1","f(x)")](comp_assoc RS subst) 1);
|
| 2034 | 2353 |
by (stac embRp_eq 1); |
2354 |
by (stac id_comp 4); |
|
| 5136 | 2355 |
by (auto_tac (claset() addIs [cont_fun,Rp_cont,commute_emb,emb_chain_cpo], |
2356 |
simpset())); |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2357 |
val lemma = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2358 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2359 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2360 |
(* Shorter proof (but lemmas): 19 vs 79 (103 - 24, due to OAssoc) *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2361 |
|
| 5136 | 2362 |
Goalw [projpair_def,rho_proj_def] (* theta_projpair *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2363 |
"[| lub(cf(E,E), lam n:nat. r(n) O Rp(DD`n,E,r(n))) = id(set(E)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2364 |
\ commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2365 |
\ emb_chain(DD,ee); cpo(E); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2366 |
\ projpair \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2367 |
\ (E,G, \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2368 |
\ lub(cf(E,G), lam n:nat. f(n) O Rp(DD`n,E,r(n))), \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2369 |
\ lub(cf(G,E), lam n:nat. r(n) O Rp(DD`n,G,f(n))))"; |
| 4152 | 2370 |
by Safe_tac; |
| 2034 | 2371 |
by (stac comp_lubs 3); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2372 |
(* The following one line is 15 lines in HOL, and includes existentials. *) |
| 5136 | 2373 |
brr[cf_cont,islub_in,cpo_lub,cpo_cf,theta_chain,theta_proj_chain] 1; |
| 4091 | 2374 |
by (simp_tac (simpset() addsimps[comp_assoc]) 1); |
| 5136 | 2375 |
by (asm_simp_tac (simpset() addsimps[lemma]) 1); |
2376 |
by (stac comp_lubs 1); |
|
2377 |
brr[cf_cont,islub_in,cpo_lub,cpo_cf,theta_chain,theta_proj_chain] 1; |
|
| 4091 | 2378 |
by (simp_tac (simpset() addsimps[comp_assoc]) 1); |
| 5136 | 2379 |
by (asm_simp_tac (simpset() addsimps[lemma]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2380 |
by (rtac dominate_islub 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2381 |
by (rtac cpo_lub 2); |
| 6153 | 2382 |
brr[commute_chain, commute_emb, islub_const, cont_cf, id_cont, |
2383 |
cpo_cf, chain_fun,chain_const] 2; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2384 |
by (rtac dominateI 1); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2385 |
by (assume_tac 1); |
| 2469 | 2386 |
by (Asm_simp_tac 1); |
| 5136 | 2387 |
by (blast_tac (claset() addIs [embRp_rel,commute_emb,emb_chain_cpo]) 1); |
| 3425 | 2388 |
qed "theta_projpair"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2389 |
|
| 5136 | 2390 |
Goalw [emb_def] |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2391 |
"[| lub(cf(E,E), lam n:nat. r(n) O Rp(DD`n,E,r(n))) = id(set(E)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2392 |
\ commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2393 |
\ emb_chain(DD,ee); cpo(E); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2394 |
\ emb(E,G,lub(cf(E,G), lam n:nat. f(n) O Rp(DD`n,E,r(n))))"; |
| 5136 | 2395 |
by (blast_tac (claset() addIs [theta_projpair]) 1); |
| 3425 | 2396 |
qed "emb_theta"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2397 |
|
| 5136 | 2398 |
Goal (* mono_lemma *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2399 |
"[| g:cont(D,D'); cpo(D); cpo(D'); cpo(E) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2400 |
\ (lam f : cont(D',E). f O g) : mono(cf(D',E),cf(D,E))"; |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2401 |
by (rtac monoI 1); |
| 1623 | 2402 |
by (REPEAT(dtac cf_cont 2)); |
| 2469 | 2403 |
by (Asm_simp_tac 2); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2404 |
by (rtac comp_mono 2); |
| 1623 | 2405 |
by (SELECT_GOAL(rewrite_goals_tac[set_def,cf_def]) 1); |
| 2469 | 2406 |
by (Asm_simp_tac 1); |
| 5136 | 2407 |
by (auto_tac (claset() addIs [lam_type,comp_pres_cont,cpo_cf,cont_cf], |
2408 |
simpset())); |
|
| 3425 | 2409 |
qed "mono_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2410 |
|
| 5136 | 2411 |
Goal "[| commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
2412 |
\ emb_chain(DD,ee); cpo(E); cpo(G); n:nat |] ==> \ |
|
2413 |
\ (lam na:nat. (lam f:cont(E, G). f O r(n)) ` \ |
|
2414 |
\ ((lam n:nat. f(n) O Rp(DD ` n, E, r(n))) ` na)) = \ |
|
2415 |
\ (lam na:nat. (f(na) O Rp(DD ` na, E, r(na))) O r(n))"; |
|
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2416 |
by (rtac fun_extension 1); |
| 6070 | 2417 |
by (fast_tac (claset() addIs [lam_type]) 1); |
|
6176
707b6f9859d2
tidied, with left_inverse & right_inverse as default simprules
paulson
parents:
6169
diff
changeset
|
2418 |
by (Asm_simp_tac 2); |
| 6169 | 2419 |
by (fast_tac (claset() addIs [lam_type]) 1); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2420 |
val lemma = result(); |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2421 |
|
| 5136 | 2422 |
Goal "[| commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
2423 |
\ emb_chain(DD,ee); cpo(E); cpo(G); n:nat |] ==> \ |
|
2424 |
\ chain(cf(DD`n,G),lam x:nat. (f(x) O Rp(DD ` x, E, r(x))) O r(n))"; |
|
2425 |
by (rtac (lemma RS subst) 1); |
|
2426 |
by (REPEAT |
|
2427 |
(blast_tac (claset() addIs[theta_chain,emb_chain_cpo, |
|
2428 |
commute_emb RS emb_cont RS mono_lemma RS mono_chain]) 1)); |
|
| 3425 | 2429 |
qed "chain_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2430 |
|
| 5136 | 2431 |
Goalw [suffix_def] (* suffix_lemma *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2432 |
"[| commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2433 |
\ emb_chain(DD,ee); cpo(E); cpo(G); cpo(DD`x); x:nat |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2434 |
\ suffix(lam n:nat. (f(n) O Rp(DD`n,E,r(n))) O r(x),x) = (lam n:nat. f(x))"; |
| 5136 | 2435 |
by (Asm_simp_tac 1); |
2436 |
by (rtac (lam_type RS fun_extension) 1); |
|
2437 |
by (REPEAT (blast_tac (claset() addIs [lam_type, comp_fun, cont_fun, Rp_cont, emb_cont, commute_emb, add_type,emb_chain_cpo]) 1)); |
|
| 2469 | 2438 |
by (Asm_simp_tac 1); |
| 5136 | 2439 |
by (subgoal_tac "f(x #+ xa) O \ |
2440 |
\ (Rp(DD ` (x #+ xa), E, r(x #+ xa)) O r(x #+ xa)) O \ |
|
2441 |
\ eps(DD, ee, x, x #+ xa) = f(x)" 1); |
|
2442 |
by (asm_simp_tac (simpset() addsimps [embRp_eq,eps_fun RS id_comp,commute_emb, |
|
2443 |
emb_chain_cpo]) 2); |
|
2444 |
by (blast_tac (claset() addIs [commute_eq,add_type,add_le_self]) 2); |
|
2445 |
by (asm_full_simp_tac |
|
2446 |
(simpset() addsimps [comp_assoc,commute_eq,add_le_self]) 1); |
|
| 3425 | 2447 |
qed "suffix_lemma"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2448 |
|
| 5136 | 2449 |
|
2450 |
||
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2451 |
val mediatingI = prove_goalw Limit.thy [mediating_def] |
| 3840 | 2452 |
"[|emb(E,G,t); !!n. n:nat ==> f(n) = t O r(n) |]==>mediating(E,G,r,f,t)" |
| 5136 | 2453 |
(fn prems => [Safe_tac,REPEAT (ares_tac prems 1)]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2454 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2455 |
val mediating_emb = prove_goalw Limit.thy [mediating_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2456 |
"!!z. mediating(E,G,r,f,t) ==> emb(E,G,t)" |
| 2469 | 2457 |
(fn prems => [Fast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2458 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2459 |
val mediating_eq = prove_goalw Limit.thy [mediating_def] |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2460 |
"!!z. [| mediating(E,G,r,f,t); n:nat |] ==> f(n) = t O r(n)" |
| 5136 | 2461 |
(fn prems => [Blast_tac 1]); |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2462 |
|
| 5136 | 2463 |
Goal (* lub_universal_mediating *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2464 |
"[| lub(cf(E,E), lam n:nat. r(n) O Rp(DD`n,E,r(n))) = id(set(E)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2465 |
\ commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2466 |
\ emb_chain(DD,ee); cpo(E); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2467 |
\ mediating(E,G,r,f,lub(cf(E,G), lam n:nat. f(n) O Rp(DD`n,E,r(n))))"; |
| 5136 | 2468 |
brr[mediatingI,emb_theta] 1; |
| 1623 | 2469 |
by (res_inst_tac[("b","r(n)")](lub_const RS subst) 1);
|
| 2034 | 2470 |
by (stac comp_lubs 3); |
| 5136 | 2471 |
by (REPEAT (blast_tac (claset() addIs [cont_cf, emb_cont, commute_emb, cpo_cf, theta_chain, chain_const, emb_chain_cpo]) 1)); |
| 2469 | 2472 |
by (Simp_tac 1); |
| 5136 | 2473 |
by (stac (lub_suffix RS sym) 1); |
2474 |
brr[chain_lemma,cpo_cf,emb_chain_cpo] 1; |
|
2475 |
by (asm_simp_tac |
|
2476 |
(simpset() addsimps [suffix_lemma, lub_const, cont_cf, emb_cont, |
|
2477 |
commute_emb, cpo_cf, emb_chain_cpo]) 1); |
|
| 3425 | 2478 |
qed "lub_universal_mediating"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2479 |
|
| 5136 | 2480 |
Goal (* lub_universal_unique *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2481 |
"[| mediating(E,G,r,f,t); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2482 |
\ lub(cf(E,E), lam n:nat. r(n) O Rp(DD`n,E,r(n))) = id(set(E)); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2483 |
\ commute(DD,ee,E,r); commute(DD,ee,G,f); \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2484 |
\ emb_chain(DD,ee); cpo(E); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2485 |
\ t = lub(cf(E,G), lam n:nat. f(n) O Rp(DD`n,E,r(n)))"; |
| 1623 | 2486 |
by (res_inst_tac[("b","t")](comp_id RS subst) 1);
|
| 5136 | 2487 |
by (etac subst 2); |
| 1623 | 2488 |
by (res_inst_tac[("b","t")](lub_const RS subst) 2);
|
| 2034 | 2489 |
by (stac comp_lubs 4); |
| 5136 | 2490 |
by (asm_simp_tac (simpset() addsimps [comp_assoc, |
2491 |
read_instantiate [("f","f")] mediating_eq]) 9);
|
|
2492 |
brr[cont_fun, emb_cont, mediating_emb, cont_cf, cpo_cf, chain_const, commute_chain,emb_chain_cpo] 1; |
|
| 3425 | 2493 |
qed "lub_universal_unique"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2494 |
|
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2495 |
(*---------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2496 |
(* Dinf yields the inverse_limit, stated as rho_emb_commute and *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2497 |
(* Dinf_universal. *) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2498 |
(*---------------------------------------------------------------------*) |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2499 |
|
| 5136 | 2500 |
Goal (* Dinf_universal *) |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2501 |
"[| commute(DD,ee,G,f); emb_chain(DD,ee); cpo(G) |] ==> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2502 |
\ mediating \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2503 |
\ (Dinf(DD,ee),G,rho_emb(DD,ee),f, \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2504 |
\ lub(cf(Dinf(DD,ee),G), \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2505 |
\ lam n:nat. f(n) O Rp(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n)))) & \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2506 |
\ (ALL t. mediating(Dinf(DD,ee),G,rho_emb(DD,ee),f,t) --> \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2507 |
\ t = lub(cf(Dinf(DD,ee),G), \ |
|
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2508 |
\ lam n:nat. f(n) O Rp(DD`n,Dinf(DD,ee),rho_emb(DD,ee,n))))"; |
| 4152 | 2509 |
by Safe_tac; |
| 5136 | 2510 |
brr[lub_universal_mediating,rho_emb_commute,rho_emb_lub,cpo_Dinf] 1; |
2511 |
by (auto_tac (claset() addIs [lub_universal_unique,rho_emb_commute,rho_emb_lub,cpo_Dinf], simpset())); |
|
| 3425 | 2512 |
qed "Dinf_universal"; |
|
1281
68f6be60ab1c
The inverse limit construction -- thanks to Sten Agerholm
paulson
parents:
diff
changeset
|
2513 |