Skip to content

Commit

Permalink
chore: remove left-over TODO
Browse files Browse the repository at this point in the history
  • Loading branch information
arthur-adjedj committed Sep 10, 2024
1 parent 84463ab commit e1b25b8
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Lean/Elab/Deriving/FromToJson.lean
Original file line number Diff line number Diff line change
Expand Up @@ -180,7 +180,7 @@ def mkFromJsonBody (ctx : Context) (e : Expr) : TermElabM Term := do
def mkFromJsonAuxFunction (ctx : Context) (i : Nat) : TermElabM Command := do
let auxFunName := ctx.auxFunNames[i]!
let indval := ctx.typeInfos[i]!
let header ← mkFromJsonHeader indval --TODO fix header info
let header ← mkFromJsonHeader indval
let binders := header.binders
Term.elabBinders binders fun _ => do
let type ← Term.elabTerm header.targetType none
Expand Down

0 comments on commit e1b25b8

Please sign in to comment.