src/FOL/FOL.thy
author oheimb
Wed, 25 Feb 1998 20:25:27 +0100
changeset 4652 d24cca140eeb
parent 4093 5e8f3d57dee7
child 4793 03fd006fb97b
permissions -rw-r--r--
factored out common code of HOL/simpdata.ML and FOL/simpdata.ML concerning combination of classical reasoner and simplifier auto_tac into Provers/clasimp.ML explicitly introducing combined type clasimpset


FOL = IFOL +

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

end

ML val thy_data = [ClasetThyData.thy_data];