src/HOL/Wellfounded.thy
changeset 71935 82b00b8f1871
parent 71827 5e315defb038
child 72164 b7c54ff7f2dd
--- a/src/HOL/Wellfounded.thy	Thu Jun 11 14:18:34 2020 +0200
+++ b/src/HOL/Wellfounded.thy	Thu Jun 11 16:13:53 2020 +0100
@@ -583,6 +583,9 @@
 lemma irrefl_less_than: "irrefl less_than"
   using irrefl_def by blast
 
+lemma asym_less_than: "asym less_than"
+  by (simp add: asym.simps irrefl_less_than)
+
 lemma total_less_than: "total less_than" and total_on_less_than [simp]: "total_on A less_than"
   using total_on_def by force+
 
@@ -798,6 +801,9 @@
 lemma total_on_lex_prod [simp]: "total_on A r \<Longrightarrow> total_on B s \<Longrightarrow> total_on (A \<times> B) (r <*lex*> s)"
   by (auto simp: total_on_def)
 
+lemma asym_lex_prod: "\<lbrakk>asym R; asym S\<rbrakk> \<Longrightarrow> asym (R <*lex*> S)"
+  by (auto simp add: asym_iff lex_prod_def)
+
 lemma total_lex_prod [simp]: "total r \<Longrightarrow> total s \<Longrightarrow> total (r <*lex*> s)"
   by (auto simp: total_on_def)