aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Ints/num/BigQ.v
blob: bd889e12f261538e799e01fe3df8eb6580e45c6c (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
Require Export QMake_base.
Require Import QpMake.
Require Import QvMake.
Require Import Q0Make.
Require Import QifMake.
Require Import QbiMake.

(* We choose for Q the implemention with
   multiple representation of 0: 0, 1/0, 2/0 etc *)
Module BigQ := Q0.

Definition bigQ := BigQ.t.

Delimit Scope bigQ_scope with bigQ.
Bind Scope bigQ_scope with bigQ.
Bind Scope bigQ_scope with BigQ.t.

Notation " i + j " := (BigQ.add i j) : bigQ_scope.
Notation " i - j " := (BigQ.sub i j) : bigQ_scope.
Notation " i * j " := (BigQ.mul i j) : bigQ_scope.
Notation " i / j " := (BigQ.div i j) : bigQ_scope.
Notation " i ?= j " := (BigQ.compare i j) : bigQ_scope.