diff -r 6ded9235c2b6 -r ee0a0eb6b738 src/HOL/Orderings.thy --- a/src/HOL/Orderings.thy Fri Sep 28 10:35:53 2007 +0200 +++ b/src/HOL/Orderings.thy Sat Sep 29 08:58:51 2007 +0200 @@ -14,13 +14,18 @@ subsection {* Partial orders *} class order = ord + - assumes less_le: "x \ y \ x \ y \ x \ y" - and order_refl [iff]: "x \ x" - and order_trans: "x \ y \ y \ z \ x \ z" - assumes antisym: "x \ y \ y \ x \ x = y" + assumes less_le: "x \<^loc>< y \ x \<^loc>\ y \ x \ y" + and order_refl [iff]: "x \<^loc>\ x" + and order_trans: "x \<^loc>\ y \ y \<^loc>\ z \ x \<^loc>\ z" + assumes antisym: "x \<^loc>\ y \ y \<^loc>\ x \ x = y" begin +notation (input) + less_eq (infix "\" 50) +and + less (infix "\" 50) + text {* Reflexivity. *} lemma eq_refl: "x = y \ x \<^loc>\ y"