Zulip Chat Archive
Stream: Is there code for X?
Topic: ite or
Yaël Dillies (Aug 05 2021 at 12:48):
Do we not have this?
lemma ite_eq_or_eq {p : Prop} [decidable p] (a b : V) :
ite p a b = a ∨ ite p a b = b :=
decidable.by_cases (λ h, or.inl (if_pos h)) (λ h, or.inr (if_neg h))
Ruben Van de Velde (Aug 05 2021 at 12:54):
docs#ite_eq_iff is a little stronger
Yaël Dillies (Aug 05 2021 at 13:06):
Argh, I want to .resolve
that.
I'll just PR it. #8557
Last updated: Dec 20 2023 at 11:08 UTC