leanprover-community / mathlib

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

Zulip Chat Archive

Stream: new members

Topic: rfl vs dec_trivial for inequality example


Joseph Corneli (Jan 24 2019 at 11:49):

This works:

theorem one_plus_one_alt : 1 + 1 = 2 := rfl

example : 1 + 1 ≤ 2 := dec_trivial

This doesn't work:

example : 1 + 1 ≤ 2 := rfl

:confused:

Rob Lewis (Jan 24 2019 at 12:01):

Look at the type of rfl? It proves equality, not inequality.

Rob Lewis (Jan 24 2019 at 12:02):

You might be looking for le_refl.


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll