leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: Is there code for X?

Topic: Iff from `a → b` and `¬a → ¬b`


Daniel Weber (Sep 26 2024 at 03:22):

Do we have

example {a b : Prop} (h₁ : a → b) (h₂ : ¬a → ¬b) : a ↔ b := ⟨h₁, h₂.mtr⟩

somewhere? I was unable to locate it

Kim Morrison (Sep 26 2024 at 03:59):

Probably not.


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll