src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy
changeset 69366 b6dacf6eabe3
parent 67399 eab6ce8368fa
child 70923 98d9b78b7f47
equal deleted inserted replaced
69365:c5b3860d29ef 69366:b6dacf6eabe3
    56   |> Path.explode
    56   |> Path.explode
    57   |> single
    57   |> single
    58 
    58 
    59 val prob_names =
    59 val prob_names =
    60   probs
    60   probs
    61   |> map (Path.base_name #> TPTP_Problem_Name.Nonstandard)
    61   |> map (Path.file_name #> TPTP_Problem_Name.Nonstandard)
    62 \<close>
    62 \<close>
    63 
    63 
    64 setup \<open>
    64 setup \<open>
    65   if test_all @{context} then I
    65   if test_all @{context} then I
    66   else
    66   else
   574   info about the inferences for which reconstruction failed.*)
   574   info about the inferences for which reconstruction failed.*)
   575 fun test_partial_reconstruction thy prob_file =
   575 fun test_partial_reconstruction thy prob_file =
   576   let
   576   let
   577     val prob_name =
   577     val prob_name =
   578       prob_file
   578       prob_file
   579       |> Path.base_name
   579       |> Path.file_name
   580       |> TPTP_Problem_Name.Nonstandard
   580       |> TPTP_Problem_Name.Nonstandard
   581 
   581 
   582     val thy' =
   582     val thy' =
   583       try
   583       try
   584        (TPTP_Reconstruct.import_thm
   584        (TPTP_Reconstruct.import_thm
   658          file leo2_on_load thy
   658          file leo2_on_load thy
   659 
   659 
   660       val ctxt = Proof_Context.init_global thy' (*FIXME pass ctxt instead of thy*)
   660       val ctxt = Proof_Context.init_global thy' (*FIXME pass ctxt instead of thy*)
   661       val prob_name =
   661       val prob_name =
   662         file
   662         file
   663         |> Path.base_name
   663         |> Path.file_name
   664         |> TPTP_Problem_Name.Nonstandard
   664         |> TPTP_Problem_Name.Nonstandard
   665     in
   665     in
   666       Timeout.apply (Time.fromSeconds (if timeout = 0 then 60 else timeout))
   666       Timeout.apply (Time.fromSeconds (if timeout = 0 then 60 else timeout))
   667        (fn prob_name =>
   667        (fn prob_name =>
   668         (can
   668         (can