src/HOL/Fun.thy
changeset 22577 1a08fce38565
parent 22453 530db8c36f53
child 22744 5cbe966d67a2
--- a/src/HOL/Fun.thy	Tue Apr 03 19:31:48 2007 +0200
+++ b/src/HOL/Fun.thy	Wed Apr 04 00:10:59 2007 +0200
@@ -579,7 +579,7 @@
     simp_tac (Simplifier.inherit_context ss current_ss) 1
 in
   val fun_upd2_simproc =
-    Simplifier.simproc (Theory.sign_of (the_context ()))
+    Simplifier.simproc @{theory}
       "fun_upd2" ["f(v := w, x := y)"]
       (fn _ => fn ss => fn t =>
         case find_double t of (T, NONE) => NONE