author | wenzelm |
Sat, 15 Oct 2005 00:08:00 +0200 | |
changeset 17851 | 2fa4f9b54761 |
parent 17721 | b943c01e1c6d |
child 17905 | 1574533861b1 |
permissions | -rw-r--r-- |
(* Title: HOL/Main.thy ID: $Id$ *) header {* Main HOL *} theory Main imports SAT Reconstruction 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} simprules and claset rules into the clause cache; cf.\ theory @{text Reconstruction}. *} setup ResAxioms.clause_setup end