Zulip Chat Archive

Stream: mathlib4

Topic: Identity map of Natural Numbers is strictly monotone


Jihoon Hyun (Jan 09 2023 at 08:38):

The proof is very trivial, but I wish I had one defined because it's very specific. Please tell me if this is not a good idea.

theorem nat_identity_strictMono :
  StrictMono (λ (n : )  n) := by
  unfold StrictMono
  simp only [imp_self, forall_const]

Chris Hughes (Jan 09 2023 at 08:47):

We already have strictMono_id which says that the identity function is strictly monotonic on any preorder.

Jihoon Hyun (Jan 09 2023 at 08:49):

oh.


Last updated: Dec 20 2023 at 11:08 UTC