src/HOL/Library/Numeral_Type.thy
changeset 49834 b27bbb021df1
parent 48063 f02b4302d5dd
child 51153 b14ee572cc7b
--- a/src/HOL/Library/Numeral_Type.thy	Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Library/Numeral_Type.thy	Fri Oct 12 18:58:20 2012 +0200
@@ -10,16 +10,16 @@
 
 subsection {* Numeral Types *}
 
-typedef (open) num0 = "UNIV :: nat set" ..
-typedef (open) num1 = "UNIV :: unit set" ..
+typedef num0 = "UNIV :: nat set" ..
+typedef num1 = "UNIV :: unit set" ..
 
-typedef (open) 'a bit0 = "{0 ..< 2 * int CARD('a::finite)}"
+typedef 'a bit0 = "{0 ..< 2 * int CARD('a::finite)}"
 proof
   show "0 \<in> {0 ..< 2 * int CARD('a)}"
     by simp
 qed
 
-typedef (open) 'a bit1 = "{0 ..< 1 + 2 * int CARD('a::finite)}"
+typedef 'a bit1 = "{0 ..< 1 + 2 * int CARD('a::finite)}"
 proof
   show "0 \<in> {0 ..< 1 + 2 * int CARD('a)}"
     by simp