src/HOL/ex/Numeral.thy
changeset 35363 09489d8ffece
parent 35113 1a0c129bb2e0
child 35430 df2862dc23a8
--- a/src/HOL/ex/Numeral.thy	Thu Feb 25 22:15:27 2010 +0100
+++ b/src/HOL/ex/Numeral.thy	Thu Feb 25 22:17:33 2010 +0100
@@ -327,7 +327,7 @@
       val k = int_of_num' n;
       val t' = Syntax.const @{syntax_const "_Numerals"} $ Syntax.free ("#" ^ string_of_int k);
     in case T
-     of Type ("fun", [_, T']) =>  (* FIXME @{type_syntax} *)
+     of Type (@{type_syntax fun}, [_, T']) =>
          if not (! show_types) andalso can Term.dest_Type T' then t'
          else Syntax.const Syntax.constrainC $ t' $ Syntax.term_of_typ show_sorts T'
       | T' => if T' = dummyT then t' else raise Match