src/HOLCF/Product_Cpo.thy
changeset 35919 676c6005ad03
parent 35914 91a7311177c4
child 36452 d37c6eed8117
--- a/src/HOLCF/Product_Cpo.thy	Mon Mar 22 21:37:48 2010 -0700
+++ b/src/HOLCF/Product_Cpo.thy	Mon Mar 22 22:41:41 2010 -0700
@@ -84,6 +84,12 @@
 
 text {* @{term fst} and @{term snd} are monotone *}
 
+lemma fst_monofun: "x \<sqsubseteq> y \<Longrightarrow> fst x \<sqsubseteq> fst y"
+unfolding below_prod_def by simp
+
+lemma snd_monofun: "x \<sqsubseteq> y \<Longrightarrow> snd x \<sqsubseteq> snd y"
+unfolding below_prod_def by simp
+
 lemma monofun_fst: "monofun fst"
 by (simp add: monofun_def below_prod_def)