| author | wenzelm | 
| Mon, 25 Mar 2019 16:45:08 +0100 | |
| changeset 69980 | f2e3adfd916f | 
| parent 64267 | b9a1486e79be | 
| permissions | -rw-r--r-- | 
| 62480 | 1 | (* Title: HOL/Nonstandard_Analysis/Nonstandard_Analysis.thy | 
| 2 | Author: Jacques D. Fleuriot, University of Cambridge | |
| 3 | Author: Lawrence C Paulson, University of Cambridge | |
| 4 | Author: Brian Huffman | |
| 5 | ||
| 6 | Nonstandard analysis. | |
| 7 | *) | |
| 8 | ||
| 9 | theory Nonstandard_Analysis | |
| 10 | imports Hypercomplex | |
| 11 | begin | |
| 12 | ||
| 64267 | 13 | end |