Zulip Chat Archive
Stream: lean4
Topic: dsimp doesn't use iffs that hold by defeq
Robin Arnez (Feb 22 2025 at 20:29):
Normally, when writing lemmas about how two Prop
s are equal, you use ... ↔ ...
instead of ... = ...
. However, these kinds of theorems don't seem to be considered when using dsimp
, which would force you to additionally write an equality theorem. A simple example of this is e.g. gt_iff_lt
:
example (x y : Nat) : x > y ↔ y < x := by
dsimp -- dsimp made no progress
This might be solvable by extending isRflProofCore
to allow Iff.refl
and Iff.rfl
and Iff.symm
.
Ruben Van de Velde (Feb 22 2025 at 20:39):
This is https://github.com/leanprover-community/mathlib4/issues/10675
Eric Wieser (Feb 22 2025 at 21:17):
Added some more context there
Marcus Rossel (Feb 23 2025 at 06:57):
https://github.com/leanprover/lean4/issues/2678
Last updated: May 02 2025 at 03:31 UTC