removing obsolete distinction between prod_case and other case expressions after merging of split and prod_case (d3daea901123) in predicate compiler
authorbulwahn
Wed, 29 Sep 2010 11:55:08 +0200
changeset 39789 533dd8cda12c
parent 39788 9ab014d47c4d
child 39790 b1640def6d44
child 39791 a91430778479
removing obsolete distinction between prod_case and other case expressions after merging of split and prod_case (d3daea901123) in predicate compiler
src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML	Wed Sep 29 11:36:16 2010 +0200
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML	Wed Sep 29 11:55:08 2010 +0200
@@ -178,17 +178,6 @@
               |> maps (fn (res, (names, prems)) =>
                 flatten' (betapply (g, res)) (names, prems))
             end)
-        | Const (@{const_name prod_case}, _) => 
-            (let
-              val (_, g :: res :: args) = strip_comb t
-              val [res1, res2] = Name.variant_list names ["res1", "res2"]
-              val (T1, T2) = HOLogic.dest_prodT (fastype_of res)
-              val (resv1, resv2) = (Free (res1, T1), Free (res2, T2))
-            in
-              flatten' (betapplys (g, (resv1 :: resv2 :: args)))
-              (res1 :: res2 :: names,
-              HOLogic.mk_Trueprop (HOLogic.mk_eq (res, HOLogic.mk_prod (resv1, resv2))) :: prems)
-            end)
         | _ =>
         case find_split_thm thy (fst (strip_comb t)) of
           SOME raw_split_thm =>