src/HOL/Tools/Sledgehammer/sledgehammer_fact_preprocessor.ML
changeset 37403 7e3d7af86215
parent 37399 34f080a12063
child 37410 2bf7e6136047
equal deleted inserted replaced
37402:12cb33916e37 37403:7e3d7af86215
   396     []
   396     []
   397   else
   397   else
   398     let
   398     let
   399       val ctxt0 = Variable.global_thm_context th
   399       val ctxt0 = Variable.global_thm_context th
   400       val (nnfth, ctxt) = to_nnf th ctxt0
   400       val (nnfth, ctxt) = to_nnf th ctxt0
       
   401 
       
   402       val inline = false
       
   403 (*
       
   404 FIXME: Reintroduce code:
   401       val inline = exists_type (exists_subtype (can dest_TFree)) (prop_of nnfth)
   405       val inline = exists_type (exists_subtype (can dest_TFree)) (prop_of nnfth)
       
   406 *)
   402       val defs = skolem_theorems_of_assume inline s nnfth
   407       val defs = skolem_theorems_of_assume inline s nnfth
   403       val (cnfs, ctxt) = Meson.make_cnf defs nnfth ctxt
   408       val (cnfs, ctxt) = Meson.make_cnf defs nnfth ctxt
   404     in
   409     in
   405       cnfs |> map introduce_combinators
   410       cnfs |> map introduce_combinators
   406            |> Variable.export ctxt ctxt0
   411            |> Variable.export ctxt ctxt0