src/HOL/Transfer.thy
changeset 47503 cb44d09d9d22
parent 47355 3d9d98e0f1a4
child 47523 1bf0e92c1ca0
--- a/src/HOL/Transfer.thy	Tue Apr 17 09:12:15 2012 +0200
+++ b/src/HOL/Transfer.thy	Tue Apr 17 11:03:08 2012 +0200
@@ -88,6 +88,8 @@
 
 setup Transfer.setup
 
+declare fun_rel_eq [relator_eq]
+
 lemma Rel_App [transfer_raw]:
   assumes "Rel (A ===> B) f g" and "Rel A x y"
   shows "Rel B (App f x) (App g y)"