Skip to content

Commit

Permalink
chore: remove deprecated html! tactic
Browse files Browse the repository at this point in the history
  • Loading branch information
Vtec234 authored Nov 24, 2024
1 parent 3e785b6 commit 3cc4cd1
Showing 1 changed file with 0 additions and 12 deletions.
12 changes: 0 additions & 12 deletions ProofWidgets/Component/HtmlDisplay.lean
Original file line number Diff line number Diff line change
Expand Up @@ -71,18 +71,6 @@ def elabHtmlCmd : CommandElab := fun
stx
| stx => throwError "Unexpected syntax {stx}."

/-- The `html!` tactic is deprecated and does nothing.
If you have a use for it,
please open an issue on https://github.com/leanprover-community/ProofWidgets4. -/
@[deprecated "The `html!` tactic is deprecated and does nothing. If you have a use for it, \
please open an issue on https://github.com/leanprover-community/ProofWidgets4."
(since := "2024-05-15")]
syntax (name := htmlTac) "html! " term : tactic

open Tactic in
@[tactic htmlTac]
def elabHtmlTac : Tactic | _ => pure ()

end HtmlCommand
end ProofWidgets

Expand Down

0 comments on commit 3cc4cd1

Please sign in to comment.