src/FOLP/ROOT
author wenzelm
Thu, 03 Apr 2014 15:40:31 +0200
changeset 56388 c771f0fe28d1
parent 51397 03b586ee5930
child 65527 0d8a7013bf36
permissions -rw-r--r--
more symbol abbrevs, e.g. relevant for list comprehension in HOL/List.thy or HOL/Library/Monad_Syntax.thy;

chapter FOLP

session FOLP = Pure +
  description {*
    Author:     Martin Coen, Cambridge University Computer Laboratory
    Copyright   1993  University of Cambridge

    Modifed version of FOL that contains proof terms.

    Presence of unknown proof term means that matching does not behave as expected.
  *}
  options [document = false]
  theories FOLP

session "FOLP-ex" in ex = FOLP +
  description {*
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1992  University of Cambridge

    Examples for First-Order Logic.
  *}
  options [document = false]
  theories
    Intro
    Nat
    Foundation
    If
    Intuitionistic
    Classical
    Propositional_Int
    Quantifiers_Int
    Propositional_Cla
    Quantifiers_Cla