src/HOL/Groups.thy
changeset 52210 0226035df99d
parent 52143 36ffe23b25f8
child 52289 83ce5d2841e7
--- a/src/HOL/Groups.thy	Tue May 28 13:14:31 2013 +0200
+++ b/src/HOL/Groups.thy	Tue May 28 16:29:11 2013 +0200
@@ -124,12 +124,10 @@
 typed_print_translation {*
   let
     fun tr' c = (c, fn ctxt => fn T => fn ts =>
-      if not (null ts) orelse T = dummyT orelse
-        not (Printer.show_type_constraint ctxt) andalso can Term.dest_Type T
-      then raise Match
-      else
+      if null ts andalso Printer.type_emphasis ctxt T then
         Syntax.const @{syntax_const "_constrain"} $ Syntax.const c $
-          Syntax_Phases.term_of_typ ctxt T);
+          Syntax_Phases.term_of_typ ctxt T
+      else raise Match);
   in map tr' [@{const_syntax Groups.one}, @{const_syntax Groups.zero}] end;
 *} -- {* show types that are presumably too general *}