Zulip Chat Archive
Stream: new members
Topic: Confusion about cases'
Chengyan Hu (Mar 28 2025 at 21:22):
It seems like in lean we can only deconstruct hypothesis in form of P \or Q, P \and Q. If I want to deal with h:P \or Q -> R the only thing I can do is apply it to hR:R or the goal R. I'm not that sure if my understanding is correct or not, and this fact seems tedious for me, is there any easier way to deal with that?
Aaron Liu (Mar 28 2025 at 21:23):
How do you expect this to be destructed?
Aaron Liu (Mar 28 2025 at 21:24):
That is, given a h : P ∨ Q → R
, what do you want to turn this into to make it easier to use?
Chengyan Hu (Mar 28 2025 at 21:32):
I mean, I would like to use P->R and Q->R
Aaron Liu (Mar 28 2025 at 21:34):
You can rw
with docs#or_imp
Kyle Miller (Mar 28 2025 at 21:34):
And here's a way you can find or_imp
:
example (p q r : Prop) : (p ∨ q → r) ↔ ((p → r) ∧ (q → r)) := by exact?
-- Try this: exact or_imp
Chengyan Hu (Mar 28 2025 at 21:35):
I see! Thx a lot
Last updated: May 02 2025 at 03:31 UTC