src/FOL/FOL.thy
author paulson
Fri, 21 May 1999 10:47:07 +0200
changeset 6674 32892a8ecb15
parent 5887 0864c6578d16
child 7355 4c43090659ca
permissions -rw-r--r--
deleted some vestigal theorems (use the equivalents on HOL/Ord.ML)


FOL = IFOL +

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

setup ClasetThyData.setup
setup attrib_setup              (* FIXME move to IFOL.thy *)

end