src/HOL/Quotient.thy
changeset 36276 92011cc923f5
parent 36215 88ff48884d26
child 37049 ca1c293e521e
--- a/src/HOL/Quotient.thy	Thu Apr 22 09:30:39 2010 +0200
+++ b/src/HOL/Quotient.thy	Thu Apr 22 11:55:19 2010 +0200
@@ -106,6 +106,10 @@
 where
 [simp]: "fun_rel E1 E2 f g = (\<forall>x y. E1 x y \<longrightarrow> E2 (f x) (g y))"
 
+lemma fun_relI [intro]:
+  assumes "\<And>a b. P a b \<Longrightarrow> Q (x a) (y b)"
+  shows "(P ===> Q) x y"
+  using assms by (simp add: fun_rel_def)
 
 lemma fun_map_id:
   shows "(id ---> id) = id"