doc-src/Locales/Locales/Locales.thy
changeset 26480 544cef16045b
parent 17567 20c0b69dd192
equal deleted inserted replaced
26479:3a2efce3e992 26480:544cef16045b
   396   If a locale has neither assumptions nor import, no predicate is
   396   If a locale has neither assumptions nor import, no predicate is
   397   defined.  If a locale has import but no assumptions, only the locale
   397   defined.  If a locale has import but no assumptions, only the locale
   398   predicate is defined.
   398   predicate is defined.
   399 *}
   399 *}
   400 (*<*)
   400 (*<*)
   401 ML_setup {*
   401 ML {*
   402   val [comm_semi_ax1, comm_semi_ax2] = thms "comm_semi.axioms";
   402   val [comm_semi_ax1, comm_semi_ax2] = thms "comm_semi.axioms";
   403   bind_thm ("comm_semi_ax1", comm_semi_ax1);
   403   bind_thm ("comm_semi_ax1", comm_semi_ax1);
   404   bind_thm ("comm_semi_ax2", comm_semi_ax2);
   404   bind_thm ("comm_semi_ax2", comm_semi_ax2);
   405 *}
   405 *}
   406 (*>*)
   406 (*>*)