src/Pure/Admin/afp.scala
changeset 78618 209607465a90
parent 78420 c157af5f346e
child 80055 42bc8ab751c1
--- a/src/Pure/Admin/afp.scala	Tue Aug 29 20:14:44 2023 +0200
+++ b/src/Pure/Admin/afp.scala	Tue Aug 29 20:19:57 2023 +0200
@@ -21,8 +21,6 @@
 
   val chapter: String = "AFP"
 
-  val force_partition1: List[String] = List("Category3", "HOL-ODE")
-
   val BASE: Path = Path.explode("$AFP_BASE")
 
   def main_dir(base_dir: Path = BASE): Path = base_dir + Path.explode("thys")
@@ -207,19 +205,4 @@
   }
  }"""
     }).mkString("[", ", ", "\n]\n")
-
-
-  /* partition sessions */
-
-  def partition(n: Int): List[String] =
-    n match {
-      case 0 => Nil
-      case 1 | 2 =>
-        val graph = sessions_structure.build_graph.restrict(sessions.toSet)
-        val force_part1 =
-          graph.all_preds(graph.all_succs(AFP.force_partition1.filter(graph.defined))).toSet
-        val (part1, part2) = graph.keys.partition(a => force_part1(a) || graph.is_isolated(a))
-        if (n == 1) part1 else part2
-      case _ => error("Bad AFP partition: " + n + " (should be 0, 1, 2)")
-    }
 }