Skip to content

Commit

Permalink
Revert "chore: complete ProofWidgets bump (#7056)"
Browse files Browse the repository at this point in the history
This reverts commit ae7a2e4.
  • Loading branch information
semorrison committed Sep 10, 2023
1 parent ff7397e commit c2c2f83
Show file tree
Hide file tree
Showing 3 changed files with 7 additions and 7 deletions.
8 changes: 4 additions & 4 deletions Mathlib/Tactic/Widget/CommDiag.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ import Mathlib.CategoryTheory.Category.Basic

import ProofWidgets.Component.PenroseDiagram
import ProofWidgets.Presentation.Expr
import ProofWidgets.Component.Panel.SelectionPanel
import ProofWidgets.Component.SelectionPanel

/-! This module defines tactic/meta infrastructure for displaying commutative diagrams in the
infoview. -/
Expand Down Expand Up @@ -58,13 +58,13 @@ open scoped Jsx in
display as labels in the diagram. -/
def mkCommDiag (sub : String) (embeds : ExprEmbeds) : MetaM Html := do
let embeds ← embeds.mapM fun (s, h) =>
return (s, <InteractiveCode fmt={← Widget.ppExprTagged h} />)
return (
return (s, Html.ofTHtml <InteractiveCode fmt={← Widget.ppExprTagged h} />)
return Html.ofTHtml
<PenroseDiagram
embeds={embeds}
dsl={include_str ".."/".."/".."/"widget"/"src"/"penrose"/"commutative.dsl"}
sty={include_str ".."/".."/".."/"widget"/"src"/"penrose"/"commutative.sty"}
sub={sub} />)
sub={sub} />

/-! ## Commutative triangles -/

Expand Down
4 changes: 2 additions & 2 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,10 +4,10 @@
[{"git":
{"url": "https://github.com/EdAyers/ProofWidgets4",
"subDir?": null,
"rev": "44e6673a20fc0449d003983d1e1f472df40f7107",
"rev": "a0c2cd0ac3245a0dade4f925bcfa97e06dd84229",
"opts": {},
"name": "proofwidgets",
"inputRev?": "v0.0.15",
"inputRev?": "v0.0.13",
"inherited": false}},
{"git":
{"url": "https://github.com/mhuisi/lean4-cli.git",
Expand Down
2 changes: 1 addition & 1 deletion test/CommDiag.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
import Mathlib.Tactic.Widget.CommDiag
import ProofWidgets.Component.Panel.GoalTypePanel
import ProofWidgets.Component.GoalTypePanel

/-! ## Example use of commutative diagram widgets -/

Expand Down

0 comments on commit c2c2f83

Please sign in to comment.