src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy
changeset 58412 f65f11f4854c
parent 58411 e3d0354d2129
child 59720 f893472fff31
equal deleted inserted replaced
58411:e3d0354d2129 58412:f65f11f4854c
   296   let
   296   let
   297     val thy = Proof_Context.theory_of ctxt
   297     val thy = Proof_Context.theory_of ctxt
   298     val pannot = TPTP_Reconstruct.get_pannot_of_prob thy prob_name
   298     val pannot = TPTP_Reconstruct.get_pannot_of_prob thy prob_name
   299   in
   299   in
   300     #meta pannot
   300     #meta pannot
   301     |> List.filter (fn (_, info) =>
   301     |> filter (fn (_, info) =>
   302         #role info = TPTP_Syntax.Role_Conjecture)
   302         #role info = TPTP_Syntax.Role_Conjecture)
   303     |> hd
   303     |> hd
   304     |> snd |> #fmla
   304     |> snd |> #fmla
   305     |> cterm_of thy
   305     |> cterm_of thy
   306   end;
   306   end;