src/HOLCF/Porder.thy
changeset 40433 3128c2a54785
parent 40432 61a1519d985f
child 40436 adb22dbb5242
--- a/src/HOLCF/Porder.thy	Wed Nov 03 15:57:39 2010 -0700
+++ b/src/HOLCF/Porder.thy	Wed Nov 03 16:39:23 2010 -0700
@@ -34,19 +34,9 @@
   assumes below_antisym: "x \<sqsubseteq> y \<Longrightarrow> y \<sqsubseteq> x \<Longrightarrow> x = y"
 begin
 
-text {* minimal fixes least element *}
-
-lemma minimal2UU[OF allI] : "\<forall>x. uu \<sqsubseteq> x \<Longrightarrow> uu = (THE u. \<forall>y. u \<sqsubseteq> y)"
-  by (blast intro: theI2 below_antisym)
-
 lemma eq_imp_below: "x = y \<Longrightarrow> x \<sqsubseteq> y"
   by simp
 
-text {* the reverse law of anti-symmetry of @{term "op <<"} *}
-(* Is this rule ever useful? *)
-lemma below_antisym_inverse: "x = y \<Longrightarrow> x \<sqsubseteq> y \<and> y \<sqsubseteq> x"
-  by simp
-
 lemma box_below: "a \<sqsubseteq> b \<Longrightarrow> c \<sqsubseteq> a \<Longrightarrow> b \<sqsubseteq> d \<Longrightarrow> c \<sqsubseteq> d"
   by (rule below_trans [OF below_trans])