added lemma asympD
authordesharna
Mon, 10 Jan 2022 13:11:18 +0100
changeset 74975 5d3a846bccf8
parent 74973 a565a2889b49
child 74976 70aab133dc8d
added lemma asympD
src/HOL/Relation.thy
--- a/src/HOL/Relation.thy	Sun Jan 09 18:50:06 2022 +0000
+++ b/src/HOL/Relation.thy	Mon Jan 10 13:11:18 2022 +0100
@@ -261,19 +261,18 @@
 lemma asymD: "\<lbrakk>asym R; (x,y) \<in> R\<rbrakk> \<Longrightarrow> (y,x) \<notin> R"
   by (simp add: asym.simps)
 
+lemma asympD: "asymp R \<Longrightarrow> R x y \<Longrightarrow> \<not> R y x"
+  by (rule asymD[to_pred])
+
 lemma asym_iff: "asym R \<longleftrightarrow> (\<forall>x y. (x,y) \<in> R \<longrightarrow> (y,x) \<notin> R)"
   by (blast intro: asymI dest: asymD)
 
-context preorder begin
-
-lemma asymp_less[simp]: "asymp (<)"
+lemma (in preorder) asymp_less[simp]: "asymp (<)"
   by (auto intro: asympI dual_order.asym)
 
-lemma asymp_greater[simp]: "asymp (>)"
+lemma (in preorder) asymp_greater[simp]: "asymp (>)"
   by (auto intro: asympI dual_order.asym)
 
-end
-
 
 subsubsection \<open>Symmetry\<close>