diff -r 73ae4f643d57 -r f53ea84bab23 src/HOL/Ord.thy --- a/src/HOL/Ord.thy Thu Feb 15 16:07:57 2001 +0100 +++ b/src/HOL/Ord.thy Thu Feb 15 16:12:27 2001 +0100 @@ -25,8 +25,8 @@ local syntax (symbols) - "op <=" :: "['a::ord, 'a] => bool" ("op \\") - "op <=" :: "['a::ord, 'a] => bool" ("(_/ \\ _)" [50, 51] 50) + "op <=" :: "['a::ord, 'a] => bool" ("op \") + "op <=" :: "['a::ord, 'a] => bool" ("(_/ \ _)" [50, 51] 50) (*Tell Blast_tac about overloading of < and <= to reduce the risk of its applying a rule for the wrong type*) @@ -87,7 +87,7 @@ "LEAST x WRT m. P" == "LeastM m (%x. P)" lemma LeastMI2: "[| P x; !!y. P y ==> m x <= m y; - !!x. [| P x; \\y. P y \\ m x \\ m y |] ==> Q x + !!x. [| P x; \y. P y --> m x \ m y |] ==> Q x |] ==> Q (LeastM m P)"; apply (unfold LeastM_def) apply (rule someI2_ex) @@ -334,10 +334,10 @@ "_leEx" :: "[idt, 'a, bool] => bool" ("(3EX _<=_./ _)" [0, 0, 10] 10) syntax (symbols) - "_lessAll" :: "[idt, 'a, bool] => bool" ("(3\\_<_./ _)" [0, 0, 10] 10) - "_lessEx" :: "[idt, 'a, bool] => bool" ("(3\\_<_./ _)" [0, 0, 10] 10) - "_leAll" :: "[idt, 'a, bool] => bool" ("(3\\_\\_./ _)" [0, 0, 10] 10) - "_leEx" :: "[idt, 'a, bool] => bool" ("(3\\_\\_./ _)" [0, 0, 10] 10) + "_lessAll" :: "[idt, 'a, bool] => bool" ("(3\_<_./ _)" [0, 0, 10] 10) + "_lessEx" :: "[idt, 'a, bool] => bool" ("(3\_<_./ _)" [0, 0, 10] 10) + "_leAll" :: "[idt, 'a, bool] => bool" ("(3\_\_./ _)" [0, 0, 10] 10) + "_leEx" :: "[idt, 'a, bool] => bool" ("(3\_\_./ _)" [0, 0, 10] 10) syntax (HOL) "_lessAll" :: "[idt, 'a, bool] => bool" ("(3! _<_./ _)" [0, 0, 10] 10)