| author | blanchet | 
| Fri, 01 Aug 2014 15:08:49 +0200 | |
| changeset 57838 | c21f2c52f54b | 
| parent 51525 | d3d170a2887f | 
| permissions | -rw-r--r-- | 
| 28952 
15a4b2cf8c34
made repository layout more coherent with logical distribution structure; stripped some $Id$s
 haftmann parents: 
27468diff
changeset | 1 | (* Title: HOL/NSA/Hyperreal.thy | 
| 27468 | 2 | Author: Jacques Fleuriot, Cambridge University Computer Laboratory | 
| 3 | Copyright 1998 University of Cambridge | |
| 4 | ||
| 5 | Construction of the Hyperreals by the Ultrapower Construction | |
| 6 | and mechanization of Nonstandard Real Analysis | |
| 7 | *) | |
| 8 | ||
| 9 | theory Hyperreal | |
| 51525 | 10 | imports HLog | 
| 27468 | 11 | begin | 
| 12 | ||
| 13 | end |