aboutsummaryrefslogtreecommitdiff
path: root/test-suite/primitive/uint63/subc.v
blob: fc4067e48be878327de76e0356df25773177e84e (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
Require Import Int63.

Set Implicit Arguments.

Open Scope int63_scope.

Check (eq_refl : 3 -c 2 = C0 1).
Check (eq_refl (C0 1) <: 3 -c 2 = C0 1).
Check (eq_refl (C0 1) <<: 3 -c 2 = C0 1).
Definition compute1 := Eval compute in 3 -c 2.
Check (eq_refl compute1 : C0 1 = C0 1).

Check (eq_refl : 0 -c 1 = C1 9223372036854775807).
Check (eq_refl (C1 9223372036854775807) <: 0 -c 1 = C1 9223372036854775807).
Check (eq_refl (C1 9223372036854775807) <<: 0 -c 1 = C1 9223372036854775807).
Definition compute2 := Eval compute in 0 -c 1.
Check (eq_refl compute2 : C1 9223372036854775807 = C1 9223372036854775807).