src/HOL/Quotient_Examples/Lift_Set.thy
changeset 49834 b27bbb021df1
parent 47308 9caab698dbe4
child 55584 a879f14b6f95
--- a/src/HOL/Quotient_Examples/Lift_Set.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Quotient_Examples/Lift_Set.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -10,7 +10,7 @@
 
 definition set where "set = (UNIV :: ('a \<Rightarrow> bool) set)"
 
-typedef (open) 'a set = "set :: ('a \<Rightarrow> bool) set"
+typedef 'a set = "set :: ('a \<Rightarrow> bool) set"
   morphisms member Set
   unfolding set_def by auto