FSet.thy
changeset 244 42dac1cfcd14
parent 241 60acf3d3a4a0
child 248 6ed87b3d358c
--- a/FSet.thy	Fri Oct 30 15:28:44 2009 +0100
+++ b/FSet.thy	Fri Oct 30 15:30:33 2009 +0100
@@ -169,9 +169,9 @@
 
 (* FIXME: does not work yet for all types*)
 quotient_def (for "'a fset")
-  fmap::"('a \<Rightarrow> 'a) \<Rightarrow> 'a fset \<Rightarrow> 'a fset"
+  fmap::"('a \<Rightarrow> 'b) \<Rightarrow> 'a fset \<Rightarrow> 'b fset"
 where
-  "fmap \<equiv> (map::('a \<Rightarrow> 'a) \<Rightarrow> 'a list \<Rightarrow> 'a list)"
+  "fmap \<equiv> (map::('a \<Rightarrow> 'b) \<Rightarrow> 'a list \<Rightarrow> 'b list)"
 
 term map
 term fmap