src/HOL/Conditionally_Complete_Lattices.thy
changeset 51775 408d937c9486
parent 51773 9328c6681f3c
child 52265 bb907eba5902
--- a/src/HOL/Conditionally_Complete_Lattices.thy	Thu Apr 25 10:35:56 2013 +0200
+++ b/src/HOL/Conditionally_Complete_Lattices.thy	Thu Apr 25 11:59:21 2013 +0200
@@ -246,6 +246,15 @@
 
 end
 
+class linear_continuum = conditionally_complete_linorder + inner_dense_linorder +
+  assumes UNIV_not_singleton: "\<exists>a b::'a. a \<noteq> b"
+begin
+
+lemma ex_gt_or_lt: "\<exists>b. a < b \<or> b < a"
+  by (metis UNIV_not_singleton neq_iff)
+
+end
+
 lemma cSup_bounds:
   fixes S :: "'a :: conditionally_complete_lattice set"
   assumes Se: "S \<noteq> {}" and l: "a <=* S" and u: "S *<= b"