author | wenzelm |
Sat, 30 Dec 2006 16:08:06 +0100 | |
changeset 21966 | edab0ecfbd7c |
parent 21254 | d53f76357f41 |
child 22840 | 643bb625a2c3 |
permissions | -rw-r--r-- |
(* Title: HOL/Main.thy ID: $Id$ *) header {* Main HOL *} theory Main imports SAT ATP_Linkup 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 ATP_Linkup}. *} setup ResAxioms.setup end