src/HOL/HOLCF/Porder.thy
changeset 41182 717404c7d59a
parent 40774 0437dbc127b3
child 42151 4da4fc77664b
--- a/src/HOL/HOLCF/Porder.thy	Wed Dec 15 20:52:20 2010 +0100
+++ b/src/HOL/HOLCF/Porder.thy	Wed Dec 15 19:15:06 2010 -0800
@@ -20,6 +20,13 @@
 notation (xsymbols)
   below (infix "\<sqsubseteq>" 50)
 
+abbreviation
+  not_below :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infix "~<<" 50)
+  where "not_below x y \<equiv> \<not> below x y"
+
+notation (xsymbols)
+  not_below (infix "\<notsqsubseteq>" 50)
+
 lemma below_eq_trans: "\<lbrakk>a \<sqsubseteq> b; b = c\<rbrakk> \<Longrightarrow> a \<sqsubseteq> c"
   by (rule subst)
 
@@ -46,7 +53,7 @@
 lemma rev_below_trans: "y \<sqsubseteq> z \<Longrightarrow> x \<sqsubseteq> y \<Longrightarrow> x \<sqsubseteq> z"
   by (rule below_trans)
 
-lemma not_below2not_eq: "\<not> x \<sqsubseteq> y \<Longrightarrow> x \<noteq> y"
+lemma not_below2not_eq: "x \<notsqsubseteq> y \<Longrightarrow> x \<noteq> y"
   by auto
 
 end