src/HOL/BNF_Def.thy
changeset 55945 e96383acecf9
parent 55811 aa1acc25126b
child 56635 b07c8ad23010
--- a/src/HOL/BNF_Def.thy	Thu Mar 06 15:29:18 2014 +0100
+++ b/src/HOL/BNF_Def.thy	Thu Mar 06 15:40:33 2014 +0100
@@ -140,8 +140,8 @@
 lemma vimage2pI: "R (f x) (g y) \<Longrightarrow> vimage2p f g R x y"
   unfolding vimage2p_def by -
 
-lemma fun_rel_iff_leq_vimage2p: "(fun_rel R S) f g = (R \<le> vimage2p f g S)"
-  unfolding fun_rel_def vimage2p_def by auto
+lemma rel_fun_iff_leq_vimage2p: "(rel_fun R S) f g = (R \<le> vimage2p f g S)"
+  unfolding rel_fun_def vimage2p_def by auto
 
 lemma convol_image_vimage2p: "<f o fst, g o snd> ` Collect (split (vimage2p f g R)) \<subseteq> Collect (split R)"
   unfolding vimage2p_def convol_def by auto