src/HOL/Quickcheck_Narrowing.thy
changeset 49834 b27bbb021df1
parent 48901 5e0455e29339
child 49962 a8cc904a6820
--- a/src/HOL/Quickcheck_Narrowing.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Quickcheck_Narrowing.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -25,7 +25,7 @@
 
 subsubsection {* Type @{text "code_int"} for Haskell Quickcheck's Int type *}
 
-typedef (open) code_int = "UNIV \<Colon> int set"
+typedef code_int = "UNIV \<Colon> int set"
   morphisms int_of of_int by rule
 
 lemma of_int_int_of [simp]: