def
Lean.Elab.Tactic.rewriteTarget
(stx : Syntax)
(symm : Bool)
(config : Meta.Rewrite.Config :=
{ transparency := Meta.TransparencyMode.reducible, offsetCnstrs := true, occs := Meta.Occurrences.all,
newGoals := Meta.ApplyNewGoals.nonDependentFirst })
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.rewriteLocalDecl
(stx : Syntax)
(symm : Bool)
(fvarId : FVarId)
(config : Meta.Rewrite.Config :=
{ transparency := Meta.TransparencyMode.reducible, offsetCnstrs := true, occs := Meta.Occurrences.all,
newGoals := Meta.ApplyNewGoals.nonDependentFirst })
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.