src/Doc/Implementation/Logic.thy
changeset 61255 15865e0c5598
parent 61246 077b88f9ec16
child 61261 ddb2da7cb2e4
equal deleted inserted replaced
61254:4918c6e52a02 61255:15865e0c5598
   665   @{index_ML Thm.add_def: "Proof.context -> bool -> bool ->
   665   @{index_ML Thm.add_def: "Proof.context -> bool -> bool ->
   666   binding * term -> theory -> (string * thm) * theory"} \\
   666   binding * term -> theory -> (string * thm) * theory"} \\
   667   \end{mldecls}
   667   \end{mldecls}
   668   \begin{mldecls}
   668   \begin{mldecls}
   669   @{index_ML Theory.add_deps: "Proof.context -> string ->
   669   @{index_ML Theory.add_deps: "Proof.context -> string ->
   670   Theory.dep -> Theory.dep list -> theory -> theory"} \\
   670   Defs.entry -> Defs.entry list -> theory -> theory"} \\
   671   \end{mldecls}
   671   \end{mldecls}
   672 
   672 
   673   \begin{description}
   673   \begin{description}
   674 
   674 
   675   \item @{ML Thm.peek_status}~@{text "thm"} informs about the current
   675   \item @{ML Thm.peek_status}~@{text "thm"} informs about the current
   764   the returned theorem.
   764   the returned theorem.
   765 
   765 
   766   \item @{ML Theory.add_deps}~@{text "ctxt name c\<^sub>\<tau> \<^vec>d\<^sub>\<sigma>"}
   766   \item @{ML Theory.add_deps}~@{text "ctxt name c\<^sub>\<tau> \<^vec>d\<^sub>\<sigma>"}
   767   declares dependencies of a named specification for constant @{text
   767   declares dependencies of a named specification for constant @{text
   768   "c\<^sub>\<tau>"}, relative to existing specifications for constants @{text
   768   "c\<^sub>\<tau>"}, relative to existing specifications for constants @{text
   769   "\<^vec>d\<^sub>\<sigma>"}.
   769   "\<^vec>d\<^sub>\<sigma>"}.  This also works for type constructors.
   770 
   770 
   771   \end{description}
   771   \end{description}
   772 \<close>
   772 \<close>
   773 
   773 
   774 
   774