Skip to content

Commit

Permalink
chore: cleanup deprecations (#89)
Browse files Browse the repository at this point in the history
* .

* chore: remove deprecated `html!` tactic

---------

Co-authored-by: Wojciech Nawrocki <[email protected]>
  • Loading branch information
kim-em and Vtec234 authored Nov 24, 2024
1 parent 4546ff0 commit 5f1a4a0
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 25 deletions.
10 changes: 0 additions & 10 deletions ProofWidgets/Component/HtmlDisplay.lean
Original file line number Diff line number Diff line change
Expand Up @@ -71,16 +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]
syntax (name := htmlTac) "html! " term : tactic

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

end HtmlCommand
end ProofWidgets

Expand Down
15 changes: 0 additions & 15 deletions ProofWidgets/Presentation/Expr.lean
Original file line number Diff line number Diff line change
Expand Up @@ -81,21 +81,6 @@ structure GetExprPresentationParams where
name : Name
deriving RpcEncodable

@[server_rpc_method]
def getExprPresentation : GetExprPresentationParams → RequestM (RequestTask Html)
| { expr := ⟨expr⟩, name } => RequestM.asTask do
let ci := expr.ci
if !exprPresenters.hasTag ci.env name then
throw <| RequestError.invalidParams s!"The constant '{name}' is not an Expr presenter."
match evalExprPresenter ci.env ci.options name with
| .ok p =>
expr.runMetaM p.present
| .error e =>
throw <| RequestError.internalError s!"Failed to evaluate Expr presenter '{name}': {e}"

-- https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/deprecation.20warning.20from.20ProofWidgets
attribute [deprecated] getExprPresentation

structure ExprPresentationProps where
expr : WithRpcRef ExprWithCtx
deriving RpcEncodable
Expand Down

0 comments on commit 5f1a4a0

Please sign in to comment.