| author | Cezary Kaliszyk <kaliszyk@in.tum.de> | 
| Fri, 04 Dec 2009 08:19:56 +0100 | |
| changeset 509 | d62b6517a0ab | 
| parent 508 | fac6069d8e80 (current diff) | 
| parent 507 | f7569f994195 (diff) | 
| child 510 | 8dbc521ee97f | 
| FSet.thy | file | annotate | diff | comparison | revisions | |
| QuotMain.thy | file | annotate | diff | comparison | revisions | 
--- a/QuotMain.thy Fri Dec 04 08:18:38 2009 +0100 +++ b/QuotMain.thy Fri Dec 04 08:19:56 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: "\<And>x y. R1 x y \<Longrightarrow> R2 (f x) (g y)" shows "(R1 ===> R2) f g"