author | blanchet |
Mon, 09 Aug 2010 12:48:40 +0200 | |
changeset 38286 | c9c7bd836894 |
parent 36899 | bcd6fce5bf06 |
child 38393 | 7c045c03598f |
permissions | -rw-r--r-- |
12024 | 1 |
header {* Main HOL *} |
2 |
||
15131 | 3 |
theory Main |
36899
bcd6fce5bf06
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
boehmes
parents:
35284
diff
changeset
|
4 |
imports Plain Predicate_Compile Nitpick SMT |
15131 | 5 |
begin |
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
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:
9619
diff
changeset
|
14 |
end |