| author | wenzelm |
| Sun, 05 Nov 2006 21:44:33 +0100 | |
| changeset 21180 | f27f12bcafb8 |
| parent 20414 | 029c4f9dc6f4 |
| child 21254 | d53f76357f41 |
| permissions | -rw-r--r-- |
(* Title: HOL/Main.thy ID: $Id$ *) header {* Main HOL *} theory Main imports SAT Reconstruction ResAtpMethods begin text {* Theory @{text Main} includes everything. Note that theory @{text PreList} already includes most HOL theories. *} text {* \medskip Late clause setup: installs \emph{all} known theorems into the clause cache; cf.\ theory @{text Reconstruction}. *} setup ResAxioms.setup end