--- a/src/HOL/Nitpick_Examples/Refute_Nits.thy Fri Oct 12 15:08:29 2012 +0200
+++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy Fri Oct 12 18:58:20 2012 +0200
@@ -541,7 +541,7 @@
definition "myTdef = insert (undefined::'a) (undefined::'a set)"
-typedef (open) 'a myTdef = "myTdef :: 'a set"
+typedef 'a myTdef = "myTdef :: 'a set"
unfolding myTdef_def by auto
lemma "(x\<Colon>'a myTdef) = y"
@@ -552,7 +552,7 @@
definition "T_bij = {(f::'a\<Rightarrow>'a). \<forall>y. \<exists>!x. f x = y}"
-typedef (open) 'a T_bij = "T_bij :: ('a \<Rightarrow> 'a) set"
+typedef 'a T_bij = "T_bij :: ('a \<Rightarrow> 'a) set"
unfolding T_bij_def by auto
lemma "P (f\<Colon>(myTdecl myTdef) T_bij)"