author | paulson |
Wed, 28 Jan 2004 17:01:01 +0100 | |
changeset 14369 | c50188fe6366 |
parent 14365 | 3d4df8c166ae |
child 14370 | b0064703967b |
permissions | -rw-r--r-- |
10751 | 1 |
(* Title : HOL/Real/Hyperreal/HyperDef.thy |
2 |
ID : $Id$ |
|
3 |
Author : Jacques D. Fleuriot |
|
4 |
Copyright : 1998 University of Cambridge |
|
5 |
Description : Construction of hyperreals using ultrafilters |
|
13487 | 6 |
*) |
10751 | 7 |
|
14299 | 8 |
theory HyperDef = Filter + Real |
9 |
files ("fuf.ML"): (*Warning: file fuf.ML refers to the name Hyperdef!*) |
|
10751 | 10 |
|
11 |
||
12 |
constdefs |
|
14299 | 13 |
|
14361
ad2f5da643b4
* Support for raw latex output in control symbols: \<^raw...>
schirmer
parents:
14348
diff
changeset
|
14 |
FreeUltrafilterNat :: "nat set set" ("\<U>") |
14299 | 15 |
"FreeUltrafilterNat == (SOME U. U \<in> FreeUltrafilter (UNIV:: nat set))" |
16 |
||
17 |
hyprel :: "((nat=>real)*(nat=>real)) set" |
|
18 |
"hyprel == {p. \<exists>X Y. p = ((X::nat=>real),Y) & |
|
10751 | 19 |
{n::nat. X(n) = Y(n)}: FreeUltrafilterNat}" |
20 |
||
14299 | 21 |
typedef hypreal = "UNIV//hyprel" |
22 |
by (auto simp add: quotient_def) |
|
10751 | 23 |
|
14299 | 24 |
instance hypreal :: ord .. |
25 |
instance hypreal :: zero .. |
|
26 |
instance hypreal :: one .. |
|
27 |
instance hypreal :: plus .. |
|
28 |
instance hypreal :: times .. |
|
29 |
instance hypreal :: minus .. |
|
30 |
instance hypreal :: inverse .. |
|
10751 | 31 |
|
32 |
||
14299 | 33 |
defs (overloaded) |
34 |
||
35 |
hypreal_zero_def: |
|
12018
ec054019c910
Numerals and simprocs for types real and hypreal. The abstract
paulson
parents:
11713
diff
changeset
|
36 |
"0 == Abs_hypreal(hyprel``{%n::nat. (0::real)})" |
10751 | 37 |
|
14299 | 38 |
hypreal_one_def: |
12018
ec054019c910
Numerals and simprocs for types real and hypreal. The abstract
paulson
parents:
11713
diff
changeset
|
39 |
"1 == Abs_hypreal(hyprel``{%n::nat. (1::real)})" |
10751 | 40 |
|
14299 | 41 |
hypreal_minus_def: |
42 |
"- P == Abs_hypreal(\<Union>X \<in> Rep_hypreal(P). hyprel``{%n::nat. - (X n)})" |
|
10751 | 43 |
|
14299 | 44 |
hypreal_diff_def: |
10751 | 45 |
"x - y == x + -(y::hypreal)" |
46 |
||
14299 | 47 |
hypreal_inverse_def: |
48 |
"inverse P == Abs_hypreal(\<Union>X \<in> Rep_hypreal(P). |
|
12018
ec054019c910
Numerals and simprocs for types real and hypreal. The abstract
paulson
parents:
11713
diff
changeset
|
49 |
hyprel``{%n. if X n = 0 then 0 else inverse (X n)})" |
10751 | 50 |
|
14299 | 51 |
hypreal_divide_def: |
10751 | 52 |
"P / Q::hypreal == P * inverse Q" |
13487 | 53 |
|
10751 | 54 |
constdefs |
55 |
||
14299 | 56 |
hypreal_of_real :: "real => hypreal" |
10834 | 57 |
"hypreal_of_real r == Abs_hypreal(hyprel``{%n::nat. r})" |
10751 | 58 |
|
10919
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
59 |
omega :: hypreal (*an infinite number = [<1,2,3,...>] *) |
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
60 |
"omega == Abs_hypreal(hyprel``{%n::nat. real (Suc n)})" |
13487 | 61 |
|
10919
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
62 |
epsilon :: hypreal (*an infinitesimal number = [<1,1/2,1/3,...>] *) |
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
63 |
"epsilon == Abs_hypreal(hyprel``{%n::nat. inverse (real (Suc n))})" |
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
64 |
|
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
65 |
syntax (xsymbols) |
14299 | 66 |
omega :: hypreal ("\<omega>") |
67 |
epsilon :: hypreal ("\<epsilon>") |
|
10919
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
10834
diff
changeset
|
68 |
|
10751 | 69 |
|
13487 | 70 |
defs |
71 |
||
14299 | 72 |
hypreal_add_def: |
73 |
"P + Q == Abs_hypreal(\<Union>X \<in> Rep_hypreal(P). \<Union>Y \<in> Rep_hypreal(Q). |
|
10834 | 74 |
hyprel``{%n::nat. X n + Y n})" |
10751 | 75 |
|
14299 | 76 |
hypreal_mult_def: |
77 |
"P * Q == Abs_hypreal(\<Union>X \<in> Rep_hypreal(P). \<Union>Y \<in> Rep_hypreal(Q). |
|
10834 | 78 |
hyprel``{%n::nat. X n * Y n})" |
10751 | 79 |
|
14299 | 80 |
hypreal_less_def: |
81 |
"P < (Q::hypreal) == \<exists>X Y. X \<in> Rep_hypreal(P) & |
|
82 |
Y \<in> Rep_hypreal(Q) & |
|
83 |
{n::nat. X n < Y n} \<in> FreeUltrafilterNat" |
|
84 |
hypreal_le_def: |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
85 |
"P \<le> (Q::hypreal) == ~(Q < P)" |
10751 | 86 |
|
14329 | 87 |
hrabs_def: "abs (r::hypreal) == (if 0 \<le> r then r else -r)" |
88 |
||
89 |
||
90 |
subsection{*The Set of Naturals is not Finite*} |
|
14299 | 91 |
|
92 |
(*** based on James' proof that the set of naturals is not finite ***) |
|
14329 | 93 |
lemma finite_exhausts [rule_format]: |
94 |
"finite (A::nat set) --> (\<exists>n. \<forall>m. Suc (n + m) \<notin> A)" |
|
14299 | 95 |
apply (rule impI) |
14301 | 96 |
apply (erule_tac F = A in finite_induct) |
97 |
apply (blast, erule exE) |
|
14299 | 98 |
apply (rule_tac x = "n + x" in exI) |
14301 | 99 |
apply (rule allI, erule_tac x = "x + m" in allE) |
14299 | 100 |
apply (auto simp add: add_ac) |
101 |
done |
|
102 |
||
14329 | 103 |
lemma finite_not_covers [rule_format (no_asm)]: |
104 |
"finite (A :: nat set) --> (\<exists>n. n \<notin>A)" |
|
14301 | 105 |
by (rule impI, drule finite_exhausts, blast) |
14299 | 106 |
|
107 |
lemma not_finite_nat: "~ finite(UNIV:: nat set)" |
|
14301 | 108 |
by (fast dest!: finite_exhausts) |
14299 | 109 |
|
14329 | 110 |
|
111 |
subsection{*Existence of Free Ultrafilter over the Naturals*} |
|
112 |
||
113 |
text{*Also, proof of various properties of @{term FreeUltrafilterNat}: |
|
114 |
an arbitrary free ultrafilter*} |
|
14299 | 115 |
|
116 |
lemma FreeUltrafilterNat_Ex: "\<exists>U. U: FreeUltrafilter (UNIV::nat set)" |
|
14301 | 117 |
by (rule not_finite_nat [THEN FreeUltrafilter_Ex]) |
14299 | 118 |
|
14301 | 119 |
lemma FreeUltrafilterNat_mem [simp]: |
14299 | 120 |
"FreeUltrafilterNat: FreeUltrafilter(UNIV:: nat set)" |
121 |
apply (unfold FreeUltrafilterNat_def) |
|
122 |
apply (rule FreeUltrafilterNat_Ex [THEN exE]) |
|
14301 | 123 |
apply (rule someI2, assumption+) |
14299 | 124 |
done |
125 |
||
126 |
lemma FreeUltrafilterNat_finite: "finite x ==> x \<notin> FreeUltrafilterNat" |
|
127 |
apply (unfold FreeUltrafilterNat_def) |
|
128 |
apply (rule FreeUltrafilterNat_Ex [THEN exE]) |
|
14301 | 129 |
apply (rule someI2, assumption) |
14299 | 130 |
apply (blast dest: mem_FreeUltrafiltersetD1) |
131 |
done |
|
132 |
||
133 |
lemma FreeUltrafilterNat_not_finite: "x: FreeUltrafilterNat ==> ~ finite x" |
|
14301 | 134 |
by (blast dest: FreeUltrafilterNat_finite) |
14299 | 135 |
|
14301 | 136 |
lemma FreeUltrafilterNat_empty [simp]: "{} \<notin> FreeUltrafilterNat" |
14299 | 137 |
apply (unfold FreeUltrafilterNat_def) |
138 |
apply (rule FreeUltrafilterNat_Ex [THEN exE]) |
|
14301 | 139 |
apply (rule someI2, assumption) |
140 |
apply (blast dest: FreeUltrafilter_Ultrafilter Ultrafilter_Filter |
|
141 |
Filter_empty_not_mem) |
|
14299 | 142 |
done |
143 |
||
14329 | 144 |
lemma FreeUltrafilterNat_Int: |
145 |
"[| X: FreeUltrafilterNat; Y: FreeUltrafilterNat |] |
|
14299 | 146 |
==> X Int Y \<in> FreeUltrafilterNat" |
147 |
apply (cut_tac FreeUltrafilterNat_mem) |
|
148 |
apply (blast dest: FreeUltrafilter_Ultrafilter Ultrafilter_Filter mem_FiltersetD1) |
|
149 |
done |
|
150 |
||
14329 | 151 |
lemma FreeUltrafilterNat_subset: |
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
152 |
"[| X: FreeUltrafilterNat; X \<subseteq> Y |] |
14299 | 153 |
==> Y \<in> FreeUltrafilterNat" |
154 |
apply (cut_tac FreeUltrafilterNat_mem) |
|
155 |
apply (blast dest: FreeUltrafilter_Ultrafilter Ultrafilter_Filter mem_FiltersetD2) |
|
156 |
done |
|
157 |
||
14329 | 158 |
lemma FreeUltrafilterNat_Compl: |
159 |
"X: FreeUltrafilterNat ==> -X \<notin> FreeUltrafilterNat" |
|
14301 | 160 |
apply safe |
161 |
apply (drule FreeUltrafilterNat_Int, assumption, auto) |
|
14299 | 162 |
done |
163 |
||
14329 | 164 |
lemma FreeUltrafilterNat_Compl_mem: |
165 |
"X\<notin> FreeUltrafilterNat ==> -X \<in> FreeUltrafilterNat" |
|
14299 | 166 |
apply (cut_tac FreeUltrafilterNat_mem [THEN FreeUltrafilter_iff [THEN iffD1]]) |
14301 | 167 |
apply (safe, drule_tac x = X in bspec) |
14299 | 168 |
apply (auto simp add: UNIV_diff_Compl) |
169 |
done |
|
170 |
||
14329 | 171 |
lemma FreeUltrafilterNat_Compl_iff1: |
172 |
"(X \<notin> FreeUltrafilterNat) = (-X: FreeUltrafilterNat)" |
|
14301 | 173 |
by (blast dest: FreeUltrafilterNat_Compl FreeUltrafilterNat_Compl_mem) |
14299 | 174 |
|
14329 | 175 |
lemma FreeUltrafilterNat_Compl_iff2: |
176 |
"(X: FreeUltrafilterNat) = (-X \<notin> FreeUltrafilterNat)" |
|
14301 | 177 |
by (auto simp add: FreeUltrafilterNat_Compl_iff1 [symmetric]) |
14299 | 178 |
|
14301 | 179 |
lemma FreeUltrafilterNat_UNIV [simp]: "(UNIV::nat set) \<in> FreeUltrafilterNat" |
180 |
by (rule FreeUltrafilterNat_mem [THEN FreeUltrafilter_Ultrafilter, THEN Ultrafilter_Filter, THEN mem_FiltersetD4]) |
|
14299 | 181 |
|
14301 | 182 |
lemma FreeUltrafilterNat_Nat_set [simp]: "UNIV \<in> FreeUltrafilterNat" |
183 |
by auto |
|
14299 | 184 |
|
14329 | 185 |
lemma FreeUltrafilterNat_Nat_set_refl [intro]: |
186 |
"{n. P(n) = P(n)} \<in> FreeUltrafilterNat" |
|
14301 | 187 |
by simp |
14299 | 188 |
|
189 |
lemma FreeUltrafilterNat_P: "{n::nat. P} \<in> FreeUltrafilterNat ==> P" |
|
14301 | 190 |
by (rule ccontr, simp) |
14299 | 191 |
|
192 |
lemma FreeUltrafilterNat_Ex_P: "{n. P(n)} \<in> FreeUltrafilterNat ==> \<exists>n. P(n)" |
|
14301 | 193 |
by (rule ccontr, simp) |
14299 | 194 |
|
195 |
lemma FreeUltrafilterNat_all: "\<forall>n. P(n) ==> {n. P(n)} \<in> FreeUltrafilterNat" |
|
14301 | 196 |
by (auto intro: FreeUltrafilterNat_Nat_set) |
14299 | 197 |
|
14329 | 198 |
|
199 |
text{*Define and use Ultrafilter tactics*} |
|
14299 | 200 |
use "fuf.ML" |
201 |
||
202 |
method_setup fuf = {* |
|
203 |
Method.ctxt_args (fn ctxt => |
|
204 |
Method.METHOD (fn facts => |
|
205 |
fuf_tac (Classical.get_local_claset ctxt, |
|
206 |
Simplifier.get_local_simpset ctxt) 1)) *} |
|
207 |
"free ultrafilter tactic" |
|
208 |
||
209 |
method_setup ultra = {* |
|
210 |
Method.ctxt_args (fn ctxt => |
|
211 |
Method.METHOD (fn facts => |
|
212 |
ultra_tac (Classical.get_local_claset ctxt, |
|
213 |
Simplifier.get_local_simpset ctxt) 1)) *} |
|
214 |
"ultrafilter tactic" |
|
215 |
||
216 |
||
14329 | 217 |
text{*One further property of our free ultrafilter*} |
218 |
lemma FreeUltrafilterNat_Un: |
|
219 |
"X Un Y: FreeUltrafilterNat |
|
14299 | 220 |
==> X: FreeUltrafilterNat | Y: FreeUltrafilterNat" |
221 |
apply auto |
|
14301 | 222 |
apply ultra |
14299 | 223 |
done |
224 |
||
225 |
||
14329 | 226 |
subsection{*Properties of @{term hyprel}*} |
227 |
||
228 |
text{*Proving that @{term hyprel} is an equivalence relation*} |
|
14299 | 229 |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
230 |
lemma hyprel_iff: "((X,Y) \<in> hyprel) = ({n. X n = Y n}: FreeUltrafilterNat)" |
14301 | 231 |
by (unfold hyprel_def, fast) |
14299 | 232 |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
233 |
lemma hyprel_refl: "(x,x) \<in> hyprel" |
14299 | 234 |
apply (unfold hyprel_def) |
235 |
apply (auto simp add: FreeUltrafilterNat_Nat_set) |
|
236 |
done |
|
237 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
238 |
lemma hyprel_sym [rule_format (no_asm)]: "(x,y) \<in> hyprel --> (y,x) \<in> hyprel" |
14301 | 239 |
by (simp add: hyprel_def eq_commute) |
14299 | 240 |
|
241 |
lemma hyprel_trans: |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
242 |
"[|(x,y) \<in> hyprel; (y,z) \<in> hyprel|] ==> (x,z) \<in> hyprel" |
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
243 |
by (unfold hyprel_def, auto, ultra) |
14299 | 244 |
|
245 |
lemma equiv_hyprel: "equiv UNIV hyprel" |
|
246 |
apply (simp add: equiv_def refl_def sym_def trans_def hyprel_refl) |
|
247 |
apply (blast intro: hyprel_sym hyprel_trans) |
|
248 |
done |
|
249 |
||
250 |
(* (hyprel `` {x} = hyprel `` {y}) = ((x,y) \<in> hyprel) *) |
|
251 |
lemmas equiv_hyprel_iff = |
|
252 |
eq_equiv_class_iff [OF equiv_hyprel UNIV_I UNIV_I, simp] |
|
253 |
||
14301 | 254 |
lemma hyprel_in_hypreal [simp]: "hyprel``{x}:hypreal" |
255 |
by (unfold hypreal_def hyprel_def quotient_def, blast) |
|
14299 | 256 |
|
257 |
lemma inj_on_Abs_hypreal: "inj_on Abs_hypreal hypreal" |
|
258 |
apply (rule inj_on_inverseI) |
|
259 |
apply (erule Abs_hypreal_inverse) |
|
260 |
done |
|
261 |
||
262 |
declare inj_on_Abs_hypreal [THEN inj_on_iff, simp] |
|
14301 | 263 |
Abs_hypreal_inverse [simp] |
14299 | 264 |
|
265 |
declare equiv_hyprel [THEN eq_equiv_class_iff, simp] |
|
266 |
||
267 |
declare hyprel_iff [iff] |
|
268 |
||
269 |
lemmas eq_hyprelD = eq_equiv_class [OF _ equiv_hyprel] |
|
270 |
||
271 |
lemma inj_Rep_hypreal: "inj(Rep_hypreal)" |
|
272 |
apply (rule inj_on_inverseI) |
|
273 |
apply (rule Rep_hypreal_inverse) |
|
274 |
done |
|
275 |
||
14301 | 276 |
lemma lemma_hyprel_refl [simp]: "x \<in> hyprel `` {x}" |
277 |
apply (unfold hyprel_def, safe) |
|
14299 | 278 |
apply (auto intro!: FreeUltrafilterNat_Nat_set) |
279 |
done |
|
280 |
||
14301 | 281 |
lemma hypreal_empty_not_mem [simp]: "{} \<notin> hypreal" |
14299 | 282 |
apply (unfold hypreal_def) |
283 |
apply (auto elim!: quotientE equalityCE) |
|
284 |
done |
|
285 |
||
14301 | 286 |
lemma Rep_hypreal_nonempty [simp]: "Rep_hypreal x \<noteq> {}" |
287 |
by (cut_tac x = x in Rep_hypreal, auto) |
|
14299 | 288 |
|
289 |
||
14329 | 290 |
subsection{*@{term hypreal_of_real}: |
291 |
the Injection from @{typ real} to @{typ hypreal}*} |
|
14299 | 292 |
|
293 |
lemma inj_hypreal_of_real: "inj(hypreal_of_real)" |
|
294 |
apply (rule inj_onI) |
|
295 |
apply (unfold hypreal_of_real_def) |
|
296 |
apply (drule inj_on_Abs_hypreal [THEN inj_onD]) |
|
297 |
apply (rule hyprel_in_hypreal)+ |
|
298 |
apply (drule eq_equiv_class) |
|
299 |
apply (rule equiv_hyprel) |
|
300 |
apply (simp_all add: split: split_if_asm) |
|
301 |
done |
|
302 |
||
303 |
lemma eq_Abs_hypreal: |
|
304 |
"(!!x y. z = Abs_hypreal(hyprel``{x}) ==> P) ==> P" |
|
305 |
apply (rule_tac x1=z in Rep_hypreal [unfolded hypreal_def, THEN quotientE]) |
|
14301 | 306 |
apply (drule_tac f = Abs_hypreal in arg_cong) |
14299 | 307 |
apply (force simp add: Rep_hypreal_inverse) |
308 |
done |
|
309 |
||
14329 | 310 |
|
311 |
subsection{*Hyperreal Addition*} |
|
312 |
||
313 |
lemma hypreal_add_congruent2: |
|
314 |
"congruent2 hyprel (%X Y. hyprel``{%n. X n + Y n})" |
|
315 |
apply (unfold congruent2_def, auto, ultra) |
|
316 |
done |
|
317 |
||
318 |
lemma hypreal_add: |
|
319 |
"Abs_hypreal(hyprel``{%n. X n}) + Abs_hypreal(hyprel``{%n. Y n}) = |
|
320 |
Abs_hypreal(hyprel``{%n. X n + Y n})" |
|
321 |
apply (unfold hypreal_add_def) |
|
322 |
apply (simp add: UN_equiv_class2 [OF equiv_hyprel hypreal_add_congruent2]) |
|
323 |
done |
|
324 |
||
325 |
lemma hypreal_add_commute: "(z::hypreal) + w = w + z" |
|
326 |
apply (rule_tac z = z in eq_Abs_hypreal) |
|
327 |
apply (rule_tac z = w in eq_Abs_hypreal) |
|
14334 | 328 |
apply (simp add: add_ac hypreal_add) |
14329 | 329 |
done |
330 |
||
331 |
lemma hypreal_add_assoc: "((z1::hypreal) + z2) + z3 = z1 + (z2 + z3)" |
|
332 |
apply (rule_tac z = z1 in eq_Abs_hypreal) |
|
333 |
apply (rule_tac z = z2 in eq_Abs_hypreal) |
|
334 |
apply (rule_tac z = z3 in eq_Abs_hypreal) |
|
335 |
apply (simp add: hypreal_add real_add_assoc) |
|
336 |
done |
|
337 |
||
14331 | 338 |
lemma hypreal_add_zero_left: "(0::hypreal) + z = z" |
14329 | 339 |
apply (unfold hypreal_zero_def) |
340 |
apply (rule_tac z = z in eq_Abs_hypreal) |
|
341 |
apply (simp add: hypreal_add) |
|
342 |
done |
|
343 |
||
344 |
instance hypreal :: plus_ac0 |
|
345 |
by (intro_classes, |
|
346 |
(assumption | |
|
347 |
rule hypreal_add_commute hypreal_add_assoc hypreal_add_zero_left)+) |
|
348 |
||
349 |
lemma hypreal_add_zero_right [simp]: "z + (0::hypreal) = z" |
|
350 |
by (simp add: hypreal_add_zero_left hypreal_add_commute) |
|
351 |
||
352 |
||
353 |
subsection{*Additive inverse on @{typ hypreal}*} |
|
14299 | 354 |
|
355 |
lemma hypreal_minus_congruent: |
|
356 |
"congruent hyprel (%X. hyprel``{%n. - (X n)})" |
|
357 |
by (force simp add: congruent_def) |
|
358 |
||
359 |
lemma hypreal_minus: |
|
360 |
"- (Abs_hypreal(hyprel``{%n. X n})) = Abs_hypreal(hyprel `` {%n. -(X n)})" |
|
361 |
apply (unfold hypreal_minus_def) |
|
14301 | 362 |
apply (rule_tac f = Abs_hypreal in arg_cong) |
363 |
apply (simp add: hyprel_in_hypreal [THEN Abs_hypreal_inverse] |
|
14299 | 364 |
UN_equiv_class [OF equiv_hyprel hypreal_minus_congruent]) |
365 |
done |
|
366 |
||
14329 | 367 |
lemma hypreal_diff: |
368 |
"Abs_hypreal(hyprel``{%n. X n}) - Abs_hypreal(hyprel``{%n. Y n}) = |
|
14299 | 369 |
Abs_hypreal(hyprel``{%n. X n - Y n})" |
14301 | 370 |
apply (simp add: hypreal_diff_def hypreal_minus hypreal_add) |
14299 | 371 |
done |
372 |
||
14301 | 373 |
lemma hypreal_add_minus [simp]: "z + -z = (0::hypreal)" |
14299 | 374 |
apply (unfold hypreal_zero_def) |
14301 | 375 |
apply (rule_tac z = z in eq_Abs_hypreal) |
14299 | 376 |
apply (simp add: hypreal_minus hypreal_add) |
377 |
done |
|
378 |
||
14331 | 379 |
lemma hypreal_add_minus_left: "-z + z = (0::hypreal)" |
14301 | 380 |
by (simp add: hypreal_add_commute hypreal_add_minus) |
14299 | 381 |
|
14329 | 382 |
|
383 |
subsection{*Hyperreal Multiplication*} |
|
14299 | 384 |
|
385 |
lemma hypreal_mult_congruent2: |
|
386 |
"congruent2 hyprel (%X Y. hyprel``{%n. X n * Y n})" |
|
14301 | 387 |
apply (unfold congruent2_def, auto, ultra) |
14299 | 388 |
done |
389 |
||
390 |
lemma hypreal_mult: |
|
391 |
"Abs_hypreal(hyprel``{%n. X n}) * Abs_hypreal(hyprel``{%n. Y n}) = |
|
392 |
Abs_hypreal(hyprel``{%n. X n * Y n})" |
|
393 |
apply (unfold hypreal_mult_def) |
|
394 |
apply (simp add: UN_equiv_class2 [OF equiv_hyprel hypreal_mult_congruent2]) |
|
395 |
done |
|
396 |
||
397 |
lemma hypreal_mult_commute: "(z::hypreal) * w = w * z" |
|
14301 | 398 |
apply (rule_tac z = z in eq_Abs_hypreal) |
399 |
apply (rule_tac z = w in eq_Abs_hypreal) |
|
14331 | 400 |
apply (simp add: hypreal_mult mult_ac) |
14299 | 401 |
done |
402 |
||
403 |
lemma hypreal_mult_assoc: "((z1::hypreal) * z2) * z3 = z1 * (z2 * z3)" |
|
14301 | 404 |
apply (rule_tac z = z1 in eq_Abs_hypreal) |
405 |
apply (rule_tac z = z2 in eq_Abs_hypreal) |
|
406 |
apply (rule_tac z = z3 in eq_Abs_hypreal) |
|
14331 | 407 |
apply (simp add: hypreal_mult mult_assoc) |
14299 | 408 |
done |
409 |
||
14331 | 410 |
lemma hypreal_mult_1: "(1::hypreal) * z = z" |
14299 | 411 |
apply (unfold hypreal_one_def) |
14301 | 412 |
apply (rule_tac z = z in eq_Abs_hypreal) |
14299 | 413 |
apply (simp add: hypreal_mult) |
414 |
done |
|
14301 | 415 |
|
14329 | 416 |
lemma hypreal_add_mult_distrib: |
417 |
"((z1::hypreal) + z2) * w = (z1 * w) + (z2 * w)" |
|
14301 | 418 |
apply (rule_tac z = z1 in eq_Abs_hypreal) |
419 |
apply (rule_tac z = z2 in eq_Abs_hypreal) |
|
420 |
apply (rule_tac z = w in eq_Abs_hypreal) |
|
14334 | 421 |
apply (simp add: hypreal_mult hypreal_add left_distrib) |
14299 | 422 |
done |
423 |
||
14331 | 424 |
text{*one and zero are distinct*} |
14299 | 425 |
lemma hypreal_zero_not_eq_one: "0 \<noteq> (1::hypreal)" |
426 |
apply (unfold hypreal_zero_def hypreal_one_def) |
|
427 |
apply (auto simp add: real_zero_not_eq_one) |
|
428 |
done |
|
429 |
||
430 |
||
14329 | 431 |
subsection{*Multiplicative Inverse on @{typ hypreal} *} |
14299 | 432 |
|
433 |
lemma hypreal_inverse_congruent: |
|
434 |
"congruent hyprel (%X. hyprel``{%n. if X n = 0 then 0 else inverse(X n)})" |
|
435 |
apply (unfold congruent_def) |
|
14301 | 436 |
apply (auto, ultra) |
14299 | 437 |
done |
438 |
||
439 |
lemma hypreal_inverse: |
|
440 |
"inverse (Abs_hypreal(hyprel``{%n. X n})) = |
|
441 |
Abs_hypreal(hyprel `` {%n. if X n = 0 then 0 else inverse(X n)})" |
|
442 |
apply (unfold hypreal_inverse_def) |
|
14301 | 443 |
apply (rule_tac f = Abs_hypreal in arg_cong) |
444 |
apply (simp add: hyprel_in_hypreal [THEN Abs_hypreal_inverse] |
|
14299 | 445 |
UN_equiv_class [OF equiv_hyprel hypreal_inverse_congruent]) |
446 |
done |
|
447 |
||
14331 | 448 |
lemma hypreal_mult_inverse: |
14299 | 449 |
"x \<noteq> 0 ==> x*inverse(x) = (1::hypreal)" |
450 |
apply (unfold hypreal_one_def hypreal_zero_def) |
|
14301 | 451 |
apply (rule_tac z = x in eq_Abs_hypreal) |
14299 | 452 |
apply (simp add: hypreal_inverse hypreal_mult) |
453 |
apply (drule FreeUltrafilterNat_Compl_mem) |
|
14334 | 454 |
apply (blast intro!: right_inverse FreeUltrafilterNat_subset) |
14299 | 455 |
done |
456 |
||
14331 | 457 |
lemma hypreal_mult_inverse_left: |
14329 | 458 |
"x \<noteq> 0 ==> inverse(x)*x = (1::hypreal)" |
14301 | 459 |
by (simp add: hypreal_mult_inverse hypreal_mult_commute) |
14299 | 460 |
|
14331 | 461 |
instance hypreal :: field |
462 |
proof |
|
463 |
fix x y z :: hypreal |
|
464 |
show "(x + y) + z = x + (y + z)" by (rule hypreal_add_assoc) |
|
465 |
show "x + y = y + x" by (rule hypreal_add_commute) |
|
466 |
show "0 + x = x" by simp |
|
467 |
show "- x + x = 0" by (simp add: hypreal_add_minus_left) |
|
468 |
show "x - y = x + (-y)" by (simp add: hypreal_diff_def) |
|
469 |
show "(x * y) * z = x * (y * z)" by (rule hypreal_mult_assoc) |
|
470 |
show "x * y = y * x" by (rule hypreal_mult_commute) |
|
471 |
show "1 * x = x" by (simp add: hypreal_mult_1) |
|
472 |
show "(x + y) * z = x * z + y * z" by (simp add: hypreal_add_mult_distrib) |
|
473 |
show "0 \<noteq> (1::hypreal)" by (rule hypreal_zero_not_eq_one) |
|
474 |
show "x \<noteq> 0 ==> inverse x * x = 1" by (simp add: hypreal_mult_inverse_left) |
|
475 |
show "y \<noteq> 0 ==> x / y = x * inverse y" by (simp add: hypreal_divide_def) |
|
14341
a09441bd4f1e
Ring_and_Field now requires axiom add_left_imp_eq for semirings.
paulson
parents:
14334
diff
changeset
|
476 |
assume eq: "z+x = z+y" |
a09441bd4f1e
Ring_and_Field now requires axiom add_left_imp_eq for semirings.
paulson
parents:
14334
diff
changeset
|
477 |
hence "(-z + z) + x = (-z + z) + y" by (simp only: eq hypreal_add_assoc) |
a09441bd4f1e
Ring_and_Field now requires axiom add_left_imp_eq for semirings.
paulson
parents:
14334
diff
changeset
|
478 |
thus "x = y" by (simp add: hypreal_add_minus_left) |
14331 | 479 |
qed |
480 |
||
481 |
||
482 |
lemma HYPREAL_INVERSE_ZERO: "inverse 0 = (0::hypreal)" |
|
483 |
by (simp add: hypreal_inverse hypreal_zero_def) |
|
484 |
||
485 |
lemma HYPREAL_DIVISION_BY_ZERO: "a / (0::hypreal) = 0" |
|
486 |
by (simp add: hypreal_divide_def HYPREAL_INVERSE_ZERO |
|
487 |
hypreal_mult_commute [of a]) |
|
488 |
||
489 |
instance hypreal :: division_by_zero |
|
490 |
proof |
|
491 |
fix x :: hypreal |
|
492 |
show "inverse 0 = (0::hypreal)" by (rule HYPREAL_INVERSE_ZERO) |
|
493 |
show "x/0 = 0" by (rule HYPREAL_DIVISION_BY_ZERO) |
|
494 |
qed |
|
495 |
||
14329 | 496 |
|
497 |
subsection{*Theorems for Ordering*} |
|
498 |
||
499 |
text{*TODO: define @{text "\<le>"} as the primitive concept and quickly |
|
500 |
establish membership in class @{text linorder}. Then proofs could be |
|
501 |
simplified, since properties of @{text "<"} would be generic.*} |
|
14299 | 502 |
|
14329 | 503 |
text{*TODO: The following theorem should be used througout the proofs |
504 |
as it probably makes many of them more straightforward.*} |
|
505 |
lemma hypreal_less: |
|
506 |
"(Abs_hypreal(hyprel``{%n. X n}) < Abs_hypreal(hyprel``{%n. Y n})) = |
|
507 |
({n. X n < Y n} \<in> FreeUltrafilterNat)" |
|
508 |
apply (unfold hypreal_less_def) |
|
509 |
apply (auto intro!: lemma_hyprel_refl, ultra) |
|
14299 | 510 |
done |
511 |
||
512 |
lemma hypreal_less_not_refl: "~ (R::hypreal) < R" |
|
14301 | 513 |
apply (rule_tac z = R in eq_Abs_hypreal) |
514 |
apply (auto simp add: hypreal_less_def, ultra) |
|
14299 | 515 |
done |
516 |
||
517 |
lemmas hypreal_less_irrefl = hypreal_less_not_refl [THEN notE, standard] |
|
518 |
declare hypreal_less_irrefl [elim!] |
|
519 |
||
520 |
lemma hypreal_not_refl2: "!!(x::hypreal). x < y ==> x \<noteq> y" |
|
14301 | 521 |
by (auto simp add: hypreal_less_not_refl) |
14299 | 522 |
|
523 |
lemma hypreal_less_trans: "!!(R1::hypreal). [| R1 < R2; R2 < R3 |] ==> R1 < R3" |
|
14301 | 524 |
apply (rule_tac z = R1 in eq_Abs_hypreal) |
525 |
apply (rule_tac z = R2 in eq_Abs_hypreal) |
|
526 |
apply (rule_tac z = R3 in eq_Abs_hypreal) |
|
527 |
apply (auto intro!: exI simp add: hypreal_less_def, ultra) |
|
14299 | 528 |
done |
529 |
||
530 |
lemma hypreal_less_asym: "!! (R1::hypreal). [| R1 < R2; R2 < R1 |] ==> P" |
|
14301 | 531 |
apply (drule hypreal_less_trans, assumption) |
14299 | 532 |
apply (simp add: hypreal_less_not_refl) |
533 |
done |
|
534 |
||
535 |
||
14329 | 536 |
subsection{*Trichotomy: the hyperreals are Linearly Ordered*} |
14299 | 537 |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
538 |
lemma lemma_hyprel_0_mem: "\<exists>x. x \<in> hyprel `` {%n. 0}" |
14299 | 539 |
apply (unfold hyprel_def) |
14301 | 540 |
apply (rule_tac x = "%n. 0" in exI, safe) |
14299 | 541 |
apply (auto intro!: FreeUltrafilterNat_Nat_set) |
542 |
done |
|
543 |
||
544 |
lemma hypreal_trichotomy: "0 < x | x = 0 | x < (0::hypreal)" |
|
545 |
apply (unfold hypreal_zero_def) |
|
14301 | 546 |
apply (rule_tac z = x in eq_Abs_hypreal) |
14299 | 547 |
apply (auto simp add: hypreal_less_def) |
14301 | 548 |
apply (cut_tac lemma_hyprel_0_mem, erule exE) |
549 |
apply (drule_tac x = xa in spec) |
|
550 |
apply (drule_tac x = x in spec) |
|
551 |
apply (cut_tac x = x in lemma_hyprel_refl, auto) |
|
552 |
apply (drule_tac x = x in spec) |
|
553 |
apply (drule_tac x = xa in spec, auto, ultra) |
|
14299 | 554 |
done |
555 |
||
556 |
lemma hypreal_trichotomyE: |
|
557 |
"[| (0::hypreal) < x ==> P; |
|
558 |
x = 0 ==> P; |
|
559 |
x < 0 ==> P |] ==> P" |
|
14301 | 560 |
apply (insert hypreal_trichotomy [of x], blast) |
14299 | 561 |
done |
562 |
||
563 |
lemma hypreal_less_minus_iff: "((x::hypreal) < y) = (0 < y + -x)" |
|
14301 | 564 |
apply (rule_tac z = x in eq_Abs_hypreal) |
565 |
apply (rule_tac z = y in eq_Abs_hypreal) |
|
14299 | 566 |
apply (auto simp add: hypreal_add hypreal_zero_def hypreal_minus hypreal_less) |
567 |
done |
|
568 |
||
569 |
lemma hypreal_less_minus_iff2: "((x::hypreal) < y) = (x + -y < 0)" |
|
14301 | 570 |
apply (rule_tac z = x in eq_Abs_hypreal) |
571 |
apply (rule_tac z = y in eq_Abs_hypreal) |
|
14299 | 572 |
apply (auto simp add: hypreal_add hypreal_zero_def hypreal_minus hypreal_less) |
573 |
done |
|
574 |
||
575 |
lemma hypreal_eq_minus_iff2: "((x::hypreal) = y) = (0 = y + - x)" |
|
576 |
apply auto |
|
14331 | 577 |
apply (rule Ring_and_Field.add_right_cancel [of _ "-x", THEN iffD1], auto) |
14299 | 578 |
done |
579 |
||
580 |
lemma hypreal_linear: "(x::hypreal) < y | x = y | y < x" |
|
581 |
apply (subst hypreal_eq_minus_iff2) |
|
14301 | 582 |
apply (rule_tac x1 = x in hypreal_less_minus_iff [THEN ssubst]) |
583 |
apply (rule_tac x1 = y in hypreal_less_minus_iff2 [THEN ssubst]) |
|
584 |
apply (rule hypreal_trichotomyE, auto) |
|
14299 | 585 |
done |
586 |
||
587 |
lemma hypreal_neq_iff: "((w::hypreal) \<noteq> z) = (w<z | z<w)" |
|
14301 | 588 |
by (cut_tac hypreal_linear, blast) |
14299 | 589 |
|
14329 | 590 |
|
591 |
subsection{*Properties of The @{text "\<le>"} Relation*} |
|
14299 | 592 |
|
593 |
lemma hypreal_le: |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
594 |
"(Abs_hypreal(hyprel``{%n. X n}) \<le> Abs_hypreal(hyprel``{%n. Y n})) = |
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
595 |
({n. X n \<le> Y n} \<in> FreeUltrafilterNat)" |
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
596 |
apply (auto simp add: hypreal_less hypreal_le_def linorder_not_less[symmetric]) |
14299 | 597 |
apply (ultra+) |
598 |
done |
|
599 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
600 |
lemma hypreal_le_imp_less_or_eq: "!!(x::hypreal). x \<le> y ==> x < y | x = y" |
14299 | 601 |
apply (unfold hypreal_le_def) |
602 |
apply (cut_tac hypreal_linear) |
|
603 |
apply (fast elim: hypreal_less_irrefl hypreal_less_asym) |
|
604 |
done |
|
605 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
606 |
lemma hypreal_less_or_eq_imp_le: "z<w | z=w ==> z \<le>(w::hypreal)" |
14299 | 607 |
apply (unfold hypreal_le_def) |
608 |
apply (cut_tac hypreal_linear) |
|
609 |
apply (fast elim: hypreal_less_irrefl hypreal_less_asym) |
|
610 |
done |
|
611 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
612 |
lemma hypreal_le_eq_less_or_eq: "(x \<le> (y::hypreal)) = (x < y | x=y)" |
14299 | 613 |
by (blast intro!: hypreal_less_or_eq_imp_le dest: hypreal_le_imp_less_or_eq) |
614 |
||
615 |
lemmas hypreal_le_less = hypreal_le_eq_less_or_eq |
|
616 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
617 |
lemma hypreal_le_refl: "w \<le> (w::hypreal)" |
14301 | 618 |
by (simp add: hypreal_le_eq_less_or_eq) |
14299 | 619 |
|
620 |
(* Axiom 'linorder_linear' of class 'linorder': *) |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
621 |
lemma hypreal_le_linear: "(z::hypreal) \<le> w | w \<le> z" |
14301 | 622 |
apply (simp add: hypreal_le_less) |
623 |
apply (cut_tac hypreal_linear, blast) |
|
14299 | 624 |
done |
625 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
626 |
lemma hypreal_le_trans: "[| i \<le> j; j \<le> k |] ==> i \<le> (k::hypreal)" |
14299 | 627 |
apply (drule hypreal_le_imp_less_or_eq) |
628 |
apply (drule hypreal_le_imp_less_or_eq) |
|
629 |
apply (rule hypreal_less_or_eq_imp_le) |
|
630 |
apply (blast intro: hypreal_less_trans) |
|
631 |
done |
|
632 |
||
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
633 |
lemma hypreal_le_anti_sym: "[| z \<le> w; w \<le> z |] ==> z = (w::hypreal)" |
14299 | 634 |
apply (drule hypreal_le_imp_less_or_eq) |
635 |
apply (drule hypreal_le_imp_less_or_eq) |
|
636 |
apply (fast elim: hypreal_less_irrefl hypreal_less_asym) |
|
637 |
done |
|
638 |
||
639 |
(* Axiom 'order_less_le' of class 'order': *) |
|
14365
3d4df8c166ae
replacing HOL/Real/PRat, PNat by the rational number development
paulson
parents:
14361
diff
changeset
|
640 |
lemma hypreal_less_le: "((w::hypreal) < z) = (w \<le> z & w \<noteq> z)" |
14301 | 641 |
apply (simp add: hypreal_le_def hypreal_neq_iff) |
14299 | 642 |
apply (blast intro: hypreal_less_asym) |
643 |
done |
|
644 |
||
14329 | 645 |
instance hypreal :: order |
646 |
by (intro_classes, |
|
647 |
(assumption | |
|
648 |
rule hypreal_le_refl hypreal_le_trans hypreal_le_anti_sym |
|
649 |
hypreal_less_le)+) |
|
650 |
||
651 |
instance hypreal :: linorder |
|
652 |
by (intro_classes, rule hypreal_le_linear) |
|
653 |
||
654 |
||
655 |
lemma hypreal_add_less_mono1: "(A::hypreal) < B ==> A + C < B + C" |
|
656 |
apply (rule_tac z = A in eq_Abs_hypreal) |
|
657 |
apply (rule_tac z = B in eq_Abs_hypreal) |
|
658 |
apply (rule_tac z = C in eq_Abs_hypreal) |
|
659 |
apply (auto intro!: exI simp add: hypreal_less_def hypreal_add, ultra) |
|
660 |
done |
|
661 |
||
662 |
lemma hypreal_mult_order: "[| 0 < x; 0 < y |] ==> (0::hypreal) < x * y" |
|
663 |
apply (unfold hypreal_zero_def) |
|
664 |
apply (rule_tac z = x in eq_Abs_hypreal) |
|
665 |
apply (rule_tac z = y in eq_Abs_hypreal) |
|
666 |
apply (auto intro!: exI simp add: hypreal_less_def hypreal_mult, ultra) |
|
667 |
apply (auto intro: real_mult_order) |
|
668 |
done |
|
669 |
||
670 |
lemma hypreal_add_left_le_mono1: "(q1::hypreal) \<le> q2 ==> x + q1 \<le> x + q2" |
|
671 |
apply (drule order_le_imp_less_or_eq) |
|
672 |
apply (auto intro: order_less_imp_le hypreal_add_less_mono1 simp add: hypreal_add_commute) |
|
673 |
done |
|
674 |
||
675 |
lemma hypreal_mult_less_mono1: "[| (0::hypreal) < z; x < y |] ==> x*z < y*z" |
|
676 |
apply (rotate_tac 1) |
|
677 |
apply (drule hypreal_less_minus_iff [THEN iffD1]) |
|
678 |
apply (rule hypreal_less_minus_iff [THEN iffD2]) |
|
679 |
apply (drule hypreal_mult_order, assumption) |
|
14331 | 680 |
apply (simp add: right_distrib hypreal_mult_commute) |
14329 | 681 |
done |
682 |
||
683 |
lemma hypreal_mult_less_mono2: "[| (0::hypreal)<z; x<y |] ==> z*x<z*y" |
|
684 |
apply (simp (no_asm_simp) add: hypreal_mult_commute hypreal_mult_less_mono1) |
|
685 |
done |
|
686 |
||
687 |
subsection{*The Hyperreals Form an Ordered Field*} |
|
688 |
||
689 |
instance hypreal :: ordered_field |
|
690 |
proof |
|
691 |
fix x y z :: hypreal |
|
14348
744c868ee0b7
Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents:
14341
diff
changeset
|
692 |
show "0 < (1::hypreal)" |
744c868ee0b7
Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents:
14341
diff
changeset
|
693 |
by (unfold hypreal_one_def hypreal_zero_def hypreal_less_def, force) |
744c868ee0b7
Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents:
14341
diff
changeset
|
694 |
show "x \<le> y ==> z + x \<le> z + y" |
744c868ee0b7
Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents:
14341
diff
changeset
|
695 |
by (rule hypreal_add_left_le_mono1) |
744c868ee0b7
Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents:
14341
diff
changeset
|
696 |
show "x < y ==> 0 < z ==> z * x < z * y" |
744c868ee0b7
Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents:
14341
diff
changeset
|
697 |
by (simp add: hypreal_mult_less_mono2) |
14329 | 698 |
show "\<bar>x\<bar> = (if x < 0 then -x else x)" |
699 |
by (auto dest: order_le_less_trans simp add: hrabs_def linorder_not_le) |
|
700 |
qed |
|
701 |
||
14331 | 702 |
lemma hypreal_mult_1_right: "z * (1::hypreal) = z" |
703 |
by (rule Ring_and_Field.mult_1_right) |
|
704 |
||
705 |
lemma hypreal_mult_minus_1 [simp]: "(- (1::hypreal)) * z = -z" |
|
706 |
by (simp) |
|
707 |
||
708 |
lemma hypreal_mult_minus_1_right [simp]: "z * (- (1::hypreal)) = -z" |
|
709 |
by (subst hypreal_mult_commute, simp) |
|
14329 | 710 |
|
711 |
(*Used ONCE: in NSA.ML*) |
|
712 |
lemma hypreal_minus_distrib1: "-(y + -(x::hypreal)) = x + -y" |
|
713 |
by (simp add: hypreal_add_commute) |
|
714 |
||
715 |
(*Used ONCE: in Lim.ML*) |
|
716 |
lemma hypreal_eq_minus_iff3: "(x = y + z) = (x + -z = (y::hypreal))" |
|
717 |
by (auto simp add: hypreal_add_assoc) |
|
718 |
||
14331 | 719 |
lemma hypreal_eq_minus_iff: "((x::hypreal) = y) = (x + - y = 0)" |
720 |
apply auto |
|
721 |
apply (rule Ring_and_Field.add_right_cancel [of _ "-y", THEN iffD1], auto) |
|
722 |
done |
|
723 |
||
724 |
(*Used 3 TIMES: in Lim.ML*) |
|
14329 | 725 |
lemma hypreal_not_eq_minus_iff: "(x \<noteq> a) = (x + -a \<noteq> (0::hypreal))" |
726 |
by (auto dest: hypreal_eq_minus_iff [THEN iffD2]) |
|
727 |
||
728 |
lemma hypreal_mult_left_cancel: "(c::hypreal) \<noteq> 0 ==> (c*a=c*b) = (a=b)" |
|
729 |
apply auto |
|
730 |
done |
|
731 |
||
732 |
lemma hypreal_mult_right_cancel: "(c::hypreal) \<noteq> 0 ==> (a*c=b*c) = (a=b)" |
|
733 |
apply auto |
|
734 |
done |
|
735 |
||
736 |
lemma hypreal_inverse_not_zero: "x \<noteq> 0 ==> inverse (x::hypreal) \<noteq> 0" |
|
737 |
by (rule Ring_and_Field.nonzero_imp_inverse_nonzero) |
|
738 |
||
739 |
lemma hypreal_mult_not_0: "[| x \<noteq> 0; y \<noteq> 0 |] ==> x * y \<noteq> (0::hypreal)" |
|
740 |
by simp |
|
741 |
||
742 |
lemma hypreal_minus_inverse: "inverse(-x) = -inverse(x::hypreal)" |
|
743 |
by (rule Ring_and_Field.inverse_minus_eq) |
|
744 |
||
745 |
lemma hypreal_inverse_distrib: "inverse(x*y) = inverse(x)*inverse(y::hypreal)" |
|
746 |
by (rule Ring_and_Field.inverse_mult_distrib) |
|
747 |
||
748 |
||
749 |
subsection{* Division lemmas *} |
|
750 |
||
751 |
lemma hypreal_divide_one: "x/(1::hypreal) = x" |
|
752 |
by (simp add: hypreal_divide_def) |
|
753 |
||
754 |
||
755 |
(** As with multiplication, pull minus signs OUT of the / operator **) |
|
756 |
||
757 |
lemma hypreal_add_divide_distrib: "(x+y)/(z::hypreal) = x/z + y/z" |
|
758 |
by (rule Ring_and_Field.add_divide_distrib) |
|
759 |
||
760 |
lemma hypreal_inverse_add: |
|
761 |
"[|(x::hypreal) \<noteq> 0; y \<noteq> 0 |] |
|
762 |
==> inverse(x) + inverse(y) = (x + y)*inverse(x*y)" |
|
763 |
by (simp add: Ring_and_Field.inverse_add mult_assoc) |
|
764 |
||
765 |
||
766 |
subsection{*@{term hypreal_of_real} Preserves Field and Order Properties*} |
|
767 |
||
14301 | 768 |
lemma hypreal_of_real_add [simp]: |
14369 | 769 |
"hypreal_of_real (w + z) = hypreal_of_real w + hypreal_of_real z" |
14299 | 770 |
apply (unfold hypreal_of_real_def) |
14331 | 771 |
apply (simp add: hypreal_add left_distrib) |
14299 | 772 |
done |
773 |
||
14301 | 774 |
lemma hypreal_of_real_mult [simp]: |
14369 | 775 |
"hypreal_of_real (w * z) = hypreal_of_real w * hypreal_of_real z" |
14299 | 776 |
apply (unfold hypreal_of_real_def) |
14331 | 777 |
apply (simp add: hypreal_mult right_distrib) |
14299 | 778 |
done |
779 |
||
14301 | 780 |
lemma hypreal_of_real_one [simp]: "hypreal_of_real 1 = (1::hypreal)" |
781 |
by (unfold hypreal_of_real_def hypreal_one_def, simp) |
|
14299 | 782 |
|
14301 | 783 |
lemma hypreal_of_real_zero [simp]: "hypreal_of_real 0 = 0" |
784 |
by (unfold hypreal_of_real_def hypreal_zero_def, simp) |
|
14299 | 785 |
|
14369 | 786 |
lemma hypreal_of_real_less_iff [simp]: |
787 |
"(hypreal_of_real w < hypreal_of_real z) = (w < z)" |
|
788 |
apply (unfold hypreal_less_def hypreal_of_real_def, auto) |
|
789 |
apply (rule_tac [2] x = "%n. w" in exI, safe) |
|
790 |
apply (rule_tac [3] x = "%n. z" in exI, auto) |
|
791 |
apply (rule FreeUltrafilterNat_P, ultra) |
|
792 |
done |
|
793 |
||
794 |
lemma hypreal_of_real_le_iff [simp]: |
|
795 |
"(hypreal_of_real w \<le> hypreal_of_real z) = (w \<le> z)" |
|
796 |
by (force simp add: hypreal_less hypreal_le_def linorder_not_less[symmetric]) |
|
797 |
||
798 |
lemma hypreal_of_real_eq_iff [simp]: |
|
799 |
"(hypreal_of_real w = hypreal_of_real z) = (w = z)" |
|
800 |
by (force intro: order_antisym hypreal_of_real_le_iff [THEN iffD1]) |
|
801 |
||
802 |
text{*As above, for 0*} |
|
803 |
||
804 |
declare hypreal_of_real_less_iff [of 0, simplified, simp] |
|
805 |
declare hypreal_of_real_le_iff [of 0, simplified, simp] |
|
806 |
declare hypreal_of_real_eq_iff [of 0, simplified, simp] |
|
807 |
||
808 |
declare hypreal_of_real_less_iff [of _ 0, simplified, simp] |
|
809 |
declare hypreal_of_real_le_iff [of _ 0, simplified, simp] |
|
810 |
declare hypreal_of_real_eq_iff [of _ 0, simplified, simp] |
|
811 |
||
812 |
text{*As above, for 1*} |
|
813 |
||
814 |
declare hypreal_of_real_less_iff [of 1, simplified, simp] |
|
815 |
declare hypreal_of_real_le_iff [of 1, simplified, simp] |
|
816 |
declare hypreal_of_real_eq_iff [of 1, simplified, simp] |
|
817 |
||
818 |
declare hypreal_of_real_less_iff [of _ 1, simplified, simp] |
|
819 |
declare hypreal_of_real_le_iff [of _ 1, simplified, simp] |
|
820 |
declare hypreal_of_real_eq_iff [of _ 1, simplified, simp] |
|
821 |
||
822 |
lemma hypreal_of_real_minus [simp]: |
|
823 |
"hypreal_of_real (-r) = - hypreal_of_real r" |
|
824 |
apply (unfold hypreal_of_real_def) |
|
825 |
apply (auto simp add: hypreal_minus) |
|
826 |
done |
|
14299 | 827 |
|
14329 | 828 |
lemma hypreal_of_real_inverse [simp]: |
829 |
"hypreal_of_real (inverse r) = inverse (hypreal_of_real r)" |
|
14299 | 830 |
apply (case_tac "r=0") |
14301 | 831 |
apply (simp add: DIVISION_BY_ZERO INVERSE_ZERO HYPREAL_INVERSE_ZERO) |
14299 | 832 |
apply (rule_tac c1 = "hypreal_of_real r" in hypreal_mult_left_cancel [THEN iffD1]) |
14369 | 833 |
apply (auto simp add: hypreal_of_real_mult [symmetric]) |
14299 | 834 |
done |
835 |
||
14329 | 836 |
lemma hypreal_of_real_divide [simp]: |
14369 | 837 |
"hypreal_of_real (w / z) = hypreal_of_real w / hypreal_of_real z" |
14301 | 838 |
by (simp add: hypreal_divide_def real_divide_def) |
14299 | 839 |
|
840 |
||
14329 | 841 |
subsection{*Misc Others*} |
14299 | 842 |
|
843 |
lemma hypreal_zero_num: "0 = Abs_hypreal (hyprel `` {%n. 0})" |
|
14301 | 844 |
by (simp add: hypreal_zero_def [THEN meta_eq_to_obj_eq, symmetric]) |
14299 | 845 |
|
846 |
lemma hypreal_one_num: "1 = Abs_hypreal (hyprel `` {%n. 1})" |
|
14301 | 847 |
by (simp add: hypreal_one_def [THEN meta_eq_to_obj_eq, symmetric]) |
14299 | 848 |
|
14301 | 849 |
lemma hypreal_omega_gt_zero [simp]: "0 < omega" |
14299 | 850 |
apply (unfold omega_def) |
851 |
apply (auto simp add: hypreal_less hypreal_zero_num) |
|
852 |
done |
|
853 |
||
14329 | 854 |
|
855 |
lemma hypreal_hrabs: |
|
856 |
"abs (Abs_hypreal (hyprel `` {X})) = |
|
857 |
Abs_hypreal(hyprel `` {%n. abs (X n)})" |
|
858 |
apply (auto simp add: hrabs_def hypreal_zero_def hypreal_le hypreal_minus) |
|
859 |
apply (ultra, arith)+ |
|
860 |
done |
|
861 |
||
14299 | 862 |
ML |
863 |
{* |
|
14329 | 864 |
val hrabs_def = thm "hrabs_def"; |
865 |
val hypreal_hrabs = thm "hypreal_hrabs"; |
|
866 |
||
14299 | 867 |
val hypreal_zero_def = thm "hypreal_zero_def"; |
868 |
val hypreal_one_def = thm "hypreal_one_def"; |
|
869 |
val hypreal_minus_def = thm "hypreal_minus_def"; |
|
870 |
val hypreal_diff_def = thm "hypreal_diff_def"; |
|
871 |
val hypreal_inverse_def = thm "hypreal_inverse_def"; |
|
872 |
val hypreal_divide_def = thm "hypreal_divide_def"; |
|
873 |
val hypreal_of_real_def = thm "hypreal_of_real_def"; |
|
874 |
val omega_def = thm "omega_def"; |
|
875 |
val epsilon_def = thm "epsilon_def"; |
|
876 |
val hypreal_add_def = thm "hypreal_add_def"; |
|
877 |
val hypreal_mult_def = thm "hypreal_mult_def"; |
|
878 |
val hypreal_less_def = thm "hypreal_less_def"; |
|
879 |
val hypreal_le_def = thm "hypreal_le_def"; |
|
880 |
||
881 |
val finite_exhausts = thm "finite_exhausts"; |
|
882 |
val finite_not_covers = thm "finite_not_covers"; |
|
883 |
val not_finite_nat = thm "not_finite_nat"; |
|
884 |
val FreeUltrafilterNat_Ex = thm "FreeUltrafilterNat_Ex"; |
|
885 |
val FreeUltrafilterNat_mem = thm "FreeUltrafilterNat_mem"; |
|
886 |
val FreeUltrafilterNat_finite = thm "FreeUltrafilterNat_finite"; |
|
887 |
val FreeUltrafilterNat_not_finite = thm "FreeUltrafilterNat_not_finite"; |
|
888 |
val FreeUltrafilterNat_empty = thm "FreeUltrafilterNat_empty"; |
|
889 |
val FreeUltrafilterNat_Int = thm "FreeUltrafilterNat_Int"; |
|
890 |
val FreeUltrafilterNat_subset = thm "FreeUltrafilterNat_subset"; |
|
891 |
val FreeUltrafilterNat_Compl = thm "FreeUltrafilterNat_Compl"; |
|
892 |
val FreeUltrafilterNat_Compl_mem = thm "FreeUltrafilterNat_Compl_mem"; |
|
893 |
val FreeUltrafilterNat_Compl_iff1 = thm "FreeUltrafilterNat_Compl_iff1"; |
|
894 |
val FreeUltrafilterNat_Compl_iff2 = thm "FreeUltrafilterNat_Compl_iff2"; |
|
895 |
val FreeUltrafilterNat_UNIV = thm "FreeUltrafilterNat_UNIV"; |
|
896 |
val FreeUltrafilterNat_Nat_set = thm "FreeUltrafilterNat_Nat_set"; |
|
897 |
val FreeUltrafilterNat_Nat_set_refl = thm "FreeUltrafilterNat_Nat_set_refl"; |
|
898 |
val FreeUltrafilterNat_P = thm "FreeUltrafilterNat_P"; |
|
899 |
val FreeUltrafilterNat_Ex_P = thm "FreeUltrafilterNat_Ex_P"; |
|
900 |
val FreeUltrafilterNat_all = thm "FreeUltrafilterNat_all"; |
|
901 |
val FreeUltrafilterNat_Un = thm "FreeUltrafilterNat_Un"; |
|
902 |
val hyprel_iff = thm "hyprel_iff"; |
|
903 |
val hyprel_refl = thm "hyprel_refl"; |
|
904 |
val hyprel_sym = thm "hyprel_sym"; |
|
905 |
val hyprel_trans = thm "hyprel_trans"; |
|
906 |
val equiv_hyprel = thm "equiv_hyprel"; |
|
907 |
val hyprel_in_hypreal = thm "hyprel_in_hypreal"; |
|
908 |
val Abs_hypreal_inverse = thm "Abs_hypreal_inverse"; |
|
909 |
val inj_on_Abs_hypreal = thm "inj_on_Abs_hypreal"; |
|
910 |
val inj_Rep_hypreal = thm "inj_Rep_hypreal"; |
|
911 |
val lemma_hyprel_refl = thm "lemma_hyprel_refl"; |
|
912 |
val hypreal_empty_not_mem = thm "hypreal_empty_not_mem"; |
|
913 |
val Rep_hypreal_nonempty = thm "Rep_hypreal_nonempty"; |
|
914 |
val inj_hypreal_of_real = thm "inj_hypreal_of_real"; |
|
915 |
val eq_Abs_hypreal = thm "eq_Abs_hypreal"; |
|
916 |
val hypreal_minus_congruent = thm "hypreal_minus_congruent"; |
|
917 |
val hypreal_minus = thm "hypreal_minus"; |
|
918 |
val hypreal_add_congruent2 = thm "hypreal_add_congruent2"; |
|
919 |
val hypreal_add = thm "hypreal_add"; |
|
920 |
val hypreal_diff = thm "hypreal_diff"; |
|
921 |
val hypreal_add_commute = thm "hypreal_add_commute"; |
|
922 |
val hypreal_add_assoc = thm "hypreal_add_assoc"; |
|
923 |
val hypreal_add_zero_left = thm "hypreal_add_zero_left"; |
|
924 |
val hypreal_add_zero_right = thm "hypreal_add_zero_right"; |
|
925 |
val hypreal_add_minus = thm "hypreal_add_minus"; |
|
926 |
val hypreal_add_minus_left = thm "hypreal_add_minus_left"; |
|
927 |
val hypreal_minus_distrib1 = thm "hypreal_minus_distrib1"; |
|
928 |
val hypreal_mult_congruent2 = thm "hypreal_mult_congruent2"; |
|
929 |
val hypreal_mult = thm "hypreal_mult"; |
|
930 |
val hypreal_mult_commute = thm "hypreal_mult_commute"; |
|
931 |
val hypreal_mult_assoc = thm "hypreal_mult_assoc"; |
|
932 |
val hypreal_mult_1 = thm "hypreal_mult_1"; |
|
933 |
val hypreal_mult_1_right = thm "hypreal_mult_1_right"; |
|
934 |
val hypreal_mult_minus_1 = thm "hypreal_mult_minus_1"; |
|
935 |
val hypreal_mult_minus_1_right = thm "hypreal_mult_minus_1_right"; |
|
936 |
val hypreal_zero_not_eq_one = thm "hypreal_zero_not_eq_one"; |
|
937 |
val hypreal_inverse_congruent = thm "hypreal_inverse_congruent"; |
|
938 |
val hypreal_inverse = thm "hypreal_inverse"; |
|
939 |
val HYPREAL_INVERSE_ZERO = thm "HYPREAL_INVERSE_ZERO"; |
|
940 |
val HYPREAL_DIVISION_BY_ZERO = thm "HYPREAL_DIVISION_BY_ZERO"; |
|
941 |
val hypreal_mult_inverse = thm "hypreal_mult_inverse"; |
|
942 |
val hypreal_mult_inverse_left = thm "hypreal_mult_inverse_left"; |
|
943 |
val hypreal_mult_left_cancel = thm "hypreal_mult_left_cancel"; |
|
944 |
val hypreal_mult_right_cancel = thm "hypreal_mult_right_cancel"; |
|
945 |
val hypreal_inverse_not_zero = thm "hypreal_inverse_not_zero"; |
|
946 |
val hypreal_mult_not_0 = thm "hypreal_mult_not_0"; |
|
947 |
val hypreal_minus_inverse = thm "hypreal_minus_inverse"; |
|
948 |
val hypreal_inverse_distrib = thm "hypreal_inverse_distrib"; |
|
949 |
val hypreal_less_not_refl = thm "hypreal_less_not_refl"; |
|
14331 | 950 |
val hypreal_less_irrefl = thm"hypreal_less_irrefl"; |
14299 | 951 |
val hypreal_not_refl2 = thm "hypreal_not_refl2"; |
952 |
val hypreal_less_trans = thm "hypreal_less_trans"; |
|
953 |
val hypreal_less_asym = thm "hypreal_less_asym"; |
|
954 |
val hypreal_less = thm "hypreal_less"; |
|
955 |
val hypreal_trichotomy = thm "hypreal_trichotomy"; |
|
956 |
val hypreal_less_minus_iff = thm "hypreal_less_minus_iff"; |
|
957 |
val hypreal_less_minus_iff2 = thm "hypreal_less_minus_iff2"; |
|
958 |
val hypreal_eq_minus_iff = thm "hypreal_eq_minus_iff"; |
|
959 |
val hypreal_eq_minus_iff2 = thm "hypreal_eq_minus_iff2"; |
|
960 |
val hypreal_eq_minus_iff3 = thm "hypreal_eq_minus_iff3"; |
|
961 |
val hypreal_not_eq_minus_iff = thm "hypreal_not_eq_minus_iff"; |
|
962 |
val hypreal_linear = thm "hypreal_linear"; |
|
963 |
val hypreal_le = thm "hypreal_le"; |
|
964 |
val hypreal_le_imp_less_or_eq = thm "hypreal_le_imp_less_or_eq"; |
|
965 |
val hypreal_le_eq_less_or_eq = thm "hypreal_le_eq_less_or_eq"; |
|
966 |
val hypreal_le_refl = thm "hypreal_le_refl"; |
|
967 |
val hypreal_le_linear = thm "hypreal_le_linear"; |
|
968 |
val hypreal_le_trans = thm "hypreal_le_trans"; |
|
969 |
val hypreal_le_anti_sym = thm "hypreal_le_anti_sym"; |
|
970 |
val hypreal_less_le = thm "hypreal_less_le"; |
|
971 |
val hypreal_of_real_add = thm "hypreal_of_real_add"; |
|
972 |
val hypreal_of_real_mult = thm "hypreal_of_real_mult"; |
|
973 |
val hypreal_of_real_less_iff = thm "hypreal_of_real_less_iff"; |
|
974 |
val hypreal_of_real_le_iff = thm "hypreal_of_real_le_iff"; |
|
975 |
val hypreal_of_real_eq_iff = thm "hypreal_of_real_eq_iff"; |
|
976 |
val hypreal_of_real_minus = thm "hypreal_of_real_minus"; |
|
977 |
val hypreal_of_real_one = thm "hypreal_of_real_one"; |
|
978 |
val hypreal_of_real_zero = thm "hypreal_of_real_zero"; |
|
979 |
val hypreal_of_real_inverse = thm "hypreal_of_real_inverse"; |
|
980 |
val hypreal_of_real_divide = thm "hypreal_of_real_divide"; |
|
981 |
val hypreal_divide_one = thm "hypreal_divide_one"; |
|
982 |
val hypreal_add_divide_distrib = thm "hypreal_add_divide_distrib"; |
|
983 |
val hypreal_inverse_add = thm "hypreal_inverse_add"; |
|
984 |
val hypreal_zero_num = thm "hypreal_zero_num"; |
|
985 |
val hypreal_one_num = thm "hypreal_one_num"; |
|
986 |
val hypreal_omega_gt_zero = thm "hypreal_omega_gt_zero"; |
|
987 |
*} |
|
988 |
||
10751 | 989 |
end |