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

FOL = IFOL +
rules
classical "(~P ==> P) ==> P"
end