Built with
doc-gen4, running Lean4.
Bubbles (
) indicate interactive fragments: hover for details, tap to reveal contents.
Use
Ctrl+โCtrl+โto navigate,
Ctrl+๐ฑ๏ธto focus.
On Mac, use
Cmdinstead of
Ctrl.
import Lean
import Std.Util.TermUnsafe
namespace Mathlib.Tactic
open Lean Meta Elab Tactic Term
/--
`apply (config := cfg) e` is like `apply e` but allows you to provide a configuration
`cfg : ApplyConfig` to pass to the underlying apply operation.
-/
elab (name := applyWith) "apply" " (" &"config" " := " cfg:term ") " e:term : tactic => do
let cfg โ unsafe evalTerm ApplyConfig (mkConst ``ApplyConfig) cfg
evalApplyLikeTactic (ยท.apply ยท cfg) e