Nominal/Nominal2.thy
changeset 3190 1b7c034c9e9e
parent 3181 ca162f0a7957
child 3201 3e6f4320669f
equal deleted inserted replaced
3189:e46d4ee64221 3190:1b7c034c9e9e
   746   opt_name -- P.and_list1 dt_parser -- bnfun_parser >> tuple3
   746   opt_name -- P.and_list1 dt_parser -- bnfun_parser >> tuple3
   747 
   747 
   748 end
   748 end
   749 
   749 
   750 (* Command Keyword *)
   750 (* Command Keyword *)
   751 val _ = Outer_Syntax.local_theory ("nominal_datatype", Keyword.thy_decl) 
   751 val _ = Outer_Syntax.local_theory @{command_spec "nominal_datatype"}
   752   "declaration of nominal datatypes" 
   752   "declaration of nominal datatypes" 
   753     (main_parser >> nominal_datatype2_cmd)
   753     (main_parser >> nominal_datatype2_cmd)
   754 *}
   754 *}
   755 
   755 
   756 
   756