src/FOL/FOL.thy
changeset 42456 13b4b6ba3593
parent 42455 6702c984bf5a
child 42459 38b9f023cc34
equal deleted inserted replaced
42455:6702c984bf5a 42456:13b4b6ba3593
   305 
   305 
   306 
   306 
   307 use "simpdata.ML"
   307 use "simpdata.ML"
   308 
   308 
   309 simproc_setup defined_Ex ("EX x. P(x)") = {*
   309 simproc_setup defined_Ex ("EX x. P(x)") = {*
   310   fn _ => fn ss => fn ct => Quantifier1.rearrange_ex (theory_of_cterm ct) ss (term_of ct)
   310   fn _ => fn ss => Quantifier1.rearrange_ex ss o term_of
   311 *}
   311 *}
   312 
   312 
   313 simproc_setup defined_All ("ALL x. P(x)") = {*
   313 simproc_setup defined_All ("ALL x. P(x)") = {*
   314   fn _ => fn ss => fn ct => Quantifier1.rearrange_all (theory_of_cterm ct) ss (term_of ct)
   314   fn _ => fn ss => Quantifier1.rearrange_all ss o term_of
   315 *}
   315 *}
   316 
   316 
   317 ML {*
   317 ML {*
   318 (*intuitionistic simprules only*)
   318 (*intuitionistic simprules only*)
   319 val IFOL_ss =
   319 val IFOL_ss =