equal
deleted
inserted
replaced
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 } |