TOML Value #
A TOML value with optional source info.
- string (ref : Lean.Syntax) (s : String) : Lake.Toml.Value
- integer (ref : Lean.Syntax) (n : Int) : Lake.Toml.Value
- float (ref : Lean.Syntax) (n : Float) : Lake.Toml.Value
- boolean (ref : Lean.Syntax) (b : Bool) : Lake.Toml.Value
- dateTime (ref : Lean.Syntax) (dt : Lake.Toml.DateTime) : Lake.Toml.Value
- array (ref : Lean.Syntax) (xs : Array Lake.Toml.Value) : Lake.Toml.Value
- table' (ref : Lean.Syntax) (xs : Lake.Toml.RBDict Lean.Name Lake.Toml.Value Lean.Name.quickCmp) : Lake.Toml.Value
Instances For
Equations
- Lake.Toml.instInhabitedValue = { default := Lake.Toml.Value.string default default }
Equations
- Lake.Toml.instBEqValue = { beq := Lake.Toml.beqValue✝ }
@[reducible, inline]
A TOML table, an ordered key-value map of TOML values (Lake.Toml.Value
).
Instances For
@[inline]
Equations
- Lake.Toml.Table.mkEmpty capacity = Lake.Toml.RBDict.mkEmpty capacity
Instances For
@[reducible, match_pattern, inline]
Equations
- Lake.Toml.Value.table ref t = Lake.Toml.Value.table'✝ ref t
Instances For
@[inline]
Equations
- (Lake.Toml.Value.string ref s).ref = ref
- (Lake.Toml.Value.integer ref n).ref = ref
- (Lake.Toml.Value.float ref n).ref = ref
- (Lake.Toml.Value.boolean ref b).ref = ref
- (Lake.Toml.Value.dateTime ref dt).ref = ref
- (Lake.Toml.Value.array ref xs).ref = ref
- (Lake.Toml.Value.table'✝ ref xs).ref = ref
Instances For
Pretty Printing #
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lake.Toml.ppSimpleKey k = if (k.all fun (c : Char) => c.isAlphanum || c == '_' || c == '-') = true then k else Lake.Toml.ppString k
Instances For
Equations
- Lake.Toml.instToStringValue = { toString := Lake.Toml.Value.toString }
Equations
- One or more equations did not get rendered due to their size.