Zulip Chat Archive

Stream: new members

Topic: Proving factor is at least 2


Gareth Ma (Jan 21 2023 at 17:10):

Hi, I am feeling slightly dumb for this question :joy: But I am trying to prove that if x >= 2 is a divisor of y, then y / x >= 2. I am struggling to make any progess. I tried using by_contradiction then splitting y / x = 0 and y / x = 1, then handling each case, but it gets quite complicated. Is there any simple / decently-short solution?

example {x y : } (h : x  y) (hx₁ : 2  x) (hx₂ : x < y) : 2  y / x :=
begin
  sorry
end

Thomas Browning (Jan 21 2023 at 17:16):

  rwa [nat.succ_le_iff, nat.lt_div_iff_mul_lt h, mul_one],

Thomas Browning (Jan 21 2023 at 17:17):

Note that hx₁ is actually unnecessary.

Gareth Ma (Jan 21 2023 at 17:19):

Thanks a lot, I was struggling to get literals like "2" to work with the nat succ stuff :(


Last updated: Dec 20 2023 at 11:08 UTC