src/HOL/Library/FSet.thy
changeset 56166 9a241bc276cd
parent 55945 e96383acecf9
child 56518 beb3b6851665
equal deleted inserted replaced
56165:dd89ce51d2c8 56166:9a241bc276cd
   141 begin
   141 begin
   142 
   142 
   143 lift_definition uminus_fset :: "'a fset \<Rightarrow> 'a fset" is uminus 
   143 lift_definition uminus_fset :: "'a fset \<Rightarrow> 'a fset" is uminus 
   144   parametric right_total_Compl_transfer Compl_transfer by simp
   144   parametric right_total_Compl_transfer Compl_transfer by simp
   145 
   145 
   146 instance by (default, simp_all only: INF_def SUP_def) (transfer, auto)+
   146 instance by (default, simp_all only: INF_def SUP_def) (transfer, simp add: Compl_partition Diff_eq)+
   147 
   147 
   148 end
   148 end
   149 
   149 
   150 abbreviation fUNIV :: "'a::finite fset" where "fUNIV \<equiv> top"
   150 abbreviation fUNIV :: "'a::finite fset" where "fUNIV \<equiv> top"
   151 abbreviation fuminus :: "'a::finite fset \<Rightarrow> 'a fset" ("|-| _" [81] 80) where "|-| x \<equiv> uminus x"
   151 abbreviation fuminus :: "'a::finite fset \<Rightarrow> 'a fset" ("|-| _" [81] 80) where "|-| x \<equiv> uminus x"