Zulip Chat Archive
Stream: Is there code for X?
Topic: Multiple apply
Matias Heikkilä (Oct 18 2023 at 14:05):
Is there tactic for writing
some_tactic [thm1, thm2, thm3]
instead of
apply thm1
apply thm2
apply thm3
Matias Heikkilä (Oct 18 2023 at 14:06):
Or some other smart way
Ruben Van de Velde (Oct 18 2023 at 14:06):
refine thm1 <| thm2 <| thm3 ?_
could work, depending on how much apply
is hiding
Alex J. Best (Oct 18 2023 at 14:10):
You can use apply_rules
for this (assuming that the greedy algorithm of apply these whenever you can is what you want) https://leanprover-community.github.io/mathlib4_docs/Mathlib/Tactic/SolveByElim.html#Mathlib.Tactic.SolveByElim.applyRulesSyntax
Matias Heikkilä (Oct 18 2023 at 14:12):
Thanks for the help, the latter worked in my case. I think I still have some work to do before I actually understand what apply
really does
Matias Heikkilä (Oct 18 2023 at 14:12):
Or refine
...
Last updated: Dec 20 2023 at 11:08 UTC