don't forget the last inference(s) after conjecture skolemization
authorblanchet
Thu, 30 Jan 2014 17:34:42 +0100
changeset 55186 fafdf2424c57
parent 55185 a0bd8d6414e6
child 55187 6d0d93316daf
child 55191 f127ab7368cf
don't forget the last inference(s) after conjecture skolemization
src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Thu Jan 30 16:40:31 2014 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Thu Jan 30 17:34:42 2014 +0100
@@ -329,7 +329,7 @@
                   [g] =>
                   if skolem andalso is_clause_tainted g then
                     let val subproof = Proof (skolems_of (prop_of_clause g), [], rev accum) in
-                      isar_steps outer (SOME l) [prove [subproof] (no_facts, skolem_methodss)] []
+                      isar_steps outer (SOME l) [prove [subproof] (no_facts, skolem_methodss)] infs
                     end
                   else
                     do_rest l (prove [] by)
@@ -339,8 +339,8 @@
             end
           | isar_steps outer predecessor accum (Cases cases :: infs) =
             let
-              fun isar_case (c, infs) =
-                isar_proof false [] [(label_of_clause c, prop_of_clause c)] [] infs
+              fun isar_case (c, subinfs) =
+                isar_proof false [] [(label_of_clause c, prop_of_clause c)] [] subinfs
               val c = succedent_of_cases cases
               val l = label_of_clause c
               val t = prop_of_clause c