src/HOL/HOL.thy
changeset 33369 470a7b233ee5
parent 33364 2bd12592c5e8
child 33523 96730ad673be
--- a/src/HOL/HOL.thy	Sun Nov 01 15:24:45 2009 +0100
+++ b/src/HOL/HOL.thy	Sun Nov 01 15:44:26 2009 +0100
@@ -853,7 +853,7 @@
       (nth (Thm.prems_of thm) (i - 1)) then Hypsubst.hyp_subst_tac i thm else no_tac thm;
 in
   Hypsubst.hypsubst_setup
-  #> ContextRules.addSWrapper (fn tac => hyp_subst_tac' ORELSE' tac)
+  #> Context_Rules.addSWrapper (fn tac => hyp_subst_tac' ORELSE' tac)
 end
 *}