diff -r 91c374abde06 -r f7569f994195 QuotMain.thy --- a/QuotMain.thy Thu Dec 03 15:03:31 2009 +0100 +++ b/QuotMain.thy Thu Dec 03 19:06:14 2009 +0100 @@ -741,6 +741,7 @@ CHANGED o (simp_tac ((Simplifier.context ctxt empty_ss) addsimps @{thms id_simps}))]) *} + lemma FUN_REL_I: assumes a: "\x y. R1 x y \ R2 (f x) (g y)" shows "(R1 ===> R2) f g"