| author | wenzelm | 
| Fri, 07 Jun 2024 15:01:16 +0200 | |
| changeset 80293 | 453eccb886f2 | 
| 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 |