src/Pure/General/date.scala
changeset 75393 87ebf5a50283
parent 74943 afd8cb7b2be1
child 75394 42267c650205
--- a/src/Pure/General/date.scala	Fri Apr 01 11:51:42 2022 +0200
+++ b/src/Pure/General/date.scala	Fri Apr 01 17:06:10 2022 +0200
@@ -15,14 +15,11 @@
 import scala.annotation.tailrec
 
 
-object Date
-{
+object Date {
   /* format */
 
-  object Format
-  {
-    def make(fmts: List[DateTimeFormatter], tune: String => String = s => s): Format =
-    {
+  object Format {
+    def make(fmts: List[DateTimeFormatter], tune: String => String = s => s): Format = {
       require(fmts.nonEmpty, "no date formats")
 
       new Format {
@@ -41,8 +38,7 @@
     val alt_date: Format = Format("uuuuMMdd")
   }
 
-  abstract class Format private
-  {
+  abstract class Format private {
     def apply(date: Date): String
     def parse(str: String): Date
 
@@ -50,8 +46,7 @@
       try { Some(parse(str)) } catch { case _: DateTimeParseException => None }
   }
 
-  object Formatter
-  {
+  object Formatter {
     def pattern(pat: String): DateTimeFormatter = DateTimeFormatter.ofPattern(pat)
 
     def variants(pats: List[String], locs: List[Locale] = Nil): List[DateTimeFormatter] =
@@ -60,9 +55,11 @@
         if (locs.isEmpty) List(fmt) else locs.map(fmt.withLocale)
       })
 
-    @tailrec def try_variants(fmts: List[DateTimeFormatter], str: String,
-      last_exn: Option[DateTimeParseException] = None): TemporalAccessor =
-    {
+    @tailrec def try_variants(
+      fmts: List[DateTimeFormatter],
+      str: String,
+      last_exn: Option[DateTimeParseException] = None
+    ): TemporalAccessor = {
       fmts match {
         case Nil =>
           throw last_exn.getOrElse(new DateTimeParseException("Failed to parse date", str, 0))
@@ -76,14 +73,12 @@
 
   /* ordering */
 
-  object Ordering extends scala.math.Ordering[Date]
-  {
+  object Ordering extends scala.math.Ordering[Date] {
     def compare(date1: Date, date2: Date): Int =
       date1.instant.compareTo(date2.instant)
   }
 
-  object Rev_Ordering extends scala.math.Ordering[Date]
-  {
+  object Rev_Ordering extends scala.math.Ordering[Date] {
     def compare(date1: Date, date2: Date): Int =
       date2.instant.compareTo(date1.instant)
   }
@@ -104,8 +99,7 @@
   def apply(t: Time, zone: ZoneId = timezone()): Date = instant(t.instant, zone)
 }
 
-sealed case class Date(rep: ZonedDateTime)
-{
+sealed case class Date(rep: ZonedDateTime) {
   def midnight: Date =
     new Date(ZonedDateTime.of(rep.toLocalDate, LocalTime.MIDNIGHT, rep.getZone))