diff -r dd58f13a8eb4 -r eb85850d3eb7 src/HOL/Orderings.thy --- a/src/HOL/Orderings.thy Fri Nov 17 02:19:55 2006 +0100 +++ b/src/HOL/Orderings.thy Fri Nov 17 02:20:03 2006 +0100 @@ -19,23 +19,25 @@ begin notation - less_eq ("op \<^loc><=") - less_eq ("(_/ \<^loc><= _)" [51, 51] 50) - less ("op \<^loc><") + less_eq ("op \<^loc><=") and + less_eq ("(_/ \<^loc><= _)" [51, 51] 50) and + less ("op \<^loc><") and less ("(_/ \<^loc>< _)" [51, 51] 50) notation (xsymbols) - less_eq ("op \<^loc>\") + less_eq ("op \<^loc>\") and less_eq ("(_/ \<^loc>\ _)" [51, 51] 50) notation (HTML output) - less_eq ("op \<^loc>\") + less_eq ("op \<^loc>\") and less_eq ("(_/ \<^loc>\ _)" [51, 51] 50) abbreviation (input) - greater (infix "\<^loc>>" 50) + greater (infix "\<^loc>>" 50) where "x \<^loc>> y \ y \<^loc>< x" - greater_eq (infix "\<^loc>>=" 50) + +abbreviation (input) + greater_eq (infix "\<^loc>>=" 50) where "x \<^loc>>= y \ y \<^loc><= x" notation (xsymbols) @@ -44,23 +46,25 @@ end notation - less_eq ("op <=") - less_eq ("(_/ <= _)" [51, 51] 50) - less ("op <") + less_eq ("op <=") and + less_eq ("(_/ <= _)" [51, 51] 50) and + less ("op <") and less ("(_/ < _)" [51, 51] 50) notation (xsymbols) - less_eq ("op \") + less_eq ("op \") and less_eq ("(_/ \ _)" [51, 51] 50) notation (HTML output) - less_eq ("op \") + less_eq ("op \") and less_eq ("(_/ \ _)" [51, 51] 50) abbreviation (input) - greater (infix ">" 50) + greater (infix ">" 50) where "x > y \ y < x" - greater_eq (infix ">=" 50) + +abbreviation (input) + greater_eq (infix ">=" 50) where "x >= y \ y <= x" notation (xsymbols) @@ -78,11 +82,11 @@ begin abbreviation (input) - greater_eq (infixl "\" 50) + greater_eq (infixl "\" 50) where "x \ y \ y \ x" abbreviation (input) - greater (infixl "\" 50) + greater (infixl "\" 50) where "x \ y \ y \ x" text {* Reflexivity. *} @@ -202,8 +206,6 @@ locale linorder = partial_order + assumes linear: "x \ y \ y \ x" - -context linorder begin lemma trichotomy: "x \ y \ x = y \ y \ x" @@ -259,9 +261,11 @@ (* min/max *) definition - min :: "'a \ 'a \ 'a" + min :: "'a \ 'a \ 'a" where "min a b = (if a \ b then a else b)" - max :: "'a \ 'a \ 'a" + +definition + max :: "'a \ 'a \ 'a" where "max a b = (if a \ b then b else a)" lemma min_le_iff_disj: