src/HOL/Set.thy
changeset 46026 83caa4f4bd56
parent 45986 c9e50153e5ae
child 46036 6a86cc88b02f
equal deleted inserted replaced
46025:64a19ea435fc 46026:83caa4f4bd56
  1802   "remove x A = A - {x}"
  1802   "remove x A = A - {x}"
  1803 
  1803 
  1804 hide_const (open) remove
  1804 hide_const (open) remove
  1805 
  1805 
  1806 definition project :: "('a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a set" where
  1806 definition project :: "('a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a set" where
  1807   "project P A = {a \<in> A. P a}"
  1807   [code_abbrev]: "project P A = {a \<in> A. P a}"
  1808 
  1808 
  1809 hide_const (open) project
  1809 hide_const (open) project
  1810 
  1810 
  1811 instantiation set :: (equal) equal
  1811 instantiation set :: (equal) equal
  1812 begin
  1812 begin