renamed "formal comments" to "document comments";
tuned section "Markup commands";
updated/tuned section "Document Antiquotations";
(* Title: HOL/Main.thy
ID: $Id$
*)
header {* Main HOL *}
theory Main
imports Plain Code_Eval Map Nat_Int_Bij Recdef
begin
text {* See further \cite{Nipkow-et-al:2002:tutorial} *}
end