src/FOL/FOL.thy
author oheimb
Wed, 12 Aug 1998 17:40:18 +0200
changeset 5307 6a699d5cdef4
parent 4854 d1850e0964f2
child 5887 0864c6578d16
permissions -rw-r--r--
minor adaption for SML/NJ


FOL = IFOL +

rules
  classical "(~P ==> P) ==> P"

setup
  ClasetThyData.setup

end