src/HOLCF/Cfun.thy
changeset 16314 7102a1aaecfd
parent 16209 36ee7f6af79f
child 16386 c6f5ade29608
--- a/src/HOLCF/Cfun.thy	Tue Jun 07 20:04:41 2005 +0200
+++ b/src/HOLCF/Cfun.thy	Wed Jun 08 00:04:38 2005 +0200
@@ -336,6 +336,14 @@
 apply simp
 done
 
+lemma injection_less:
+  "\<forall>x. f\<cdot>(g\<cdot>x) = x \<Longrightarrow> (g\<cdot>x \<sqsubseteq> g\<cdot>y) = (x \<sqsubseteq> y)"
+apply (rule iffI)
+apply (drule_tac f=f in monofun_cfun_arg)
+apply simp
+apply (erule monofun_cfun_arg)
+done
+
 lemma injection_defined_rev:
   "\<lbrakk>\<forall>x. f\<cdot>(g\<cdot>x) = x; g\<cdot>z = \<bottom>\<rbrakk> \<Longrightarrow> z = \<bottom>"
 apply (drule_tac f=f in cfun_arg_cong)