Zulip Chat Archive
Stream: general
Topic: exclude one lemma from exact?
Filippo A. E. Nuccio (Feb 01 2024 at 10:49):
I am preparing a class and I would like to run exact?
but preventing it to find a very specific lemma (namely nsmul_add_nsmul_eq_zero
) so that I can explain some other feature. The problem is that the files I am importing all import Mathlib.Algebra.GroupPower.Basic
, where the above lemma is defined, so I cannot get rid of it by simply avoiding a certain import. Is there a way to achieve this?
Johan Commelin (Feb 01 2024 at 10:52):
cc @Scott Morrison
Kim Morrison (Feb 01 2024 at 10:56):
You could put a check in exact?
for that specific lemma?
Kim Morrison (Feb 01 2024 at 10:57):
I can't think of a way to do this without modifying exact?
Filippo A. E. Nuccio (Feb 01 2024 at 10:57):
What do you mean by a "check in exact?
"?
Eric Rodriguez (Feb 01 2024 at 11:04):
I think Scott means editing the tactic itself
Filippo A. E. Nuccio (Feb 01 2024 at 11:05):
OK, I'll give it a try. Thanks!
Last updated: May 02 2025 at 03:31 UTC