Zulip Chat Archive

Stream: new members

Topic: Reducing iff statements


Jack M (May 12 2022 at 20:38):

In general, if I have hypotheses of the form

p : a  1   b  1
q : a = 1  b = 1

how might I deduce

r : a < 1  b < 1

Eric Wieser (May 12 2022 at 20:39):

I would guess docs#iff.or and docs#iff.not would help

Eric Wieser (May 12 2022 at 20:40):

That is, p.or q.not should get you almost to your goal

Mario Carneiro (May 12 2022 at 20:55):

I would do something like simp [lt_iff_le_and_ne, p, q]

Adam Topaz (May 12 2022 at 20:57):

Here's Mario's proof:

import tactic
import data.real.basic

example {a b : } (h1 : a  1  b  1) (h2 : a = 1  b = 1) :
  a < 1  b < 1 :=
by simp [lt_iff_le_and_ne, h1, h2]

Last updated: Dec 20 2023 at 11:08 UTC