src/HOL/ROOT
author wenzelm
Tue, 24 Jul 2012 12:38:33 +0200
changeset 48470 7483aa690b4f
parent 48458 09710d6fc3d1
child 48481 2c828c830ad7
permissions -rw-r--r--
clarified "document" again, eliminated redundant "no_document";

session HOL! (1) in "." = Pure +
  description {* Classical Higher-order Logic *}
  options [document_graph]
  theories Complex_Main
  files "document/root.tex" "document/root.bib"

session "HOL-Base"! in "." = Pure +
  description {* Raw HOL base, with minimal tools *}
  options [document = false]
  theories HOL

session "HOL-Plain"! in "." = Pure +
  description {* HOL side-entry after bootstrap of many tools and packages *}
  options [document = false]
  theories Plain

session "HOL-Main"! in "." = Pure +
  description {* HOL side-entry for Main only, without Complex_Main *}
  options [document = false]
  theories Main

session "HOL-Proofs"! (2) in "." = Pure +
  description {* HOL-Main with proof terms *}
  options [document = false, proofs = 2, parallel_proofs = 0]
  theories Main

session HOLCF! (3) = HOL +
  description {*
    Author:     Franz Regensburger
    Author:     Brian Huffman

    HOLCF -- a semantic extension of HOL by the LCF logic.
  *}
  options [document_graph]
  theories [document = false]
    "~~/src/HOL/Library/Nat_Bijection"
    "~~/src/HOL/Library/Countable"
  theories Plain_HOLCF Fixrec HOLCF
  files "document/root.tex"