| author | wenzelm | 
| Sat, 23 Aug 2008 17:22:53 +0200 | |
| changeset 27952 | 0576c91a6803 | 
| parent 27367 | a75d71c73362 | 
| child 28091 | 50f2d6ba024c | 
| permissions | -rw-r--r-- | 
| 17602 | 1 | (* Title: HOL/Main.thy | 
| 2 | ID: $Id$ | |
| 3 | *) | |
| 9619 | 4 | |
| 12024 | 5 | header {* Main HOL *}
 | 
| 6 | ||
| 15131 | 7 | theory Main | 
| 27367 | 8 | imports Plain Map Presburger Recdef | 
| 15131 | 9 | begin | 
| 9650 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 10 | |
| 25223 | 11 | ML {* val HOL_proofs = ! Proofterm.proofs *}
 | 
| 23165 | 12 | |
| 27367 | 13 | text {* See further \cite{Nipkow-et-al:2002:tutorial} *}
 | 
| 25964 | 14 | |
| 9650 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 15 | end |