| author | huffman | 
| Mon, 02 Oct 2006 21:30:05 +0200 | |
| changeset 20830 | 65ba80cae6df | 
| parent 17635 | 9234108fdfb1 | 
| child 22983 | 3314057c3b57 | 
| permissions | -rw-r--r-- | 
| 13958 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 1 | (* Title: HOL/Hyperreal/Hyperreal.thy | 
| 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 2 | ID: $Id$ | 
| 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 3 | Author: Jacques Fleuriot, Cambridge University Computer Laboratory | 
| 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 4 | Copyright 1998 University of Cambridge | 
| 10751 | 5 | |
| 13958 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 6 | Construction of the Hyperreals by the Ultrapower Construction | 
| 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 7 | and mechanization of Nonstandard Real Analysis | 
| 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 8 | *) | 
| 
c1c67582c9b5
New material on integration, etc.  Moving Hyperreal/ex
 paulson parents: 
12224diff
changeset | 9 | |
| 15131 | 10 | theory Hyperreal | 
| 17635 | 11 | imports Poly Taylor HLog | 
| 15131 | 12 | begin | 
| 10751 | 13 | |
| 14 | end |