declare Quotient_Examples/FSet.thy as almost obsolete
authorkuncar
Mon, 14 Oct 2013 15:01:41 +0200
changeset 54336 9a21e5c6e5d9
parent 54335 03b10317ba78
child 54337 2cf5d0a560ec
declare Quotient_Examples/FSet.thy as almost obsolete
src/HOL/Quotient_Examples/FSet.thy
--- a/src/HOL/Quotient_Examples/FSet.thy	Mon Oct 14 15:01:41 2013 +0200
+++ b/src/HOL/Quotient_Examples/FSet.thy	Mon Oct 14 15:01:41 2013 +0200
@@ -5,6 +5,13 @@
 Type of finite sets.
 *)
 
+(********************************************************************
+  WARNING: There is a formalization of 'a fset as a subtype of sets in
+  HOL/Library/FSet.thy using Lifting/Transfer. The user should use
+  that file rather than this file unless there are some very specific
+  reasons.
+*********************************************************************)
+
 theory FSet
 imports "~~/src/HOL/Library/Multiset" "~~/src/HOL/Library/Quotient_List"
 begin