src/HOL/Tools/Predicate_Compile/predicate_compile_proof.ML
changeset 52732 b4da1f2ec73f
parent 52230 1105b3b5aa77
child 54742 7a86358a3c0b
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_proof.ML	Thu Jul 25 16:46:53 2013 +0200
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_proof.ML	Sat Jul 27 16:35:51 2013 +0200
@@ -83,8 +83,7 @@
         let
           val prems' = maps dest_conjunct_prem (take nargs prems)
         in
-          Simplifier.rewrite_goal_tac
-            (map (fn th => th RS @{thm sym} RS @{thm eq_reflection}) prems') 1
+          rewrite_goal_tac (map (fn th => th RS @{thm sym} RS @{thm eq_reflection}) prems') 1
         end) ctxt 1
     | Abs _ => raise Fail "prove_param: No valid parameter term"
   in
@@ -169,7 +168,7 @@
                 let
                   val prems' = maps dest_conjunct_prem (take nargs prems)
                 in
-                  Simplifier.rewrite_goal_tac
+                  rewrite_goal_tac
                     (map (fn th => th RS @{thm sym} RS @{thm eq_reflection}) prems') 1
                 end
              THEN REPEAT_DETERM (rtac @{thm refl} 1))
@@ -210,8 +209,7 @@
               let
                 val prems' = maps dest_conjunct_prem (take nargs prems)
               in
-                Simplifier.rewrite_goal_tac
-                  (map (fn th => th RS @{thm sym} RS @{thm eq_reflection}) prems') 1
+                rewrite_goal_tac (map (fn th => th RS @{thm sym} RS @{thm eq_reflection}) prems') 1
               end) ctxt 1
       THEN (rtac (if null clause_out_ts then @{thm singleI_unit} else @{thm singleI}) 1)
     | prove_prems out_ts ((p, deriv) :: ps) =