Zulip Chat Archive
Stream: new members
Topic: nat_abs vs lifted nat
Will Midwood (Oct 09 2022 at 18:02):
Hi there,
In one of my theorems, I have arrived needing to solve this goal:
x y : ℤ,
e : ℕ,
hex : e ∣ x.nat_abs,
hey : e ∣ y.nat_abs
⊢ ↑e ∣ x ∧ ↑e ∣ y
This seems like I need to switch between types, but I'm not exactly sure how to do that.
Will Midwood (Oct 09 2022 at 18:03):
Thanks in advance ^
Ruben Van de Velde (Oct 09 2022 at 18:06):
There's a lemma in mathlib that says exactly this, try split, library_search
Ruben Van de Velde (Oct 09 2022 at 18:07):
Will probably be called something like int.dvd_nat_abs
Ruben Van de Velde (Oct 09 2022 at 18:08):
Ah, no. It's docs#int.coe_nat_dvd_left
Last updated: Dec 20 2023 at 11:08 UTC