Nominal/Nominal2.thy
changeset 2679 e003e5e36bae
parent 2665 16b5a67ee279
child 2733 5f6fefdbf055
equal deleted inserted replaced
2678:494b859bfc16 2679:e003e5e36bae
   651     ||>> prepare_bn_funs bn_fun_strs bn_eq_strs 
   651     ||>> prepare_bn_funs bn_fun_strs bn_eq_strs 
   652     ||>> prepare_bclauses dt_strs 
   652     ||>> prepare_bclauses dt_strs 
   653 
   653 
   654   val bclauses' = complete dt_strs bclauses
   654   val bclauses' = complete dt_strs bclauses
   655 in
   655 in
   656   timeit (fn () => nominal_datatype2 opt_thms_name dts bn_funs bn_eqs bclauses' lthy)
   656   nominal_datatype2 opt_thms_name dts bn_funs bn_eqs bclauses' lthy
   657 end
   657 end
   658 *}
   658 *}
   659 
   659 
   660 ML {* 
   660 ML {* 
   661 (* nominal datatype parser *)
   661 (* nominal datatype parser *)
   703 (* Command Keyword *)
   703 (* Command Keyword *)
   704 val _ = Outer_Syntax.local_theory "nominal_datatype" "test" Keyword.thy_decl
   704 val _ = Outer_Syntax.local_theory "nominal_datatype" "test" Keyword.thy_decl
   705   (main_parser >> nominal_datatype2_cmd)
   705   (main_parser >> nominal_datatype2_cmd)
   706 *}
   706 *}
   707 
   707 
       
   708 (*
   708 ML {*
   709 ML {*
   709 trace := true
   710 trace := true
   710 *}
   711 *}
   711 
   712 *)
   712 
   713 
   713 end
   714 end
   714 
   715 
   715 
   716 
   716 
   717