tuned names: avoid overlap with instances of class Resources;
authorwenzelm
Fri, 16 Dec 2022 15:14:09 +0100
changeset 76652 90abc28523d7
parent 76643 f8826fc8c419
child 76653 f8b1a75dbea7
tuned names: avoid overlap with instances of class Resources;
src/Pure/Tools/jedit.ML
src/Tools/jEdit/src/jedit_jar.scala
--- a/src/Pure/Tools/jedit.ML	Fri Dec 16 09:55:22 2022 +0100
+++ b/src/Pure/Tools/jedit.ML	Fri Dec 16 15:14:09 2022 +0100
@@ -40,7 +40,7 @@
     (parse_resources o map File.read)
       [\<^file>\<open>~~/src/Tools/jEdit/jedit_main/actions.xml\<close>,
        \<^file>\<open>~~/src/Tools/jEdit/jedit_main/dockables.xml\<close>] @
-    (parse_resources o \<^scala>\<open>jEdit.resources\<close>) ["actions.xml", "dockables.xml"]
+    (parse_resources o \<^scala>\<open>jEdit.resource\<close>) ["actions.xml", "dockables.xml"]
     |> sort_strings);
 
 fun get_actions () = Lazy.force lazy_actions;
--- a/src/Tools/jEdit/src/jedit_jar.scala	Fri Dec 16 09:55:22 2022 +0100
+++ b/src/Tools/jEdit/src/jedit_jar.scala	Fri Dec 16 15:14:09 2022 +0100
@@ -19,10 +19,10 @@
     else using(s)(File.read_stream)
   }
 
-  object JEdit_Resources extends Scala.Fun_Strings("jEdit.resources") {
+  object JEdit_Resource extends Scala.Fun_Strings("jEdit.resource") {
     val here = Scala_Project.here
     def apply(args: List[String]): List[String] = args.map(get_resource)
   }
 
-  class Scala_Functions extends Scala.Functions(JEdit_Resources)
+  class Scala_Functions extends Scala.Functions(JEdit_Resource)
 }