src/HOL/Library/Cardinality.thy
changeset 52143 36ffe23b25f8
parent 51188 9b5bf1a9a710
child 52147 9943f8067f11
--- a/src/HOL/Library/Cardinality.thy	Sat May 25 15:00:53 2013 +0200
+++ b/src/HOL/Library/Cardinality.thy	Sat May 25 15:37:53 2013 +0200
@@ -43,7 +43,7 @@
 
 translations "CARD('t)" => "CONST card (CONST UNIV \<Colon> 't set)"
 
-typed_print_translation (advanced) {*
+typed_print_translation {*
   let
     fun card_univ_tr' ctxt _ [Const (@{const_syntax UNIV}, Type (_, [T]))] =
       Syntax.const @{syntax_const "_type_card"} $ Syntax_Phases.term_of_typ ctxt T