Quot/Examples/FSet.thy
changeset 787 5cf83fa5b36c
parent 779 3b21b24a5fb6
child 918 7be9b054f672
--- a/Quot/Examples/FSet.thy	Thu Dec 24 00:58:50 2009 +0100
+++ b/Quot/Examples/FSet.thy	Thu Dec 24 22:28:19 2009 +0100
@@ -23,7 +23,7 @@
   done
 
 quotient_type 
-  fset = "'a list" / "list_eq"
+  'a fset = "'a list" / "list_eq"
   by (rule equivp_list_eq)
 
 quotient_definition
@@ -280,7 +280,7 @@
 apply (lifting list_induct_part)
 done
 
-quotient_type fset2 = "'a list" / "list_eq"
+quotient_type 'a fset2 = "'a list" / "list_eq"
   by (rule equivp_list_eq)
 
 quotient_definition