src/FOL/fol.thy
author wenzelm
Wed, 19 Jan 1994 14:21:26 +0100
changeset 237 a7d3e712767a
parent 0 a5a9c433f639
permissions -rw-r--r--
MAJOR INTERNAL CHANGE: extend and merge operations of syntax tables now much leaner (eliminated gramgraph, all data except tables of old parser are shared); simplified the internal interfaces for syntax extension;

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