src/HOL/HOL.thy
changeset 51798 ad3a241def73
parent 51717 9e7d1c139569
child 52143 36ffe23b25f8
--- a/src/HOL/HOL.thy	Sat Apr 27 11:37:50 2013 +0200
+++ b/src/HOL/HOL.thy	Sat Apr 27 20:50:20 2013 +0200
@@ -849,15 +849,15 @@
 let
   fun non_bool_eq (@{const_name HOL.eq}, Type (_, [T, _])) = T <> @{typ bool}
     | non_bool_eq _ = false;
-  val hyp_subst_tac' =
+  fun hyp_subst_tac' ctxt =
     SUBGOAL (fn (goal, i) =>
       if Term.exists_Const non_bool_eq goal
-      then Hypsubst.hyp_subst_tac i
+      then Hypsubst.hyp_subst_tac ctxt i
       else no_tac);
 in
   Hypsubst.hypsubst_setup
   (*prevent substitution on bool*)
-  #> Context_Rules.addSWrapper (fn tac => hyp_subst_tac' ORELSE' tac)
+  #> Context_Rules.addSWrapper (fn ctxt => fn tac => hyp_subst_tac' ctxt ORELSE' tac)
 end
 *}