src/Pure/System/registry.scala
changeset 78947 2a27d2c8eae8
parent 78945 73162a487f94
child 78950 cd350dcd912a
equal deleted inserted replaced
78946:87ac093e4d1a 78947:2a27d2c8eae8
    32       }
    32       }
    33   }
    33   }
    34 
    34 
    35   object Host extends Table[List[Options.Spec]]("host") {
    35   object Host extends Table[List[Options.Spec]]("host") {
    36     def options_spec(a: TOML.Key, b: TOML.T): Option[Options.Spec] =
    36     def options_spec(a: TOML.Key, b: TOML.T): Option[Options.Spec] =
    37       TOML.Scalar.unapply(b).map(Options.Spec.eq(a, _, permissive = true))
    37       TOML.Scalar.unapply(b).map(Options.Spec.eq(a, _))
    38 
    38 
    39     override def table_value(a: String, t: TOML.Table): List[Options.Spec] =
    39     override def table_value(a: String, t: TOML.Table): List[Options.Spec] =
    40       for ((a, b) <- t.any.values; s <- options_spec(a, b)) yield s
    40       for ((a, b) <- t.any.values; s <- options_spec(a, b)) yield s
    41   }
    41   }
    42 }
    42 }