Skip to content

Commit

Permalink
chore: rebase on 2022-07-10
Browse files Browse the repository at this point in the history
  • Loading branch information
Vtec234 committed Jul 11, 2022
1 parent 8f6100e commit 680f66a
Showing 1 changed file with 3 additions and 4 deletions.
7 changes: 3 additions & 4 deletions src/Lean/Widget/UserWidget.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,6 +7,7 @@ Authors: E.W.Ayers
import Lean.Widget.Basic
import Lean.Data.Json
import Lean.Environment
import Lean.Elab.Eval
import Lean.Server

open Lean
Expand Down Expand Up @@ -145,10 +146,8 @@ def saveWidgetInfo [Monad m] [MonadEnv m] [MonadError m] [MonadInfoTree m] (widg

syntax (name := widgetCmd) "#widget " ident term : command

private unsafe def evalJsonUnsafe (stx : Syntax) : TermElabM Json := do
let e ← Term.elabTerm stx (mkConst ``Json)
let e ← Meta.instantiateMVars e
Term.evalExpr Json ``Json e
private unsafe def evalJsonUnsafe (stx : Syntax) : TermElabM Json := do
Term.evalTerm Json (mkConst ``Json) stx

@[implementedBy evalJsonUnsafe]
private opaque evalJson (stx : Syntax) : TermElabM Json
Expand Down

0 comments on commit 680f66a

Please sign in to comment.