Configuration for try?.
- main : Bool
If
mainistrue, all functions in the current module are considered for function induction, unfolding, etc. - name : Bool
If
nameistrue, all functions in the same namespace are considered for function induction, unfolding, etc. - targetOnly : Bool
If
targetOnlyistrue,try?collects information using the goal target only. - max : Nat
Maximum number of suggestions.
- missing : Bool
If
missingistrue, allows the construction of partial solutions where some of the subgoals aresorry. - only : Bool
- harder : Bool
If
harderistrue, more expensive tactics and operations are tried. - merge : Bool
- wrapWithBy : Bool
If
wrapWithByistrue, suggestions are wrapped withbyfor term mode usage.
Instances For
Equations
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
Helper internal tactic for implementing the tactic try?.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Helper internal tactic used to implement evalSuggest in try?
Equations
- One or more equations did not get rendered due to their size.
Instances For
register_try?_tactic tac registers a tactic tac as a suggestion generator for the try? tactic.
An optional priority can be specified with register_try?_tactic (priority := 500) tac.
Higher priority generators are tried first. The default priority is 1000.
Equations
- One or more equations did not get rendered due to their size.
Instances For
∎ (typed as \qed) is a macro that expands to try? in tactic mode.
Equations
- «tactic∎» = Lean.ParserDescr.node `«tactic∎» 1024 (Lean.ParserDescr.nonReservedSymbol "∎" false)
Instances For
∎ (typed as \qed) is a macro that expands to by try? (wrapWithBy := true) in term mode.
The wrapWithBy config option causes suggestions to be prefixed with by.
Equations
- «term∎» = Lean.ParserDescr.node `«term∎» 1024 (Lean.ParserDescr.symbol "∎")