src/HOL/Quotient_Examples/FSet.thy
changeset 40672 abd4e7358847
parent 40467 dc0439fdd7c5
child 40688 a961ec75fc29
--- a/src/HOL/Quotient_Examples/FSet.thy	Mon Nov 22 09:37:39 2010 +0100
+++ b/src/HOL/Quotient_Examples/FSet.thy	Mon Nov 22 17:46:51 2010 +0100
@@ -25,7 +25,7 @@
   unfolding reflp_def symp_def transp_def
   by auto
 
-text {* Fset type *}
+text {* Cset type *}
 
 quotient_type
   'a fset = "'a list" / "list_eq"