Zulip Chat Archive

Stream: new members

Topic: M40001 Sheet 1


Michael (Aug 07 2021 at 14:46):

Hello, sorry if this is a silly question but how do I get rid of a universal quantifier in a hypothesis?

lemma question_2a_false : ¬ ( P Q : Prop, (P  Q)  (Q  P)) :=
begin
  intro h,
  sorry
end

leaves me with

h:  (P Q : Prop), (P  Q)  Q  P
 false

and I don't know how to make any more progress.

Alex J. Best (Aug 07 2021 at 14:54):

A forall is an implication, so its really a function that you can plug input into.
In this case its a function from propositions to some implications between their proofs so you can apply it to some specific (well-chosen) propositions of interest using have to make a new hypothesis (called this by default, specialising the old one), e.g.:

lemma question_2a_false : ¬ ( P Q : Prop, (P  Q)  (Q  P)) :=
begin
  intro h,
  have := h true false,
  sorry
end

this is just a random example, not a spoiler / hint (probably).

Eric Wieser (Aug 07 2021 at 14:55):

What's your maths proof?

Michael (Aug 07 2021 at 14:59):

Since the question asks whether → is symmetric, I have a counter-example to the idea that → is symmetric: if P is false and Q is true then P → Q is true and Q → P is false and so we have true → false which is false.

Eric Wieser (Aug 07 2021 at 15:09):

"set P to false and Q to true" is spelt have := h false true


Last updated: Dec 20 2023 at 11:08 UTC