src/FOL/FOL.thy
author oheimb
Wed, 12 Nov 1997 18:58:50 +0100
changeset 4223 f60e3d2c81d3
parent 4093 5e8f3d57dee7
child 4793 03fd006fb97b
permissions -rw-r--r--
added thin_refl to hyp_subst_tac


FOL = IFOL +

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

end

ML val thy_data = [ClasetThyData.thy_data];