src/HOL/Induct/QuoDataType.thy
changeset 49834 b27bbb021df1
parent 45694 4a8743618257
child 58305 57752a91eec4
--- a/src/HOL/Induct/QuoDataType.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Induct/QuoDataType.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -125,7 +125,7 @@
 
 definition "Msg = UNIV//msgrel"
 
-typedef (open) msg = Msg
+typedef msg = Msg
   morphisms Rep_Msg Abs_Msg
   unfolding Msg_def by (auto simp add: quotient_def)