src/Pure/Thy/presentation.scala
changeset 75891 a63ccf1a583e
parent 75890 a1336e2d7680
child 75892 c8a8b3bff1b4
--- a/src/Pure/Thy/presentation.scala	Wed Aug 17 16:03:36 2022 +0200
+++ b/src/Pure/Thy/presentation.scala	Wed Aug 17 16:07:10 2022 +0200
@@ -192,27 +192,27 @@
 
   /* formal entities */
 
-  object Entity_Context {
-    object Theory_Ref {
-      def unapply(props: Properties.T): Option[Document.Node.Name] =
-        (props, props, props) match {
-          case (Markup.Kind(Markup.THEORY), Markup.Name(theory), Position.Def_File(thy_file)) =>
-            Some(Resources.file_node(Path.explode(thy_file), theory = theory))
-          case _ => None
-        }
-    }
+  object Theory_Ref {
+    def unapply(props: Properties.T): Option[Document.Node.Name] =
+      (props, props, props) match {
+        case (Markup.Kind(Markup.THEORY), Markup.Name(theory), Position.Def_File(thy_file)) =>
+          Some(Resources.file_node(Path.explode(thy_file), theory = theory))
+        case _ => None
+      }
+  }
 
-    object Entity_Ref {
-      def unapply(props: Properties.T): Option[(Path, Option[String], String, String)] =
-        (props, props, props, props) match {
-          case (Markup.Entity.Ref.Prop(_), Position.Def_File(def_file),
-              Markup.Kind(kind), Markup.Name(name)) =>
-            val def_theory = Position.Def_Theory.unapply(props)
-            Some((Path.explode(def_file), def_theory, kind, name))
-          case _ => None
-        }
-    }
+  object Entity_Ref {
+    def unapply(props: Properties.T): Option[(Path, Option[String], String, String)] =
+      (props, props, props, props) match {
+        case (Markup.Entity.Ref.Prop(_), Position.Def_File(def_file),
+        Markup.Kind(kind), Markup.Name(name)) =>
+          val def_theory = Position.Def_Theory.unapply(props)
+          Some((Path.explode(def_file), def_theory, kind, name))
+        case _ => None
+      }
+  }
 
+  object Entity_Context {
     val empty: Entity_Context = new Entity_Context
 
     def make(