diff -r 91c374abde06 -r fac6069d8e80 QuotMain.thy --- a/QuotMain.thy Thu Dec 03 15:03:31 2009 +0100 +++ b/QuotMain.thy Fri Dec 04 08:18:38 2009 +0100 @@ -957,7 +957,7 @@ (* (op =) ===> (op =) \ (op =), needed in order to apply respectfulness theorems *) (* global simplification *) - NDT ctxt "H" (CHANGED o (asm_full_simp_tac ((Simplifier.context ctxt empty_ss) addsimps @{thms eq_reflection[OF 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] eq_reflection[OF LIST_REL_EQ]})))]) *} ML {*