Equations
- One or more equations did not get rendered due to their size.
Instances For
The ! modifier instructs grind to consider only minimal indexable subexpressions
when selecting patterns.
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
Instances For
Equations
- Lean.Parser.Tactic.Grind.grind_filter_ = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.grind_filter_ 1024 (Lean.ParserDescr.const `ident)
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.
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.
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.
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.
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.
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.
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.
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.
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.
Instances For
(grindSeq) runs the grindSeq in sequence on the current list of targets.
This is pure grouping with no added effects.
Equations
- One or more equations did not get rendered due to their size.
Instances For
skip does nothing.
Equations
- Lean.Parser.Tactic.Grind.skip = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.skip 1024 (Lean.ParserDescr.nonReservedSymbol "skip" false)
Instances For
lia linear integer arithmetic.
Equations
- Lean.Parser.Tactic.Grind.lia = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.lia 1024 (Lean.ParserDescr.nonReservedSymbol "lia" false)
Instances For
ring (commutative) rings and fields.
Equations
- Lean.Parser.Tactic.Grind.ring = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.ring 1024 (Lean.ParserDescr.nonReservedSymbol "ring" false)
Instances For
ac associativity and commutativity procedure.
Equations
- Lean.Parser.Tactic.Grind.ac = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.ac 1024 (Lean.ParserDescr.nonReservedSymbol "ac" false)
Instances For
linarith linear arithmetic.
Equations
- Lean.Parser.Tactic.Grind.linarith = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.linarith 1024 (Lean.ParserDescr.nonReservedSymbol "linarith" false)
Instances For
The sorry tactic is a temporary placeholder for an incomplete tactic proof.
Equations
- Lean.Parser.Tactic.Grind.sorry = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.sorry 1024 (Lean.ParserDescr.nonReservedSymbol "sorry" false)
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.
Instances For
Instantiates theorems using E-matching.
The approx modifier is just a marker for users to easily identify automatically generated instantiate tactics
that may have redundant arguments.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Shows asserted facts.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Shows propositions known to be True.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Shows propositions known to be False.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Shows equivalence classes of terms.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Show case-split candidates.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Show grind state.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Show active local theorems and their anchors for heuristic instantiation.
Equations
- Lean.Parser.Tactic.Grind.showLocalThms = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.showLocalThms 1024 (Lean.ParserDescr.nonReservedSymbol "show_local_thms" false)
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Parser.Tactic.Grind.grind_ref_ = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.grind_ref_ 1024 Lean.Parser.Tactic.Grind.anchor
Instances For
Equations
- Lean.Parser.Tactic.Grind.grind_ref__1 = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.grind_ref__1 1022 (Lean.ParserDescr.cat `term 0)
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.
Instances For
done succeeds iff there are no remaining goals.
Equations
- Lean.Parser.Tactic.Grind.done = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.done 1024 (Lean.ParserDescr.nonReservedSymbol "done" false)
Instances For
finish tries to close the current goal using grind's default strategy
Equations
- Lean.Parser.Tactic.Grind.finish = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.finish 1024 (Lean.ParserDescr.nonReservedSymbol "finish" false)
Instances For
finish? tries to close the current goal using grind's default strategy and suggests a tactic script.
Equations
- Lean.Parser.Tactic.Grind.finishTrace = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.finishTrace 1024 (Lean.ParserDescr.nonReservedSymbol "finish?" false)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Executes the given tactic block to close the current goal.
Equations
- One or more equations did not get rendered due to their size.
Instances For
all_goals tac runs tac on each goal, concatenating the resulting goals.
If the tactic fails on any goal, the entire all_goals tactic fails.
Equations
- One or more equations did not get rendered due to their size.
Instances For
focus tac focuses on the main goal, suppressing all other goals, and runs tac on it.
Usually · tac, which enforces that the goal is closed by tac, should be preferred.
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
any_goals tac applies the tactic tac to every goal,
concatenating the resulting goals for successful tactic applications.
If the tactic fails on all of the goals, the entire any_goals tactic fails.
This tactic is like all_goals try tac except that it fails if none of the applications of tac succeeds.
Equations
- One or more equations did not get rendered due to their size.
Instances For
with_annotate_state stx t annotates the lexical range of stx : Syntax with
the initial and final state of running tactic t.
Equations
- One or more equations did not get rendered due to their size.
Instances For
tac <;> tac' runs tac on the main goal and tac' on each produced goal,
concatenating all goals produced by tac'.
Equations
- One or more equations did not get rendered due to their size.
Instances For
first | tac | ... runs each tac until one succeeds, or else fails.
Equations
- One or more equations did not get rendered due to their size.
Instances For
try tac runs tac and succeeds even if tac failed.
Equations
- One or more equations did not get rendered due to their size.
Instances For
fail_if_success t fails if the tactic t succeeds.
Equations
- One or more equations did not get rendered due to their size.
Instances For
admit is a synonym for sorry.
Equations
- Lean.Parser.Tactic.Grind.grindAdmit = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.grindAdmit 1024 (Lean.ParserDescr.nonReservedSymbol "admit" false)
Instances For
fail msg is a tactic that always fails, and produces an error using the given message.
Equations
- One or more equations did not get rendered due to their size.
Instances For
repeat tac repeatedly applies tac so long as it succeeds.
The tactic tac may be a tactic sequence, and if tac fails at any point in its execution,
repeat will revert any partial changes that tac made to the tactic state.
The tactic tac should eventually fail, otherwise repeat tac will run indefinitely.
Equations
- One or more equations did not get rendered due to their size.
Instances For
rename_i x_1 ... x_n renames the last n inaccessible names using the given names.
Equations
- One or more equations did not get rendered due to their size.
Instances For
expose_names renames all inaccessible variables with accessible names, making them available
for reference in generated tactics. However, this renaming introduces machine-generated names
that are not fully under user control. expose_names is primarily intended as a preamble for
generated grind tactic scripts.
Equations
- Lean.Parser.Tactic.Grind.exposeNames = Lean.ParserDescr.node `Lean.Parser.Tactic.Grind.exposeNames 1024 (Lean.ParserDescr.nonReservedSymbol "expose_names" false)
Instances For
set_option opt val in tacs (the tactic) acts like set_option opt val at the command level,
but it sets the option only within the tactics tacs.
Equations
- One or more equations did not get rendered due to their size.