aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Num/DiscrProps.v
blob: 7c84d2b354eb70024331e794f1810209d6edcdaa (plain)
1
2
3
4
5
6
7
8
9
10
11
(*i $Id$ i*)

Require Export DiscrAxioms.
Require Export LtProps.

(*s Properties of a discrete order *)

Lemma lt_le_Sx_y : (x,y:N)(x<y) -> ((S x)<=y).
EAuto with num.
Save.
Hints Resolve lt_le_Sx_y : num.