src/HOL/ex/PER.thy
changeset 49834 b27bbb021df1
parent 45694 4a8743618257
child 58889 5b7a9633cfa8
--- a/src/HOL/ex/PER.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/ex/PER.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -153,7 +153,7 @@
 
 definition "quot = {{x. a \<sim> x}| a::'a::partial_equiv. True}"
 
-typedef (open) 'a quot = "quot :: 'a::partial_equiv set set"
+typedef 'a quot = "quot :: 'a::partial_equiv set set"
   unfolding quot_def by blast
 
 lemma quotI [intro]: "{x. a \<sim> x} \<in> quot"