src/FOL/FOL.thy
author paulson
Thu, 06 Nov 1997 10:29:37 +0100
changeset 4179 cc4b6791d5dc
parent 4093 5e8f3d57dee7
child 4793 03fd006fb97b
permissions -rw-r--r--
hyp_subst_tac checks if the equality has type variables and uses a suitable method if so. Affects the dest_eq function


FOL = IFOL +

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

end

ML val thy_data = [ClasetThyData.thy_data];