src/HOL/Library/Dlist.thy
changeset 49834 b27bbb021df1
parent 48282 39bfb2844b9e
child 55467 a5c9002bc54d
--- a/src/HOL/Library/Dlist.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Library/Dlist.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -8,7 +8,7 @@
 
 subsection {* The type of distinct lists *}
 
-typedef (open) 'a dlist = "{xs::'a list. distinct xs}"
+typedef 'a dlist = "{xs::'a list. distinct xs}"
   morphisms list_of_dlist Abs_dlist
 proof
   show "[] \<in> {xs. distinct xs}" by simp