src/HOL/Fun.thy
changeset 55990 41c6b99c5fb7
parent 55467 a5c9002bc54d
child 56015 57e2cfba9c6e
--- a/src/HOL/Fun.thy	Fri Mar 07 22:19:52 2014 +0100
+++ b/src/HOL/Fun.thy	Fri Mar 07 22:30:58 2014 +0100
@@ -895,7 +895,7 @@
           SOME (Goal.prove ctxt [] [] (Logic.mk_equals (t, rhs))
             (fn _ =>
               rtac eq_reflection 1 THEN
-              rtac ext 1 THEN
+              rtac @{thm ext} 1 THEN
               simp_tac (put_simpset ss ctxt) 1))
     end
 in proc end