src/FOL/FOL.thy
author oheimb
Wed, 12 Aug 1998 16:21:18 +0200
changeset 5304 c133f16febc7
parent 4854 d1850e0964f2
child 5887 0864c6578d16
permissions -rw-r--r--
the splitter is now defined as a functor moved addsplits, delsplits, Addsplits, Delsplits to Provers/splitter.ML moved split_thm_info to Provers/splitter.ML definined atomize via general mk_atomize removed superfluous rot_eq_tac from simplifier.ML HOL/simpdata.ML: renamed mk_meta_eq to meta_eq, re-renamed mk_meta_eq_simp to mk_meta_eq added Eps_eq to simpset


FOL = IFOL +

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

setup
  ClasetThyData.setup

end