src/HOL/Library/RBT.thy
changeset 49834 b27bbb021df1
parent 48622 caaa1a02c650
child 49927 cde0a46b4224
--- a/src/HOL/Library/RBT.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Library/RBT.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -10,7 +10,7 @@
 
 subsection {* Type definition *}
 
-typedef (open) ('a, 'b) rbt = "{t :: ('a\<Colon>linorder, 'b) RBT_Impl.rbt. is_rbt t}"
+typedef ('a, 'b) rbt = "{t :: ('a\<Colon>linorder, 'b) RBT_Impl.rbt. is_rbt t}"
   morphisms impl_of RBT
 proof -
   have "RBT_Impl.Empty \<in> ?rbt" by simp