type annotations in specifications; fun_rel_def is no simp rule by default
authorhaftmann
Tue, 09 Nov 2010 14:02:12 +0100
changeset 40464 e1db06cf6254
parent 40463 75e544159549
child 40465 2989f9f3aa10
type annotations in specifications; fun_rel_def is no simp rule by default
src/HOL/Library/Quotient_Option.thy
--- a/src/HOL/Library/Quotient_Option.thy	Tue Nov 09 14:02:12 2010 +0100
+++ b/src/HOL/Library/Quotient_Option.thy	Tue Nov 09 14:02:12 2010 +0100
@@ -9,7 +9,7 @@
 begin
 
 fun
-  option_rel
+  option_rel :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a option \<Rightarrow> 'a option \<Rightarrow> bool"
 where
   "option_rel R None None = True"
 | "option_rel R (Some x) None = False"
@@ -56,7 +56,7 @@
 lemma option_Some_rsp[quot_respect]:
   assumes q: "Quotient R Abs Rep"
   shows "(R ===> option_rel R) Some Some"
-  by simp
+  by auto
 
 lemma option_None_prs[quot_preserve]:
   assumes q: "Quotient R Abs Rep"