src/HOL/List.thy
changeset 82823 71cbfcda66d6
parent 82802 547335b41005
child 82824 7ddae44464d4
equal deleted inserted replaced
82822:638c73041d96 82823:71cbfcda66d6
  8508 begin
  8508 begin
  8509 
  8509 
  8510 qualified definition Least :: \<open>'a::linorder set \<Rightarrow> 'a\<close> \<comment> \<open>only for code generation\<close>
  8510 qualified definition Least :: \<open>'a::linorder set \<Rightarrow> 'a\<close> \<comment> \<open>only for code generation\<close>
  8511   where Least_eq [code_abbrev, simp]: \<open>Least S = (LEAST x. x \<in> S)\<close>
  8511   where Least_eq [code_abbrev, simp]: \<open>Least S = (LEAST x. x \<in> S)\<close>
  8512 
  8512 
  8513 qualified lemma Min_filter_eq [code_abbrev]:
  8513 qualified lemma Least_filter_eq [code_abbrev]:
  8514   \<open>Least (Set.filter P S) = (LEAST x. x \<in> S \<and> P x)\<close>
  8514   \<open>Least (Set.filter P S) = (LEAST x. x \<in> S \<and> P x)\<close>
  8515   by simp
  8515   by simp
  8516 
  8516 
  8517 qualified definition Least_abort :: \<open>'a set \<Rightarrow> 'a::linorder\<close>
  8517 qualified definition Least_abort :: \<open>'a set \<Rightarrow> 'a::linorder\<close>
  8518   where \<open>Least_abort = Least\<close>
  8518   where \<open>Least_abort = Least\<close>