src/HOL/Ord.ML
changeset 6109 82b50115564c
parent 6073 fba734ba6894
child 6115 c70bce7deb0f
--- a/src/HOL/Ord.ML	Tue Jan 12 17:19:53 1999 +0100
+++ b/src/HOL/Ord.ML	Wed Jan 13 08:41:28 1999 +0100
@@ -144,3 +144,9 @@
 
 (*** eliminates ~= in premises ***)
 bind_thm("linorder_neqE", linorder_neq_iff RS iffD1 RS disjE);
+
+Goal "!!x::'a::linorder. (~ x < y) = (y <= x)";
+by (simp_tac (simpset() addsimps [order_less_le]) 1);
+by (cut_facts_tac [linorder_linear] 1);
+by (blast_tac (claset() addIs [order_antisym]) 1);
+qed "linorder_not_less";