diff -r 5455b19ef138 -r 8d51795ef54d Quot/QuotOption.thy --- a/Quot/QuotOption.thy Mon Jan 25 20:35:42 2010 +0100 +++ b/Quot/QuotOption.thy Mon Jan 25 20:47:20 2010 +0100 @@ -82,7 +82,7 @@ done lemma option_rel_eq[id_simps]: - shows "option_rel op = \ op =" + shows "option_rel (op =) \ (op =)" apply(rule eq_reflection) apply(auto simp add: expand_fun_eq) apply(case_tac x)