Quot/QuotOption.thy
changeset 925 8d51795ef54d
parent 923 0419b20ee83c
child 927 04ef4bd3b936
child 932 7781c7cbd27e
--- 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 = \<equiv> op ="
+  shows "option_rel (op =) \<equiv> (op =)"
   apply(rule eq_reflection)
   apply(auto simp add: expand_fun_eq)
   apply(case_tac x)