Zulip Chat Archive
Stream: new members
Topic: ennreal not \le itself?
Rémy Degenne (Oct 07 2020 at 18:41):
Hello everyone. I am new to lean and a small problem is currently puzzling me: I cannot find how to complete the following goal,
example (a : ennreal) : a ≤ a :=
begin
sorry,
end
Replacing sorry by refl or by simp fails, and I don't understand why.
Thanks!
Johan Commelin (Oct 07 2020 at 18:42):
Hmm, both should work
Johan Commelin (Oct 07 2020 at 18:46):
import data.real.ennreal
example (x : ennreal) : x ≤ x :=
begin
exact le_refl x
end
this works...
Johan Commelin (Oct 07 2020 at 18:46):
But I can't replace the exact le_refl x
by apply le_refl
Johan Commelin (Oct 07 2020 at 18:46):
very strange
Rémy Degenne (Oct 07 2020 at 18:49):
Thank you. At least I can get the other parts of my code to work. But it is indeed very strange.
Reid Barton (Oct 07 2020 at 18:50):
Presumably the apply bug. Does refl
use apply
perhaps?
Johan Commelin (Oct 07 2020 at 18:51):
example (x : ennreal) : x ≤ x :=
begin
refl' -- works
end
Kevin Buzzard (Oct 07 2020 at 21:36):
Nice work Rémy, you (re)discovered an annoying bug which is surprisingly hard to fix :-) Fortunately we have workarounds
Last updated: Dec 20 2023 at 11:08 UTC