Skip to content

Commit

Permalink
chore: fix import
Browse files Browse the repository at this point in the history
  • Loading branch information
Vtec234 committed Sep 19, 2023
1 parent c81d255 commit 65bba72
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions ProofWidgets/Demos/Euclidean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ import Lean.Data.HashMap
import Lean.Elab.Tactic
import ProofWidgets.Component.PenroseDiagram
import ProofWidgets.Component.HtmlDisplay
import ProofWidgets.Component.Panel
import ProofWidgets.Component.Panel.Basic

open Lean Meta Server
open ProofWidgets
Expand Down Expand Up @@ -46,13 +46,13 @@ abbrev ExprEmbeds := Array (String × Expr)
open scoped Jsx in
def mkEuclideanDiag (sub : String) (embeds : ExprEmbeds) : MetaM Html := do
let embeds ← embeds.mapM fun (s, h) =>
return (s, Html.ofTHtml <InteractiveCode fmt={← Widget.ppExprTagged h} />)
return Html.ofTHtml
return (s, <InteractiveCode fmt={← Widget.ppExprTagged h} />)
return (
<PenroseDiagram
embeds={embeds}
dsl={include_str ".."/".."/"widget"/"penrose"/"euclidean.dsl"}
sty={include_str ".."/".."/"widget"/"penrose"/"euclidean.sty"}
sub={sub} />
sub={sub} />)

def isEuclideanGoal? (hyps : Array LocalDecl) : MetaM (Option Html) := do
let mut sub := "AutoLabel All\n"
Expand Down

0 comments on commit 65bba72

Please sign in to comment.