Equations
- Lean.Elab.Deriving.FromToJson.mkJsonField n = let s := Lean.Name.toString n; let s₁ := String.dropRightWhile s fun a => a == Char.ofNat 63; (s != s₁, { raw := (Lean.Syntax.mkStrLit s₁).raw })
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Deriving.FromToJson.mkToJsonInstanceHandler.mkAlts
(indVal : Lean.InductiveVal)
(rhs : Lean.ConstructorVal → Array (Lean.Ident × Lean.Expr) → Option (Array Lean.Name) → Lean.Elab.TermElabM Lean.Term)
:
Lean.Elab.TermElabM (Array (Lean.TSyntax `Lean.Parser.Term.matchAlt))
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.
def
Lean.Elab.Deriving.FromToJson.mkFromJsonInstanceHandler.mkAlts
(indVal : Lean.InductiveVal)
(fromJsonFuncId : Lean.Ident)
:
Equations
- One or more equations did not get rendered due to their size.