clarified signature;
authorwenzelm
Wed, 27 Jul 2022 09:03:06 +0200
changeset 75701 84990c95712d
parent 75700 953953504590
child 75702 97e8f4c938bf
clarified signature;
src/Pure/General/file.scala
src/Pure/General/path.scala
src/Tools/VSCode/src/dynamic_output.scala
src/Tools/VSCode/src/state_panel.scala
src/Tools/jEdit/src/jedit_lib.scala
--- a/src/Pure/General/file.scala	Tue Jul 26 20:35:42 2022 +0200
+++ b/src/Pure/General/file.scala	Wed Jul 27 09:03:06 2022 +0200
@@ -13,7 +13,7 @@
 import java.nio.file.{StandardOpenOption, Path => JPath, Files, SimpleFileVisitor,
   FileVisitOption, FileVisitResult}
 import java.nio.file.attribute.BasicFileAttributes
-import java.net.{URL, MalformedURLException}
+import java.net.{URI, URL, MalformedURLException}
 import java.util.zip.{GZIPInputStream, GZIPOutputStream}
 import java.util.EnumSet
 
@@ -62,6 +62,12 @@
   def path(file: JFile): Path = Path.explode(standard_path(file))
   def pwd(): Path = path(Path.current.absolute_file)
 
+  def uri(file: JFile): URI = file.toURI
+  def uri(path: Path): URI = path.file.toURI
+
+  def url(file: JFile): URL = uri(file).toURL
+  def url(path: Path): URL = url(path.file)
+
 
   /* relative paths */
 
--- a/src/Pure/General/path.scala	Tue Jul 26 20:35:42 2022 +0200
+++ b/src/Pure/General/path.scala	Wed Jul 27 09:03:06 2022 +0200
@@ -11,7 +11,6 @@
 import java.util.{Map => JMap}
 import java.io.{File => JFile}
 import java.nio.file.{Path => JPath}
-import java.net.{URI, URL}
 
 import scala.util.matching.Regex
 
@@ -314,9 +313,6 @@
   def is_file: Boolean = file.isFile
   def is_dir: Boolean = file.isDirectory
 
-  def uri: URI = file.toURI
-  def url: URL = uri.toURL
-
   def java_path: JPath = file.toPath
 
   def absolute_file: JFile = File.absolute(file)
--- a/src/Tools/VSCode/src/dynamic_output.scala	Tue Jul 26 20:35:42 2022 +0200
+++ b/src/Tools/VSCode/src/dynamic_output.scala	Wed Jul 27 09:03:06 2022 +0200
@@ -42,7 +42,7 @@
                 thy_file <- Position.Def_File.unapply(props)
                 def_line <- Position.Def_Line.unapply(props)
                 source <- resources.source_file(thy_file)
-                uri = Path.explode(source).absolute_file.toURI
+                uri = File.uri(Path.explode(source).absolute_file)
               } yield HTML.link(uri.toString + "#" + def_line, body)
           }
         val elements = Presentation.elements2.copy(entity = Markup.Elements.full)
--- a/src/Tools/VSCode/src/state_panel.scala	Tue Jul 26 20:35:42 2022 +0200
+++ b/src/Tools/VSCode/src/state_panel.scala	Wed Jul 27 09:03:06 2022 +0200
@@ -66,7 +66,7 @@
                   thy_file <- Position.Def_File.unapply(props)
                   def_line <- Position.Def_Line.unapply(props)
                   source <- server.resources.source_file(thy_file)
-                  uri = Path.explode(source).absolute_file.toURI
+                  uri = File.uri(Path.explode(source).absolute_file)
                 } yield HTML.link(uri.toString + "#" + def_line, body)
             }
           val elements = Presentation.elements2.copy(entity = Markup.Elements.full)
--- a/src/Tools/jEdit/src/jedit_lib.scala	Tue Jul 26 20:35:42 2022 +0200
+++ b/src/Tools/jEdit/src/jedit_lib.scala	Wed Jul 27 09:03:06 2022 +0200
@@ -287,7 +287,7 @@
   def load_icon(name: String): Icon = {
     val name1 =
       if (name.startsWith("idea-icons/")) {
-        val file = Path.explode("$ISABELLE_IDEA_ICONS").uri.toASCIIString
+        val file = File.uri(Path.explode("$ISABELLE_IDEA_ICONS")).toASCIIString
         "jar:" + file + "!/" + name
       }
       else name