src/FOL/FOL.thy
author wenzelm
Sat, 04 Apr 1998 12:28:39 +0200
changeset 4793 03fd006fb97b
parent 4093 5e8f3d57dee7
child 4854 d1850e0964f2
permissions -rw-r--r--
replaced thy_data by thy_setup;


FOL = IFOL +

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

end

ML val thy_setup = [ClasetThyData.setup];