(* Title: HOL/Main.thy ID: $Id$ *) header {* Main HOL *} theory Main imports Plain Map Nat_Int_Bij Recdef begin ML {* val HOL_proofs = ! Proofterm.proofs *} text {* See further \cite{Nipkow-et-al:2002:tutorial} *} end