Zulip Chat Archive
Stream: general
Topic: minimal imports to have the goodies?
Siyuan Yan (Nov 04 2022 at 18:47):
new user of mathlib here, was trying something simple
open nat
example (q d : ℕ) (hqd: q ≥ 2 ∧ d ≥ 2) (a: ℤ) : int.gcd a d = 1 ∧ int.gcd a q = 1 ↔ int.gcd a q = 1 :=
begin
split,
-- ...
end
But then I find basic things like rintro
, linarith
and library_search
missing. What's a sane default import to have those things?
Adam Topaz (Nov 04 2022 at 18:55):
import tactic
Siyuan Yan (Nov 04 2022 at 18:59):
that worked thanks
Kevin Buzzard (Nov 04 2022 at 19:08):
@Siyuan Yan if you posted in #new members then you wouldn't have to continually apologise for being a new user, it would be taken for granted :-) Please continue to ask questions, it's definitely the best way to learn :-)
Siyuan Yan (Nov 04 2022 at 19:09):
Thanks! I didn't know the channel existed
Kevin Buzzard said:
Siyuan Yan if you posted in #new members then you wouldn't have to continually apologise for being a new user, it would be taken for granted :-) Please continue to ask questions, it's definitely the best way to learn :-)
Kevin Buzzard (Nov 04 2022 at 19:09):
PS are you sure about your simple theorem? What if a=d=2 and q=3?
Adam Topaz (Nov 04 2022 at 19:14):
Kevin Buzzard said:
Siyuan Yan if you posted in #new members then you wouldn't have to continually apologise for being a new user, it would be taken for granted :-) Please continue to ask questions, it's definitely the best way to learn :-)
Yes, #new members is probably the best channel for questions like this, but let me reemphasize that you should continue to ask questions!
Last updated: Dec 20 2023 at 11:08 UTC