src/FOL/FOL.thy
author wenzelm
Mon, 16 Nov 1998 11:11:42 +0100
changeset 5887 0864c6578d16
parent 4854 d1850e0964f2
child 7355 4c43090659ca
permissions -rw-r--r--
attrib_setup;


FOL = IFOL +

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

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

end