Zulip Chat Archive

Stream: new members

Topic: lt_le_trans?


Marcus Rossel (Dec 26 2020 at 11:58):

Is there a theorem along the lines of:

theorem lt_le_trans {a b c : } (lt : a < b) (le : b  c) : a < c

I haven't been able to find one. Thanks :pray:🏻

Bryan Gin-ge Chen (Dec 26 2020 at 12:15):

docs#lt_of_lt_of_le

Eric Wieser (Dec 26 2020 at 12:21):

If you've already gone as far as writing out the lemma statement as you have there, try := by library_search to find the lemma

Damiano Testa (Dec 26 2020 at 16:54):

There is also its companion lt_of_le_of_lt

Floris van Doorn (Dec 28 2020 at 18:55):

There is also nice projection notation:

theorem lt_le_trans {a b c : } (lt : a < b) (le : b  c) : a < c := lt.trans_le le

Last updated: Dec 20 2023 at 11:08 UTC