src/Doc/Implementation/Local_Theory.thy
changeset 81116 0fb1e2dd4122
parent 76987 4c275405faae
--- a/src/Doc/Implementation/Local_Theory.thy	Fri Oct 04 23:38:04 2024 +0200
+++ b/src/Doc/Implementation/Local_Theory.thy	Sat Oct 05 14:58:36 2024 +0200
@@ -91,7 +91,7 @@
 text %mlref \<open>
   \begin{mldecls}
   @{define_ML_type local_theory = Proof.context} \\
-  @{define_ML Named_Target.init: "string list -> string -> theory -> local_theory"} \\[1ex]
+  @{define_ML Named_Target.init: "Bundle.name list -> string -> theory -> local_theory"} \\[1ex]
   @{define_ML Local_Theory.define: "(binding * mixfix) * (Attrib.binding * term) ->
     local_theory -> (term * (string * thm)) * local_theory"} \\
   @{define_ML Local_Theory.note: "Attrib.binding * thm list ->