Restriction of DataValue
that covers exactly those cases that Lean is able to handle when passed via the -D
flag.
- ofString (s : String) : LeanOptionValue
- ofBool (b : Bool) : LeanOptionValue
- ofNat (n : Nat) : LeanOptionValue
Instances For
Equations
Equations
- Lean.instReprLeanOptionValue = { reprPrec := Lean.instReprLeanOptionValue.repr }
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.LeanOptionValue.ofDataValue? (Lean.DataValue.ofString s) = some (Lean.LeanOptionValue.ofString s)
- Lean.LeanOptionValue.ofDataValue? (Lean.DataValue.ofBool b) = some (Lean.LeanOptionValue.ofBool b)
- Lean.LeanOptionValue.ofDataValue? (Lean.DataValue.ofNat n) = some (Lean.LeanOptionValue.ofNat n)
- Lean.LeanOptionValue.ofDataValue? x✝ = none
Instances For
Equations
Instances For
Equations
- Lean.instValueLeanOptionValue = { toDataValue := Lean.LeanOptionValue.toDataValue, ofDataValue? := Lean.LeanOptionValue.ofDataValue? }
Equations
Equations
Equations
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Formats the lean option value as a CLI flag argument.
Equations
Instances For
An option that is used by Lean as if it was passed using -D
.
- name : Name
The option's name.
- value : LeanOptionValue
The option's value.
Instances For
Instances For
Equations
Equations
- Lean.instReprLeanOption = { reprPrec := Lean.instReprLeanOption.repr }
Equations
- One or more equations did not get rendered due to their size.
Instances For
Options that are used by Lean as if they were passed using -D
.
- values : NameMap LeanOptionValue
Instances For
Equations
- Lean.instInhabitedLeanOptions.default = { values := default }
Instances For
Equations
Equations
- Lean.instReprLeanOptions = { reprPrec := Lean.instReprLeanOptions.repr }
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Add the options from new
, overriding those in self
.
Equations
- self.append new = { values := Std.TreeMap.mergeWith (fun (x : Lean.Name) (x_1 b : Lean.LeanOptionValue) => b) self.values new.values }
Instances For
Equations
- Lean.instAppendLeanOptions = { append := Lean.LeanOptions.append }
Add the options from new
, overriding those in self
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.instFromJsonLeanOptions = { fromJson? := fun (j : Lean.Json) => Lean.LeanOptions.mk <$> Lean.fromJson? j }
Equations
- Lean.instToJsonLeanOptions = { toJson := fun (options : Lean.LeanOptions) => Lean.toJson options.values }