--- a/src/Pure/Admin/build_release.scala Sat Jan 27 21:12:16 2024 +0100
+++ b/src/Pure/Admin/build_release.scala Sat Jan 27 22:15:40 2024 +0100
@@ -490,7 +490,7 @@
}
}
- def default_platform_families: List[Platform.Family] = Platform.Family.list0
+ def default_platform_families: List[Platform.Family] = Platform.Family.list
def build_release(
options: Options,
--- a/src/Pure/Admin/isabelle_cronjob.scala Sat Jan 27 21:12:16 2024 +0100
+++ b/src/Pure/Admin/isabelle_cronjob.scala Sat Jan 27 22:15:40 2024 +0100
@@ -295,6 +295,9 @@
val remote_builds1: List[List[Remote_Build]] = {
List(
+ List(Remote_Build("Linux (ARM)", "server-arm",
+ options = "-m32 -B -M1x2" +
+ " -e ISABELLE_SWIPL=swipl")),
List(Remote_Build("Linux B", "lxbroy10", history = 90,
options = "-m32 -B -M1x4,2,4,6", args = "-N -g timing")),
List(
--- a/src/Pure/System/platform.scala Sat Jan 27 21:12:16 2024 +0100
+++ b/src/Pure/System/platform.scala Sat Jan 27 22:15:40 2024 +0100
@@ -25,7 +25,6 @@
else error("Failed to determine current platform family")
object Family {
- val list0: List[Family] = List(Family.linux, Family.windows, Family.macos)
val list: List[Family] = List(Family.linux, Family.linux_arm, Family.windows, Family.macos)
def unapply(name: String): Option[Family] =