new lemma flat_less_iff
authorhuffman
Thu, 03 Jan 2008 23:59:51 +0100
changeset 25826 f9aa43287e42
parent 25825 94c075b912ff
child 25827 c2adeb1bae5c
new lemma flat_less_iff
src/HOLCF/Pcpo.thy
--- a/src/HOLCF/Pcpo.thy	Thu Jan 03 23:58:27 2008 +0100
+++ b/src/HOLCF/Pcpo.thy	Thu Jan 03 23:59:51 2008 +0100
@@ -329,6 +329,11 @@
 
 text {* flat subclass of chfin; @{text adm_flat} not needed *}
 
+lemma flat_less_iff:
+  fixes x y :: "'a::flat"
+  shows "(x \<sqsubseteq> y) = (x = \<bottom> \<or> x = y)"
+by (safe dest!: ax_flat [rule_format])
+
 lemma flat_eq: "(a::'a::flat) \<noteq> \<bottom> \<Longrightarrow> a \<sqsubseteq> b = (a = b)"
 by (safe dest!: ax_flat [rule_format])