src/HOL/BNF_Wellorder_Constructions.thy
changeset 75624 22d1c5f2b9f4
parent 72127 a0768f16bccd
child 75669 43f5dfb7fa35
--- a/src/HOL/BNF_Wellorder_Constructions.thy	Sat Jun 25 09:50:40 2022 +0000
+++ b/src/HOL/BNF_Wellorder_Constructions.thy	Mon Jun 27 15:54:18 2022 +0200
@@ -561,6 +561,10 @@
 "r <o r' \<Longrightarrow> \<not> r' \<le>o r"
 using ordLess_ordLeq_trans ordLess_irreflexive by blast
 
+lemma not_ordLeq_ordLess:
+"r \<le>o r' \<Longrightarrow> \<not> r' <o r"
+using not_ordLess_ordLeq by blast
+
 lemma ordLess_or_ordLeq:
 assumes WELL: "Well_order r" and WELL': "Well_order r'"
 shows "r <o r' \<or> r' \<le>o r"