removed "poly_tags_light_bang" since highly unsound
authorblanchet
Thu, 19 May 2011 10:24:13 +0200
changeset 42851 3bb63850488b
parent 42850 c8709be8a40f
child 42852 40649ab0cead
removed "poly_tags_light_bang" since highly unsound
src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML	Thu May 19 10:24:13 2011 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML	Thu May 19 10:24:13 2011 +0200
@@ -127,20 +127,21 @@
                   | NONE => (NONE, s))
   |> (fn (poly, (level, (heaviness, core))) =>
          case (core, (poly, level, heaviness)) of
-           ("simple_types", (NONE, level, NONE)) => Simple_Types level
-         | ("preds", (SOME Polymorphic, level, _)) =>
+           ("simple_types", (NONE, _, NONE)) => Simple_Types level
+         | ("preds", (SOME Polymorphic, _, _)) =>
            if level = All_Types then
              Preds (Polymorphic, level, heaviness |> the_default Light)
            else
              raise Same.SAME
-         | ("preds", (SOME poly, level, _)) =>
+         | ("preds", (SOME poly, _, _)) =>
            Preds (poly, level, heaviness |> the_default Light)
-         | ("tags", (SOME Polymorphic, level, _)) =>
-           if level = All_Types orelse level = Finite_Types then
-             Tags (Polymorphic, level, heaviness |> the_default Light)
-           else
-             raise Same.SAME
-         | ("tags", (SOME poly, level, _)) =>
+         | ("tags", (SOME Polymorphic, All_Types, _)) =>
+           Tags (Polymorphic, All_Types, heaviness |> the_default Light)
+         | ("tags", (SOME Polymorphic, Finite_Types, _)) =>
+           if heaviness = SOME Light then raise Same.SAME
+           else Tags (Polymorphic, Finite_Types, Heavy)
+         | ("tags", (SOME Polymorphic, _, _)) => raise Same.SAME
+         | ("tags", (SOME poly, _, _)) =>
            Tags (poly, level, heaviness |> the_default Light)
          | ("args", (SOME poly, All_Types (* naja *), NONE)) =>
            Preds (poly, Const_Arg_Types, Light)