src/FOL/FOL.thy
author wenzelm
Sun, 25 Oct 1998 12:33:27 +0100
changeset 5769 6a422b22ba02
parent 4854 d1850e0964f2
child 5887 0864c6578d16
permissions -rw-r--r--
tuned checklist;


FOL = IFOL +

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

setup
  ClasetThyData.setup

end