aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega/int63.v
blob: 15146187ca2c04bc4fbf560f6f7c4418d92838db (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
Require Import ZArith  Lia.
Require Import Int63.
Require ZifyInt63.

Open Scope int63_scope.

Goal forall (x:int), 0 <= x = true.
Proof. lia. Qed.

Goal max_int = 9223372036854775807.
Proof. lia. Qed.

Goal digits = 63.
Proof. lia. Qed.

Goal wB = (2^63)%Z.
Proof. lia. Qed.

Goal forall x y, x + y <= max_int = true.
Proof. lia. Qed.

Goal forall x, x <> 0 -> x / x = 1.
Proof.
  nia.
Qed.