Tactic wishlist #10361
Labels
enhancement
New feature or request
help-wanted
The author needs attention to resolve issues
please-adopt
Inactive PR (would be valuable to adopt)
t-meta
Tactics, attributes or user commands
There has been some discussion of what tactics we would like in a few threads on Zulip. I am making this tracking issue to try to organize these ideas and put them in a visible place. Anyone with repo permission should feel free to edit or add to the list.
TODO: Integrate suggestions from this thread.
New Tactics
0/0
etc).Continuous.tendsto' (by continuity) _ _ (by simp)
.exp(-1/x)
tends to𝓝[>] 0
asx
tends toatTop
.*Should know that 1/x tends to cobounded as
x
tends to𝓝[≠] 0
and vice versa (for any normed field, not only reals)(δ : Real) (h : 0 < δ) ⊢ ∃ ε > 0, ε ^ 2 + 5 * ε + sin ε < δ ∧ 3 * ε < δ
by provingTendsto (fun ε ↦ ε ^ 2 + 5 * ε + sin ε) (nhds 0) (nhds 0)
, similarly for3 * ε
, then using this fact to get a witnessexpr ≠ 0
.field_simp
currently uses (it tries several tactics);a ≠ 0 → -a ≠ 0, a ≠ 0 → b ≠ 0 → a * b ≠ 0 and a ≠ 0 → a ^ n ≠ 0
;+
) and there is aPartialOrder
instancecompute_degree
)omega
?)pi
exp
log
push
tactic that generalizespush_neg
fromneg
to any def. #21841push Real.log
would applylog_mul
.field
field tactic #4837module_nf
recommend
finish
/terminal
: It would be nice if tactics that were capable of finishing a proof were tagged with some kind offinishing
orterminal
attribute, so that they could be collected into a single tactic that would try them all.?
version that gives aTry This
on success.Enhancements of existing Tactics
0 ≤ f a
, never0 < f a
, or we always can prove0 < f a
)expr < 0
, so that it can prove-3 * ε - δ < 0
zify!
zify!
tactic #7450rify
should work forNNreal
.by_contra!
similar tocontrapose!
0 ≤ n%d
n%d < d
d * n/d + n%d = n
d = 0
these do not all hold.abel
work for multiplicative monoids/groups.abel
for multiplicative Groups/Monoids #13233linear_combination
work for groups.polyrith
in pure Lean, removing the dependence on sage and an internet connection.omega
into a full decision procedure for Presburger arithmetic.cleanup
: A tactic to identify and remove redundant terms/hypotheses from the context, doing the work of clear but automatically.simp_rw
that can create new goals for side-conditionsfield_simp
that collects non-zeroness as side conditions.?
versions of tacticsunfold?
to list possible unfold applications. ([Merged by Bors] - feat: interactiveunfold?
tactic #12016)assumption?
(replaces byexact
)linarith?/nlinarith?
linarith only
)linear_combination
norm_cast
useFin.cast_val_eq_self
, soNat.cast (Fin.val n)
simplifies ton
.cases (r:ℚ)
should replacer
with_ / _
instead of an application ofRat.mk'
linear_combination
be used nonterminally.suffices
should work with incremental elaborationAs-Yet Unported mathlib3 Tactics
The text was updated successfully, but these errors were encountered: