added lemmas antisymp_ge[simp], antisymp_greater[simp], antisymp_le[simp], and antisymp_less[simp]
authordesharna
Tue, 11 Oct 2022 11:48:04 +0200
changeset 76258 2f10e7a2ff01
parent 76257 61a5b5ad3a6e
child 76263 5ede2fce5b01
added lemmas antisymp_ge[simp], antisymp_greater[simp], antisymp_le[simp], and antisymp_less[simp]
NEWS
src/HOL/Relation.thy
--- a/NEWS	Tue Oct 11 11:07:07 2022 +0200
+++ b/NEWS	Tue Oct 11 11:48:04 2022 +0200
@@ -13,7 +13,11 @@
   - Strengthened lemma total_on_singleton. Minor INCOMPATIBILITY.
   - Added lemmas.
       antisym_if_asymp
+      antisymp_ge[simp]
+      antisymp_greater[simp]
       antisymp_if_asymp
+      antisymp_le[simp]
+      antisymp_less[simp]
       irreflD
       irreflpD
       reflp_ge[simp]
--- a/src/HOL/Relation.thy	Tue Oct 11 11:07:07 2022 +0200
+++ b/src/HOL/Relation.thy	Tue Oct 11 11:48:04 2022 +0200
@@ -441,6 +441,18 @@
 lemma antisymp_if_asymp: "asymp R \<Longrightarrow> antisymp R"
   by (rule antisym_if_asym[to_pred])
 
+lemma (in preorder) antisymp_less[simp]: "antisymp (<)"
+  by (rule antisymp_if_asymp[OF asymp_less])
+
+lemma (in preorder) antisymp_greater[simp]: "antisymp (>)"
+  by (rule antisymp_if_asymp[OF asymp_greater])
+
+lemma (in order) antisymp_le[simp]: "antisymp (\<le>)"
+  by (simp add: antisympI)
+
+lemma (in order) antisymp_ge[simp]: "antisymp (\<ge>)"
+  by (simp add: antisympI)
+
 
 subsubsection \<open>Transitivity\<close>