src/HOL/Wellfounded.thy
changeset 71766 1249b998e377
parent 71544 66bc4b668d6e
child 71827 5e315defb038
--- a/src/HOL/Wellfounded.thy	Fri Apr 17 17:32:11 2020 +0200
+++ b/src/HOL/Wellfounded.thy	Fri Apr 17 20:55:53 2020 +0100
@@ -580,8 +580,8 @@
 lemma less_than_iff [iff]: "((x,y) \<in> less_than) = (x<y)"
   by (simp add: less_than_def less_eq)
 
-lemma total_less_than: "total less_than"
-  using total_on_def by force
+lemma total_less_than: "total less_than" and total_on_less_than [simp]: "total_on A less_than"
+  using total_on_def by force+
 
 lemma wf_less: "wf {(x, y::nat). x < y}"
   by (rule Wellfounded.wellorder_class.wf)