| author | nipkow | 
| Mon, 09 Feb 2009 18:50:10 +0100 | |
| changeset 29849 | a2baf1b221be | 
| parent 29820 | 07f53494cf20 | 
| child 29888 | ab97183f1694 | 
| permissions | -rw-r--r-- | 
| 12024 | 1 | header {* Main HOL *}
 | 
| 2 | ||
| 15131 | 3 | theory Main | 
| 29820 
07f53494cf20
Rearrange Refute/SAT theory dependencies so as to use even more antiquotations in refute.ML +
 blanchet parents: 
29304diff
changeset | 4 | imports Plain Code_Eval Map Nat_Int_Bij Recdef SAT | 
| 15131 | 5 | begin | 
| 9650 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 6 | |
| 29304 | 7 | text {*
 | 
| 8 | Classical Higher-order Logic -- only ``Main'', excluding real and | |
| 9 | complex numbers etc. | |
| 10 | *} | |
| 11 | ||
| 27367 | 12 | text {* See further \cite{Nipkow-et-al:2002:tutorial} *}
 | 
| 25964 | 13 | |
| 9650 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 14 | end |