src/HOL/List.thy
changeset 25277 95128fcdd7e8
parent 25221 5ded95dda5df
child 25287 094dab519ff5
equal deleted inserted replaced
25276:f9237f6f3a8d 25277:95128fcdd7e8
  2579 apply (auto simp: sorted_distinct_set_unique)
  2579 apply (auto simp: sorted_distinct_set_unique)
  2580 done
  2580 done
  2581 
  2581 
  2582 end
  2582 end
  2583 
  2583 
       
  2584 lemma sorted_upt[simp]: "sorted[i..<j]"
       
  2585 by (induct j) (simp_all add:sorted_append)
       
  2586 
  2584 
  2587 
  2585 subsubsection {* @{text sorted_list_of_set} *}
  2588 subsubsection {* @{text sorted_list_of_set} *}
  2586 
  2589 
  2587 text{* This function maps (finite) linearly ordered sets to sorted
  2590 text{* This function maps (finite) linearly ordered sets to sorted
  2588 lists. Warning: in most cases it is not a good idea to convert from
  2591 lists. Warning: in most cases it is not a good idea to convert from