src/HOL/Wellfounded.thy
changeset 71766 1249b998e377
parent 71544 66bc4b668d6e
child 71827 5e315defb038
equal deleted inserted replaced
71763:3b36fc4916af 71766:1249b998e377
   578   by (simp add: less_than_def)
   578   by (simp add: less_than_def)
   579 
   579 
   580 lemma less_than_iff [iff]: "((x,y) \<in> less_than) = (x<y)"
   580 lemma less_than_iff [iff]: "((x,y) \<in> less_than) = (x<y)"
   581   by (simp add: less_than_def less_eq)
   581   by (simp add: less_than_def less_eq)
   582 
   582 
   583 lemma total_less_than: "total less_than"
   583 lemma total_less_than: "total less_than" and total_on_less_than [simp]: "total_on A less_than"
   584   using total_on_def by force
   584   using total_on_def by force+
   585 
   585 
   586 lemma wf_less: "wf {(x, y::nat). x < y}"
   586 lemma wf_less: "wf {(x, y::nat). x < y}"
   587   by (rule Wellfounded.wellorder_class.wf)
   587   by (rule Wellfounded.wellorder_class.wf)
   588 
   588 
   589 
   589