src/Doc/Isar_Ref/Spec.thy
changeset 59905 678c9e625782
parent 59901 840d03805755
child 59917 9830c944670f
equal deleted inserted replaced
59904:9d04e2c188b3 59905:678c9e625782
   258   \end{description}
   258   \end{description}
   259 
   259 
   260   Here is an artificial example of bundling various configuration
   260   Here is an artificial example of bundling various configuration
   261   options:\<close>
   261   options:\<close>
   262 
   262 
       
   263 (*<*)experiment begin(*>*)
   263 bundle trace = [[simp_trace, linarith_trace, metis_trace, smt_trace]]
   264 bundle trace = [[simp_trace, linarith_trace, metis_trace, smt_trace]]
   264 
   265 
   265 lemma "x = x"
   266 lemma "x = x"
   266   including trace by metis
   267   including trace by metis
       
   268 (*<*)end(*>*)
   267 
   269 
   268 
   270 
   269 section \<open>Term definitions \label{sec:term-definitions}\<close>
   271 section \<open>Term definitions \label{sec:term-definitions}\<close>
   270 
   272 
   271 text \<open>
   273 text \<open>
  1203   other serves as parameter.  Here are examples for these two cases:
  1205   other serves as parameter.  Here are examples for these two cases:
  1204 
  1206 
  1205   \end{description}
  1207   \end{description}
  1206 \<close>
  1208 \<close>
  1207 
  1209 
       
  1210 (*<*)experiment begin(*>*)
  1208   attribute_setup my_rule =
  1211   attribute_setup my_rule =
  1209     \<open>Attrib.thms >> (fn ths =>
  1212     \<open>Attrib.thms >> (fn ths =>
  1210       Thm.rule_attribute
  1213       Thm.rule_attribute
  1211         (fn context: Context.generic => fn th: thm =>
  1214         (fn context: Context.generic => fn th: thm =>
  1212           let val th' = th OF ths
  1215           let val th' = th OF ths
  1216     \<open>Attrib.thms >> (fn ths =>
  1219     \<open>Attrib.thms >> (fn ths =>
  1217       Thm.declaration_attribute
  1220       Thm.declaration_attribute
  1218         (fn th: thm => fn context: Context.generic =>
  1221         (fn th: thm => fn context: Context.generic =>
  1219           let val context' = context
  1222           let val context' = context
  1220           in context' end))\<close>
  1223           in context' end))\<close>
       
  1224 (*<*)end(*>*)
  1221 
  1225 
  1222 text \<open>
  1226 text \<open>
  1223   \begin{description}
  1227   \begin{description}
  1224 
  1228 
  1225   \item @{attribute ML_print_depth} controls the printing depth of the ML
  1229   \item @{attribute ML_print_depth} controls the printing depth of the ML