Quot/Examples/AbsRepTest.thy
changeset 796 64f9c76f70c7
parent 795 a28f805df355
child 803 6f6ee78c7357
--- a/Quot/Examples/AbsRepTest.thy	Sat Dec 26 21:36:20 2009 +0100
+++ b/Quot/Examples/AbsRepTest.thy	Sat Dec 26 23:20:46 2009 +0100
@@ -93,8 +93,8 @@
 
 ML {*
 test_funs absF @{context} 
-     (@{typ "('a list) list \<Rightarrow> 'a"}, 
-      @{typ "('a fset) fset \<Rightarrow> 'a"})
+     (@{typ "('a list) list \<Rightarrow> 'a list"}, 
+      @{typ "('a fset) fset \<Rightarrow> 'a fset"})
 *}