src/HOL/Main.thy
author wenzelm
Thu, 07 Jul 2011 23:55:15 +0200
changeset 44572 91c4d7397f0e
parent 43565 a94ad372b2f5
child 45195 d972b91ed09d
permissions -rw-r--r--
simplified make_option/dest_option;
added make_variant/dest_variant -- usual representation of datatypes;
     1 header {* Main HOL *}
     2 
     3 theory Main
     4 imports Plain Predicate_Compile Nitpick
     5 begin
     6 
     7 text {*
     8   Classical Higher-order Logic -- only ``Main'', excluding real and
     9   complex numbers etc.
    10 *}
    11 
    12 text {* See further \cite{Nipkow-et-al:2002:tutorial} *}
    13 
    14 end