src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy
changeset 55597 25d7b485df81
parent 55596 928b9f677165
child 56265 785569927666
--- a/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy	Wed Feb 19 15:57:02 2014 +0000
+++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy	Wed Feb 19 15:57:02 2014 +0000
@@ -6,12 +6,30 @@
 NOTE
   - Makes use of the PolyML structure.
   - looks for THF proofs in the path indicated by $THF_PROOFS
+  - these proofs are generated using LEO-II with the following
+    configuration choices: -po 1 -nux -nuc --expand_extuni
+    You can simply filter LEO-II's output using the filter_proof
+    script which is distributed with LEO-II.
 *)
 
 theory TPTP_Proof_Reconstruction_Test
 imports TPTP_Test TPTP_Proof_Reconstruction
 begin
 
+section "Main function"
+text "This function wraps all the reconstruction-related functions. Simply
+ point it at a THF proof produced by LEO-II (using the configuration described
+ above), and it will try to reconstruct it into an Isabelle/HOL theorem.
+ It also returns the theory (into which the axioms and definitions used in the
+ proof have been imported), but note that you can get the theory value from
+ the theorem value."
+
+ML {*
+  reconstruct_leo2 (Path.explode "$THF_PROOFS/NUM667^1.p.out") @{theory}
+*}
+
+section "Prep for testing the component functions"
+
 declare [[
   tptp_trace_reconstruction = false,
   tptp_test_all = false,