src/FOL/fol.thy
author nipkow
Mon, 21 Oct 1996 09:51:18 +0200
changeset 2116 73bbf2cc7651
parent 0 a5a9c433f639
permissions -rw-r--r--
Used trans_tac (see Provers/nat_transitive.ML) to automate arithmetic.

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