Zulip Chat Archive

Stream: mathlib4

Topic: gt_iff_lt proves a weird goal


Jireh Loreaux (Aug 01 2024 at 15:39):

Found this with exact?%. I'm so confused. The kernel accepts the proof.

import Mathlib

open unitInterval

lemma coe_pos {x : I} : (0 : ) < x  0 < x := gt_iff_lt

Yaël Dillies (Aug 01 2024 at 15:40):

gt_iff_lt is just Iff.rfl specialised to a < b. (0 : ℝ) < x ↔ 0 < x is defeq to (0 : ℝ) < x ↔ (0 : ℝ) < x. So it works.

Jireh Loreaux (Aug 01 2024 at 15:41):

lol I tried rfl instead of Iff.rfl without thinking before I did exact?%. Thanks. I'm just being stupid.


Last updated: May 02 2025 at 03:31 UTC