src/HOL/Product_Type.thy
changeset 50107 289181e3e524
parent 50104 de19856feb54
child 51173 3cbb4e95a565
--- a/src/HOL/Product_Type.thy	Sat Nov 17 17:42:19 2012 +0100
+++ b/src/HOL/Product_Type.thy	Sat Nov 17 17:55:52 2012 +0100
@@ -407,7 +407,6 @@
 
 ML {*
   (* replace parameters of product type by individual component parameters *)
-  val safe_full_simp_tac = generic_simp_tac true (true, false, false);
   local (* filtering with exists_paired_all is an essential optimization *)
     fun exists_paired_all (Const ("all", _) $ Abs (_, T, t)) =
           can HOLogic.dest_prodT T orelse exists_paired_all t
@@ -423,7 +422,7 @@
     val unsafe_split_all_tac = SUBGOAL (fn (t, i) =>
       if exists_paired_all t then full_simp_tac ss i else no_tac);
     fun split_all th =
-   if exists_paired_all (Thm.prop_of th) then full_simplify ss th else th;
+      if exists_paired_all (Thm.prop_of th) then full_simplify ss th else th;
   end;
 *}