src/HOL/Tools/ATP/atp_problem_generate.ML
changeset 54768 ee0881a54c72
parent 54757 4960647932ec
child 54788 a898e15b522a
equal deleted inserted replaced
54767:81290fe85890 54768:ee0881a54c72
  1956           else
  1956           else
  1957             fact :: reorder [] (facts @ skipped)
  1957             fact :: reorder [] (facts @ skipped)
  1958         end
  1958         end
  1959   in List.partition (curry (op =) Definition o #role) #>> reorder [] #> op @ end
  1959   in List.partition (curry (op =) Definition o #role) #>> reorder [] #> op @ end
  1960 
  1960 
       
  1961 fun s_not_prop (@{const Trueprop} $ t) = @{const Trueprop} $ s_not t
       
  1962   | s_not_prop (@{const "==>"} $ t $ @{prop False}) = t
       
  1963   | s_not_prop t = @{const "==>"} $ t $ @{prop False}
       
  1964 
  1961 fun translate_formulas ctxt prem_role format type_enc lam_trans presimp hyp_ts
  1965 fun translate_formulas ctxt prem_role format type_enc lam_trans presimp hyp_ts
  1962                        concl_t facts =
  1966                        concl_t facts =
  1963   let
  1967   let
  1964     val thy = Proof_Context.theory_of ctxt
  1968     val thy = Proof_Context.theory_of ctxt
  1965     val trans_lams = trans_lams_of_string ctxt type_enc lam_trans
  1969     val trans_lams = trans_lams_of_string ctxt type_enc lam_trans