fixed embarrassing bug where conjecture and fact offsets were swapped
authorblanchet
Sun, 01 May 2011 18:37:25 +0200
changeset 42585 723b9d1e8ba5
parent 42584 8121a31b6754
child 42586 59e0ca92bb0b
fixed embarrassing bug where conjecture and fact offsets were swapped
src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML	Sun May 01 18:37:25 2011 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML	Sun May 01 18:37:25 2011 +0200
@@ -898,8 +898,8 @@
   in
     (problem,
      case pool of SOME the_pool => snd the_pool | NONE => Symtab.empty,
+     offset_of_heading_in_problem conjsN problem 0,
      offset_of_heading_in_problem factsN problem 0,
-     offset_of_heading_in_problem conjsN problem 0,
      fact_names |> Vector.fromList)
   end