tuned signature;
authorwenzelm
Tue, 08 Apr 2014 22:01:08 +0200
changeset 56475 710dee42b3d0
parent 56474 4df2727a0b5f
child 56476 dd596c2b5897
tuned signature;
src/Pure/PIDE/command.scala
src/Pure/PIDE/document.scala
--- a/src/Pure/PIDE/command.scala	Tue Apr 08 21:48:09 2014 +0200
+++ b/src/Pure/PIDE/command.scala	Tue Apr 08 22:01:08 2014 +0200
@@ -81,11 +81,11 @@
     def add(index: Markup_Index, markup: Text.Markup): Markups =
       new Markups(rep + (index -> (this(index) + markup)))
 
-    def other_id_iterator: Iterator[Document_ID.Generic] =
-      for (Markup_Index(_, Text.Chunk.Id(other_id)) <- rep.keysIterator)
-        yield other_id
+    def redirection_iterator: Iterator[Document_ID.Generic] =
+      for (Markup_Index(_, Text.Chunk.Id(id)) <- rep.keysIterator)
+        yield id
 
-    def retarget(other_id: Document_ID.Generic): Markups =
+    def redirect(other_id: Document_ID.Generic): Markups =
       new Markups(
         (for {
           (Markup_Index(status, Text.Chunk.Id(id)), markup) <- rep.iterator
@@ -135,8 +135,8 @@
 
     def markup(index: Markup_Index): Markup_Tree = markups(index)
 
-    def retarget(other_command: Command): State =
-      new State(other_command, Nil, Results.empty, markups.retarget(other_command.id))
+    def redirect(other_command: Command): State =
+      new State(other_command, Nil, Results.empty, markups.redirect(other_command.id))
 
 
     def eq_content(other: State): Boolean =
--- a/src/Pure/PIDE/document.scala	Tue Apr 08 21:48:09 2014 +0200
+++ b/src/Pure/PIDE/document.scala	Tue Apr 08 22:01:08 2014 +0200
@@ -494,7 +494,7 @@
     /*command-exec assignment for each version*/
     val assignments: Map[Document_ID.Version, State.Assignment] = Map.empty,
     /*commands with markup produced by other commands (imm_succs)*/
-    val augmented_commands: Graph[Document_ID.Command, Unit] = Graph.long,
+    val commands_redirection: Graph[Document_ID.Command, Unit] = Graph.long,
     /*explicit (linear) history*/
     val history: History = History.init)
   {
@@ -540,8 +540,8 @@
       (execs.get(id) orElse commands.get(id)).map(st =>
         ((Text.Chunk.Id(st.command.id), st.command.chunk)))
 
-    private def augmented(st: Command.State): Graph[Document_ID.Command, Unit] =
-      (augmented_commands /: st.markups.other_id_iterator)({ case (graph, id) =>
+    private def redirection(st: Command.State): Graph[Document_ID.Command, Unit] =
+      (commands_redirection /: st.markups.redirection_iterator)({ case (graph, id) =>
         graph.default_node(id, ()).default_node(st.command.id, ()).add_edge(id, st.command.id) })
 
     def accumulate(id: Document_ID.Generic, message: XML.Elem): (Command.State, State) =
@@ -550,13 +550,13 @@
         case Some(st) =>
           val new_st = st.accumulate(self_id(st), other_id _, message)
           val execs1 = execs + (id -> new_st)
-          (new_st, copy(execs = execs1, augmented_commands = augmented(new_st)))
+          (new_st, copy(execs = execs1, commands_redirection = redirection(new_st)))
         case None =>
           commands.get(id) match {
             case Some(st) =>
               val new_st = st.accumulate(self_id(st), other_id _, message)
               val commands1 = commands + (id -> new_st)
-              (new_st, copy(commands = commands1, augmented_commands = augmented(new_st)))
+              (new_st, copy(commands = commands1, commands_redirection = redirection(new_st)))
             case None => fail
           }
       }
@@ -654,7 +654,7 @@
         blobs = blobs1,
         commands = commands1,
         execs = execs1,
-        augmented_commands = augmented_commands.restrict(commands1.isDefinedAt(_)),
+        commands_redirection = commands_redirection.restrict(commands1.isDefinedAt(_)),
         assignments = assignments1)
     }
 
@@ -680,15 +680,15 @@
     {
       val self = command_states_self(version, command)
       val others =
-        if (augmented_commands.defined(command.id)) {
+        if (commands_redirection.defined(command.id)) {
           (for {
-            command_id <- augmented_commands.imm_succs(command.id).iterator
+            command_id <- commands_redirection.imm_succs(command.id).iterator
             (id, st) <- command_states_self(version, the_static_state(command_id).command)
             if !self.exists(_._1 == id)
           } yield (id, st)).toMap.valuesIterator.toList
         }
         else Nil
-      self.map(_._2) ::: others.map(_.retarget(command))
+      self.map(_._2) ::: others.map(_.redirect(command))
     }
 
     def command_results(version: Version, command: Command): Command.Results =