Equations
- One or more equations did not get rendered due to their size.
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.
Introduce one or more hypotheses, optionally naming and/or pattern-matching them.
For each hypothesis to be introduced, the remaining main goal's target type must be a let
or function type.
intro
by itself introduces one anonymous hypothesis, which can be accessed by e.g.assumption
.intro x y
introduces two hypotheses and names them. Individual hypotheses can be anonymized via_
, or matched against a pattern:-- ... ⊢ α × β → ... intro (a, b) -- ..., a : α, b : β ⊢ ...
- Alternatively,
intro
can be combined with pattern matching much likefun
:intro | n + 1, 0 => tac | ...
Equations
- One or more equations did not get rendered due to their size.
rename t => x
renames the most recent hypothesis whose type matches t
(which may contain placeholders) to x
,
or fails if no such hypothesis could be found.
Equations
- One or more equations did not get rendered due to their size.
clear x...
removes the given hypotheses, or fails if there are remaining references to a hypothesis.
Equations
- One or more equations did not get rendered due to their size.
subst x...
substitutes each x
with e
in the goal if there is a hypothesis of type x = e
or e = x
.
If x
is itself a hypothesis of type y = e
or e = y
, y
is substituted instead.
Equations
- One or more equations did not get rendered due to their size.
Apply subst
to all hypotheses of the form h : x = t
or h : t = x
.
Equations
- Lean.Parser.Tactic.substVars = Lean.ParserDescr.node `Lean.Parser.Tactic.substVars 1024 (Lean.ParserDescr.nonReservedSymbol "subst_vars" false)
assumption
tries to solve the main goal using a hypothesis of compatible type, or else fails.
Note also the ‹t›
term notation, which is a shorthand for show t by assumption
.
Equations
- Lean.Parser.Tactic.assumption = Lean.ParserDescr.node `Lean.Parser.Tactic.assumption 1024 (Lean.ParserDescr.nonReservedSymbol "assumption" false)
contradiction
closes the main goal if its hypotheses are "trivially contradictory".
- Inductive type/family with no applicable constructors
example (h : False) : p := by contradiction
- Injectivity of constructors
example (h : none = some true) : p := by contradiction --
- Decidable false proposition
example (h : 2 + 2 = 3) : p := by contradiction
- Contradictory hypotheses
example (h : p) (h' : ¬ p) : q := by contradiction
- Other simple contradictions such as
example (x : Nat) (h : x ≠ x) : p := by contradiction
Equations
- Lean.Parser.Tactic.contradiction = Lean.ParserDescr.node `Lean.Parser.Tactic.contradiction 1024 (Lean.ParserDescr.nonReservedSymbol "contradiction" false)
apply e
tries to match the current goal against the conclusion of e
's type.
If it succeeds, then the tactic returns as many subgoals as the number of premises that
have not been fixed by type inference or type class resolution.
Non-dependent premises are added before dependent ones.
The apply
tactic uses higher-order pattern matching, type class resolution, and first-order unification with dependent types.
Equations
- One or more equations did not get rendered due to their size.
exact e
closes the main goal if its target type matches that of e
.
Equations
- One or more equations did not get rendered due to their size.
refine e
behaves like exact e
, except that named (?x
) or unnamed (?_
) holes in e
that are not solved
by unification with the main goal's target type are converted into new goals, using the hole's name, if any, as the goal case name.
Equations
- One or more equations did not get rendered due to their size.
If the main goal's target type is an inductive type, constructor
solves it with the first matching constructor, or else fails.
Equations
- Lean.Parser.Tactic.constructor = Lean.ParserDescr.node `Lean.Parser.Tactic.constructor 1024 (Lean.ParserDescr.nonReservedSymbol "constructor" false)
case'
is similar to the case tag => tac
tactic, but does not ensure the goal has been solved after applying tac
, nor
admits the goal if tac
failed. Recall that case
closes the goal using sorry
when tac
fails, and
the tactic execution is not interrupted.
Equations
- One or more equations did not get rendered due to their size.
next => tac
focuses on the next goal solves it using tac
, or else fails.
next x₁ ... xₙ => tac
additionally renames the n
most recent hypotheses with inaccessible names to the given names.
Equations
- One or more equations did not get rendered due to their size.
all_goals tac
runs tac
on each goal, concatenating the resulting goals, if any.
Equations
- One or more equations did not get rendered due to their size.
any_goals tac
applies the tactic tac
to every goal, and succeeds if at least one application succeeds.
Equations
- One or more equations did not get rendered due to their size.
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.
skip
does nothing.
Equations
- Lean.Parser.Tactic.skip = Lean.ParserDescr.node `Lean.Parser.Tactic.skip 1024 (Lean.ParserDescr.nonReservedSymbol "skip" false)
done
succeeds iff there are no remaining goals.
Equations
- Lean.Parser.Tactic.done = Lean.ParserDescr.node `Lean.Parser.Tactic.done 1024 (Lean.ParserDescr.nonReservedSymbol "done" false)
trace_state
displays the current state in the info view.
Equations
- Lean.Parser.Tactic.traceState = Lean.ParserDescr.node `Lean.Parser.Tactic.traceState 1024 (Lean.ParserDescr.nonReservedSymbol "trace_state" false)
trace msg
displays msg
in the info view.
Equations
- One or more equations did not get rendered due to their size.
fail_if_success t
fails if the tactic t
succeeds.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
first | tac | ...
runs each tac
until one succeeds, or else fails.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
try tac
runs tac
and succeeds even if tac
failed.
Equations
- One or more equations did not get rendered due to their size.
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.
eq_refl
is equivalent to exact rfl
, but has a few optimizations.
Equations
- Lean.Parser.Tactic.refl = Lean.ParserDescr.node `Lean.Parser.Tactic.refl 1024 (Lean.ParserDescr.nonReservedSymbol "eq_refl" false)
rfl
tries to close the current goal using reflexivity.
This is supposed to be an extensible tactic and users can add their own support
for new reflexive relations.
Equations
- Lean.Parser.Tactic.tacticRfl = Lean.ParserDescr.node `Lean.Parser.Tactic.tacticRfl 1024 (Lean.ParserDescr.nonReservedSymbol "rfl" false)
rfl'
is similar to rfl
, but disables smart unfolding and unfolds all kinds of definitions,
theorems included (relevant for declarations defined by well-founded recursion).
Equations
- Lean.Parser.Tactic.tacticRfl' = Lean.ParserDescr.node `Lean.Parser.Tactic.tacticRfl' 1024 (Lean.ParserDescr.nonReservedSymbol "rfl'" false)
Equations
- Lean.Parser.Tactic.ac_refl = Lean.ParserDescr.node `Lean.Parser.Tactic.ac_refl 1024 (Lean.ParserDescr.nonReservedSymbol "ac_refl " false)
admit
is a shorthand for exact sorry
.
Equations
- Lean.Parser.Tactic.tacticAdmit = Lean.ParserDescr.node `Lean.Parser.Tactic.tacticAdmit 1024 (Lean.ParserDescr.nonReservedSymbol "admit" false)
The sorry
tactic is a shorthand for exact sorry
.
Equations
- Lean.Parser.Tactic.tacticSorry = Lean.ParserDescr.node `Lean.Parser.Tactic.tacticSorry 1024 (Lean.ParserDescr.nonReservedSymbol "sorry" false)
infer_instance
is an abbreviation for exact inferInstance
Equations
- Lean.Parser.Tactic.tacticInfer_instance = Lean.ParserDescr.node `Lean.Parser.Tactic.tacticInfer_instance 1024 (Lean.ParserDescr.nonReservedSymbol "infer_instance" false)
Optional configuration option for tactics
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Parser.Tactic.locationWildcard = Lean.ParserDescr.nodeWithAntiquot "locationWildcard" `Lean.Parser.Tactic.locationWildcard (Lean.ParserDescr.symbol "*")
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
rewrite [e]
applies identity e
as a rewrite rule to the target of the main goal.
If e
is preceded by left arrow (←
or <-
), the rewrite is applied in the reverse direction.
If e
is a defined constant, then the equational theorems associated with e
are used. This provides a convenient way to unfold e
.
rewrite [e₁, ..., eₙ]
applies the given rules sequentially.rewrite [e] at l
rewritese
at location(s)l
, wherel
is either*
or a list of hypotheses in the local context. In the latter case, a turnstile⊢
or|-
can also be used, to signify the target of the goal.
Equations
- One or more equations did not get rendered due to their size.
rw
is like rewrite
, but also tries to close the goal by "cheap" (reducible) rfl
afterwards.
Equations
- One or more equations did not get rendered due to their size.
The injection
tactic is based on the fact that constructors of inductive data types are injections.
That means that if c
is a constructor of an inductive datatype, and if (c t₁)
and (c t₂)
are two terms that are equal then t₁
and t₂
are equal too.
If q
is a proof of a statement of conclusion t₁ = t₂
, then injection applies injectivity to derive the equality of all arguments of t₁
and t₂
placed in the same positions. For example, from (a::b) = (c::d)
we derive a=c
and b=d
. To use this tactic t₁
and t₂
should be constructor applications of the same constructor.
Given h : a::b = c::d
, the tactic injection h
adds two new hypothesis with types a = c
and b = d
to the main goal.
The tactic injection h with h₁ h₂
uses the names h₁
and h₂
to name the new hypotheses.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Parser.Tactic.injections = Lean.ParserDescr.node `Lean.Parser.Tactic.injections 1024 (Lean.ParserDescr.nonReservedSymbol "injections" false)
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Parser.Tactic.simpPre = Lean.ParserDescr.nodeWithAntiquot "simpPre" `Lean.Parser.Tactic.simpPre (Lean.ParserDescr.symbol "↓")
Equations
- Lean.Parser.Tactic.simpPost = Lean.ParserDescr.nodeWithAntiquot "simpPost" `Lean.Parser.Tactic.simpPost (Lean.ParserDescr.symbol "↑")
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Parser.Tactic.simpStar = Lean.ParserDescr.nodeWithAntiquot "simpStar" `Lean.Parser.Tactic.simpStar (Lean.ParserDescr.symbol "*")
The simp
tactic uses lemmas and hypotheses to simplify the main goal target or non-dependent hypotheses. It has many variants.
simp
simplifies the main goal target using lemmas tagged with the attribute[simp]
.simp [h₁, h₂, ..., hₙ]
simplifies the main goal target using the lemmas tagged with the attribute[simp]
and the givenhᵢ
's, where thehᵢ
's are expressions. If anhᵢ
is a defined constantf
, then the equational lemmas associated withf
are used. This provides a convenient way to unfoldf
.simp [*]
simplifies the main goal target using the lemmas tagged with the attribute[simp]
and all hypotheses.simp only [h₁, h₂, ..., hₙ]
is likesimp [h₁, h₂, ..., hₙ]
but does not use[simp]
lemmassimp [-id₁, ..., -idₙ]
simplifies the main goal target using the lemmas tagged with the attribute[simp]
, but removes the ones namedidᵢ
.simp at h₁ h₂ ... hₙ
simplifies the hypothesesh₁ : T₁
...hₙ : Tₙ
. If the target or another hypothesis depends onhᵢ
, a new simplified hypothesishᵢ
is introduced, but the old one remains in the local context.simp at *
simplifies all the hypotheses and the target.simp [*] at *
simplifies target and all (propositional) hypotheses using the other hypotheses.
Equations
- One or more equations did not get rendered due to their size.
simp_all
is a stronger version of simp [*] at *
where the hypotheses and target are simplified
multiple times until no simplication is applicable.
Only non-dependent propositional hypotheses are considered.
Equations
- One or more equations did not get rendered due to their size.
unfold id,+
unfolds definition id
. For non-recursive definitions, this tactic is identical to delta
.
For recursive definitions, it hides the encoding tricks used by the Lean frontend to convince the
kernel that the definition terminates.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
have h : t := e
adds the hypothesis h : t
to the current goal if e
a term of type t
. If t
is omitted, it will be inferred.
If h
is omitted, the name this
is used.
The variant have pattern := e
is equivalent to match e with | pattern => _
, and it is convenient for types that have only applicable constructor.
Example: given h : p ∧ q ∧ r
, have ⟨h₁, h₂, h₃⟩ := h
produces the hypotheses h₁ : p
, h₂ : q
, and h₃ : r
.
Equations
- One or more equations did not get rendered due to their size.
have h := e
adds the hypothesis h : t
if e : t
.
Equations
- One or more equations did not get rendered due to their size.
Given a main goal ctx |- t
, suffices h : t' from e
replaces the main goal with ctx |- t'
,
e
must have type t
in the context ctx, h : t'
.
The variant suffices h : t' by tac
is a shorthand for suffices h : t' from by tac
.
If h :
is omitted, the name this
is used.
Equations
- One or more equations did not get rendered due to their size.
let h : t := e
adds the hypothesis h : t := e
to the current goal if e
a term of type t
.
If t
is omitted, it will be inferred.
The variant let pattern := e
is equivalent to match e with | pattern => _
, and it is convenient for types that have only applicable constructor.
Example: given h : p ∧ q ∧ r
, let ⟨h₁, h₂, h₃⟩ := h
produces the hypotheses h₁ : p
, h₂ : q
, and h₃ : r
.
Equations
- One or more equations did not get rendered due to their size.
show t
finds the first goal whose target unifies with t
. It makes that the main goal,
performs the unification, and replaces the target with the unified version of t
.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Assuming x
is a variable in the local context with an inductive type, induction x
applies induction on x
to the main goal,
producing one goal for each constructor of the inductive type, in which the target is replaced by a general instance of that constructor
and an inductive hypothesis is added for each recursive argument to the constructor.
If the type of an element in the local context depends on x
, that element is reverted and reintroduced afterward,
so that the inductive hypothesis incorporates that hypothesis as well.
For example, given n : Nat
and a goal with a hypothesis h : P n
and target Q n
, induction n
produces one goal
with hypothesis h : P 0
and target Q 0
, and one goal with hypotheses h : P (Nat.succ a)
and ih₁ : P a → Q a
and target Q (Nat.succ a)
.
Here the names a
and ih₁
are chosen automatically and are not accessible. You can use with
to provide the variables names for each constructor.
induction e
, wheree
is an expression instead of a variable, generalizese
in the goal, and then performs induction on the resulting variable.induction e using r
allows the user to specify the principle of induction that should be used. Herer
should be a theorem whose result type must be of the formC t
, whereC
is a bound variable andt
is a (possibly empty) sequence of bound variablesinduction e generalizing z₁ ... zₙ
, wherez₁ ... zₙ
are variables in the local context, generalizes overz₁ ... zₙ
before applying the induction but then introduces them in each goal. In other words, the net effect is that each inductive hypothesis is generalized.- Given
x : Nat
,induction x with | zero => tac₁ | succ x' ih => tac₂
uses tactictac₁
for thezero
case, andtac₂
for thesucc
case.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
generalize ([h :] e = x),+
replaces all occurrences e
s in the main goal with a fresh hypothesis x
s.
If h
is given, h : e = x
is introduced as well.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Assuming x
is a variable in the local context with an inductive type, cases x
splits the main goal,
producing one goal for each constructor of the inductive type, in which the target is replaced by a general instance of that constructor.
If the type of an element in the local context depends on x
, that element is reverted and reintroduced afterward,
so that the case split affects that hypothesis as well. cases
detects unreachable cases and closes them automatically.
For example, given n : Nat
and a goal with a hypothesis h : P n
and target Q n
, cases n
produces one goal with hypothesis h : P 0
and target Q 0
,
and one goal with hypothesis h : P (Nat.succ a)
and target Q (Nat.succ a)
. Here the name a
is chosen automatically and are not accessible. You can use with
to provide the variables names for each constructor.
cases e
, wheree
is an expression instead of a variable, generalizese
in the goal, and then cases on the resulting variable.- Given
as : List α
,cases as with | nil => tac₁ | cons a as' => tac₂
, uses tactictac₁
for thenil
case, andtac₂
for thecons
case, anda
andas'
are used as names for the new variables introduced. cases h : e
, wheree
is a variable or an expression, performs cases one
as above, but also adds a hypothesish : e = ...
to each hypothesis, where...
is the constructor instance for that particular case.
Equations
- One or more equations did not get rendered due to their size.
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.
repeat tac
applies tac
to main goal. If the application succeeds,
the tactic is applied recursively to the generated subgoals until it eventually fails.
Equations
- One or more equations did not get rendered due to their size.
trivial
tries different simple tactics (e.g., rfl
, contradiction
, ...) to close the current goal.
You can use the command macro_rules
to extend the set of tactics used. Example:
macro_rules | `(tactic| trivial) => `(tactic| simp)
Equations
- Lean.Parser.Tactic.tacticTrivial = Lean.ParserDescr.node `Lean.Parser.Tactic.tacticTrivial 1024 (Lean.ParserDescr.nonReservedSymbol "trivial" false)
Equations
- One or more equations did not get rendered due to their size.
stop
is a helper tactic for "discarding" the rest of a proof. It is useful when working on the middle of a complex proofs,
and less messy than commenting the remainder of the proof.
Equations
- One or more equations did not get rendered due to their size.
The tactic specialize h a₁ ... aₙ
works on local hypothesis h
.
The premises of this hypothesis, either universal quantifications or non-dependent implications,
are instantiated by concrete terms coming either from arguments a₁
... aₙ
.
The tactic adds a new hypothesis with the same name h := h a₁ ... aₙ
and tries to clear the previous one.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
fail msg
is a tactic that always fail and produces an error using the given message.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Parser.Tactic.save = Lean.ParserDescr.node `Lean.Parser.Tactic.save 1024 (Lean.ParserDescr.nonReservedSymbol "save" false)
The tactic sleep ms
sleeps for ms
milliseconds and does nothing. It is used for debugging purposes only.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
‹t›
resolves to an (arbitrary) hypothesis of type t
. It is useful for referring to hypotheses without accessible names.
t
may contain holes that are solved by unification with the expected type; in particular, ‹_›
is a shortcut for by assumption
.
Equations
- One or more equations did not get rendered due to their size.