Zulip Chat Archive
Stream: new members
Topic: prop
BANGJI HU (Oct 24 2024 at 09:43):
import Mathlib.Tactic
variable (P Q R: Prop)
theorem q1 : ((P↔Q)↔R) ↔ (P↔(Q↔R)) := by
constructor
intro h
constructor
intro p
constructor
intro q
BANGJI HU (Oct 24 2024 at 09:44):
Can you give me some hints?
Yoh Tanimoto (Oct 24 2024 at 10:17):
I think, when you introduce two goals for ↔
, it's better to indent like this
import Mathlib.Tactic
variable (P Q R: Prop)
theorem q1 : ((P↔Q)↔R) ↔ (P↔(Q↔R)) := by
constructor
· intro h
constructor
· intro p
constructor
· intro q
Note that if h: A↔B
, then h.mp : A → B
and h.mpr : B → A
BANGJI HU (Oct 24 2024 at 10:21):
(deleted)
Last updated: May 02 2025 at 03:31 UTC