src/HOL/List.thy
changeset 61566 c3d6e570ccef
parent 61468 7d1127ac2251
child 61605 1bf7b186542e
equal deleted inserted replaced
61565:352c73a689da 61566:c3d6e570ccef
  5149 
  5149 
  5150 definition sorted_list_of_set :: "'a set \<Rightarrow> 'a list" where
  5150 definition sorted_list_of_set :: "'a set \<Rightarrow> 'a list" where
  5151   "sorted_list_of_set = folding.F insort []"
  5151   "sorted_list_of_set = folding.F insort []"
  5152 
  5152 
  5153 sublocale sorted_list_of_set!: folding insort Nil
  5153 sublocale sorted_list_of_set!: folding insort Nil
  5154 where
  5154 rewrites
  5155   "folding.F insort [] = sorted_list_of_set"
  5155   "folding.F insort [] = sorted_list_of_set"
  5156 proof -
  5156 proof -
  5157   interpret comp_fun_commute insort by (fact comp_fun_commute_insort)
  5157   interpret comp_fun_commute insort by (fact comp_fun_commute_insort)
  5158   show "folding insort" by standard (fact comp_fun_commute)
  5158   show "folding insort" by standard (fact comp_fun_commute)
  5159   show "folding.F insort [] = sorted_list_of_set" by (simp only: sorted_list_of_set_def)
  5159   show "folding.F insort [] = sorted_list_of_set" by (simp only: sorted_list_of_set_def)