aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/LraTest.v
blob: bf3a87da25abd83950844f3cc20f5c9d8e2fc681 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
Require Import Reals.
Require Import Lra.

Open Scope R_scope.

Lemma l1 : forall x y z : R, Rabs (x - z) <= Rabs (x - y) + Rabs (y - z).
intros; split_Rabs; lra.
Qed.

Lemma l2 :
 forall x y : R, x < Rabs y -> y < 1 -> x >= 0 -> - y <= 1 -> Rabs x <= 1.
intros.
split_Rabs; lra.
Qed.