src/HOL/Library/FSet.thy
changeset 55738 303123344459
parent 55732 07906fc6af7a
child 55933 12ee2c407dad
--- a/src/HOL/Library/FSet.thy	Tue Feb 25 19:07:40 2014 +0100
+++ b/src/HOL/Library/FSet.thy	Tue Feb 25 19:07:42 2014 +0100
@@ -186,9 +186,8 @@
 
 lift_definition fthe_elem :: "'a fset \<Rightarrow> 'a" is the_elem .
 
-(* FIXME why is not invariant here unfolded ? *)
-lift_definition fbind :: "'a fset \<Rightarrow> ('a \<Rightarrow> 'b fset) \<Rightarrow> 'b fset" is Set.bind parametric bind_transfer
-unfolding invariant_def Set.bind_def by clarsimp metis
+lift_definition fbind :: "'a fset \<Rightarrow> ('a \<Rightarrow> 'b fset) \<Rightarrow> 'b fset" is Set.bind parametric bind_transfer 
+by (simp add: Set.bind_def)
 
 lift_definition ffUnion :: "'a fset fset \<Rightarrow> 'a fset" is Union parametric Union_transfer by simp