Zulip Chat Archive

Stream: new members

Topic: The equivalence of iff and entailment


edmund (Mar 31 2025 at 10:38):

semantics.lean
can anybody help me with proving this: v v_atoms (p_iff ϕ ψ) = v v_atoms (p_and (p_imp ϕ ψ) (p_imp ψ ϕ))

Kim Morrison (Mar 31 2025 at 11:41):

If you can prepare a #mwe, that works in the sandbox, you're much more likely to get helpful answers. (But you may still!)

edmund (Mar 31 2025 at 12:06):

I'm stuck! :smiling_face_with_tear:

Johan Commelin (Mar 31 2025 at 12:24):

Sure. And Kim is suggesting that following the instructions on #mwe is a good first step to get unstuck.

Notification Bot (Apr 01 2025 at 00:37):

This topic was moved here from #maths > The equivalence of iff and entailment by Yury G. Kudryashov.

Yury G. Kudryashov (Apr 01 2025 at 00:37):

@edmund I moved your topic to a more appropriate channel (judging by your account's registration date).

Robin Arnez (Apr 01 2025 at 12:20):

This works:

example : v v_atoms (p_iff ϕ ψ) = v v_atoms (p_and (p_imp ϕ ψ) (p_imp ψ ϕ)) := by
  simp [v]
  cases v v_atoms ϕ <;> cases v v_atoms ψ <;> simp

Last updated: May 02 2025 at 03:31 UTC