src/HOL/HOL.thy
changeset 52230 1105b3b5aa77
parent 52143 36ffe23b25f8
child 52432 c03090937c3b
--- a/src/HOL/HOL.thy	Thu May 30 08:27:51 2013 +0200
+++ b/src/HOL/HOL.thy	Thu May 30 12:35:40 2013 +0200
@@ -1499,8 +1499,7 @@
                 in if is_conj P then SOME @{thm induct_conj_curry} else NONE end
               | _ => NONE))]
     |> Simplifier.set_mksimps (fn ss => Simpdata.mksimps Simpdata.mksimps_pairs ss #>
-      map (Simplifier.rewrite_rule (map Thm.symmetric
-        @{thms induct_rulify_fallback})))))
+      map (rewrite_rule (map Thm.symmetric @{thms induct_rulify_fallback})))))
 *}
 
 text {* Pre-simplification of induction and cases rules *}