src/HOL/Orderings.thy
changeset 22348 ab505d281015
parent 22344 eddeabf16b5d
child 22377 61610b1beedf
--- a/src/HOL/Orderings.thy	Fri Feb 23 08:39:20 2007 +0100
+++ b/src/HOL/Orderings.thy	Fri Feb 23 08:39:21 2007 +0100
@@ -124,8 +124,6 @@
 
 class order = preorder + 
   assumes antisym: "x \<sqsubseteq> y \<Longrightarrow> y \<sqsubseteq> x \<Longrightarrow> x = y"
-
-context order
 begin
 
 text {* Asymmetry. *}
@@ -815,6 +813,13 @@
 lemma le_boolD: "P \<le> Q \<Longrightarrow> P \<longrightarrow> Q"
   by (simp add: le_bool_def)
 
+lemma [code func]:
+  "False \<le> b \<longleftrightarrow> True"
+  "True \<le> b \<longleftrightarrow> b"
+  "False < b \<longleftrightarrow> b"
+  "True < b \<longleftrightarrow> False"
+  unfolding le_bool_def less_bool_def by simp_all
+
 subsection {* Monotonicity, syntactic least value operator and min/max *}
 
 locale mono =