src/Doc/Codegen/Further.thy
changeset 51717 9e7d1c139569
parent 51172 16eb76ca1e4a
child 52378 08dbf9ff2140
equal deleted inserted replaced
51709:19b47bfac6ef 51717:9e7d1c139569
   253 text %mlref {*
   253 text %mlref {*
   254   \begin{mldecls}
   254   \begin{mldecls}
   255   @{index_ML Code.read_const: "theory -> string -> string"} \\
   255   @{index_ML Code.read_const: "theory -> string -> string"} \\
   256   @{index_ML Code.add_eqn: "thm -> theory -> theory"} \\
   256   @{index_ML Code.add_eqn: "thm -> theory -> theory"} \\
   257   @{index_ML Code.del_eqn: "thm -> theory -> theory"} \\
   257   @{index_ML Code.del_eqn: "thm -> theory -> theory"} \\
   258   @{index_ML Code_Preproc.map_pre: "(simpset -> simpset) -> theory -> theory"} \\
   258   @{index_ML Code_Preproc.map_pre: "(Proof.context -> Proof.context) -> theory -> theory"} \\
   259   @{index_ML Code_Preproc.map_post: "(simpset -> simpset) -> theory -> theory"} \\
   259   @{index_ML Code_Preproc.map_post: "(Proof.context -> Proof.context) -> theory -> theory"} \\
   260   @{index_ML Code_Preproc.add_functrans: "
   260   @{index_ML Code_Preproc.add_functrans: "
   261     string * (theory -> (thm * bool) list -> (thm * bool) list option)
   261     string * (theory -> (thm * bool) list -> (thm * bool) list option)
   262       -> theory -> theory"} \\
   262       -> theory -> theory"} \\
   263   @{index_ML Code_Preproc.del_functrans: "string -> theory -> theory"} \\
   263   @{index_ML Code_Preproc.del_functrans: "string -> theory -> theory"} \\
   264   @{index_ML Code.add_datatype: "(string * typ) list -> theory -> theory"} \\
   264   @{index_ML Code.add_datatype: "(string * typ) list -> theory -> theory"} \\