changeset 452 | 7ba2c16fe0c8 |
parent 451 | 586e3dc4afdb |
child 453 | c22ab554a32d |
--- a/QuotMain.thy Sun Nov 29 08:48:06 2009 +0100 +++ b/QuotMain.thy Sun Nov 29 09:38:07 2009 +0100 @@ -952,7 +952,7 @@ (* (op =) ===> (op =) \<Longrightarrow> (op =), needed in order to apply respectfulness theorems *) (* global simplification *) - NDT ctxt "H" (CHANGED o (asm_full_simp_tac (HOL_ss addsimps @{thms FUN_REL_EQ})))]) + NDT ctxt "H" (CHANGED o (asm_full_simp_tac ((Simplifier.context ctxt empty_ss) addsimps @{thms eq_reflection[OF FUN_REL_EQ]})))]) *} ML {*