src/FOLP/ROOT
author wenzelm
Sat, 01 Jun 2019 11:29:59 +0200
changeset 70299 83774d669b51
parent 69319 baccaf89ca0d
child 75992 1f6d79b62222
permissions -rw-r--r--
Added tag Isabelle2019-RC4 for changeset ad2d84c42380

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.
  "
  theories
    IFOLP (global)
    FOLP (global)

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.
  "
  theories
    Intro
    Nat
    Foundation
    If
    Intuitionistic
    Classical
    Propositional_Int
    Quantifiers_Int
    Propositional_Cla
    Quantifiers_Cla