# HG changeset patch
# User fleuriot
# Date 970747496 -7200
# Node ID 9d4d5852eb478708f28fbb27444d9a52f95be8ce
# Parent 6263a4a60e38ddf8460a0d6b5dbe3a8527c45f7e
Updated README file for HOL/Real
diff -r 6263a4a60e38 -r 9d4d5852eb47 src/HOL/Real/Hyperreal/Star.ML
--- a/src/HOL/Real/Hyperreal/Star.ML Wed Oct 04 22:21:10 2000 +0200
+++ b/src/HOL/Real/Hyperreal/Star.ML Thu Oct 05 14:04:56 2000 +0200
@@ -492,6 +492,12 @@
by (Fuf_tac 1);
qed "inf_close_FreeUltrafilterNat_iff";
+Goal "inj starfun";
+by (rtac injI 1);
+by (rtac ext 1 THEN rtac ccontr 1);
+by (dres_inst_tac [("x","Abs_hypreal(hyprel ^^{%n. xa})")] fun_cong 1);
+by (auto_tac (claset(),simpset() addsimps [starfun]));
+qed "inj_starfun";
diff -r 6263a4a60e38 -r 9d4d5852eb47 src/HOL/Real/README.html
--- a/src/HOL/Real/README.html Wed Oct 04 22:21:10 2000 +0200
+++ b/src/HOL/Real/README.html Thu Oct 05 14:04:56 2000 +0200
@@ -7,13 +7,71 @@
PNat The positive integers (very much the same as Nat.thy!)
PRat The positive rationals
PReal The positive reals constructed using Dedekind cuts
-Real The real numbers
+RealDef The real numbers
+RealOrd More real numbers theorems- ordering
+properties
+RealInt Embedding of the integers in the reals
+RealBin Binary arithmetic for the reals
+
Lubs Definition of upper bounds, lubs and so on.
(Useful e.g. in Fleuriot's NSA theory)
RComplete Proof of completeness of reals in form of the supremum
property. Also proofs that the reals have the Archimedean
property.
RealAbs The absolute value function defined for the reals
+
+
+Hyperreal--Ultrapower Construction of the Non-Standard Reals
+ See J. D. Fleuriot and L. C. Paulson. Mechanizing Nonstandard
+Real Analysis. LMS J. Computation and Mathematics 3 (2000), 140-190.
+
+
+- Zorn
+Zorn's Lemma: proof based on the ZF version
+
+
- Filter
+Theory of Filters and Ultrafilters.
+Main result is a version of the Ultrafilter Theorem proved using
+Zorn's Lemma.
+
+
- HyperDef
+Ultrapower construction of the hyperreals
+
+
- HyperOrd
+More hyperreal numbers theorems- ordering properties
+
+
- HRealAbs The absolute value function
+defined for the hyperreals
+
+
+
- NSA
+Theory defining sets of infinite numbers, infinitesimals,
+the infinitely close relation, and their various algebraic properties.
+
+
- HyperNat
+Ultrapower construction of the hypernaturals
+
+
- HyperPow
+Powers theory for the hyperreals
+
+
- Star
+Nonstandard extensions of real sets and real functions
+
+
- NatStar
+Nonstandard extensions of sets of naturals and functions on the natural
+numbers
+
+
- SEQ
+Theory of sequences developed using standard and nonstandard analysis
+
+
- Lim
+Theory of limits, continuous functions, and derivatives
+
+
- Series
+Standard theory of finite summation and infinite series
+
+
+
Last modified on $Date$