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 26 27 28 29 30 31 32
|
Require Import Extraction BinPos.
Require Import ExtrOcamlNatInt.
Require Import Extraction BinPos.
Definition test (a:Decimal.int) n m (H:m>0) :=
let (q,r,_,_) := Euclid.eucl_dev m H n in
(Decimal.norm a, Nat.compare n (q*m+r)).
Extraction TestCompile test.
(* Test combination of Decimal.int with ExtrOcamlInt63 *)
Require Import ExtrOCamlInt63.
Definition f n p := (CompOpp n, Decimal.norm p).
Extraction TestCompile f.
(* Test combination of Decimal.int with ExtrOcamlIntConv *)
Require Import ExtrOcamlIntConv.
Definition g n p := (n_of_int n, Decimal.norm p).
Extraction TestCompile g.
(* Test combination of Decimal.int with ExtrOcamlZInt *)
Require Import ExtrOcamlZInt ZArith.
Extraction TestCompile Z.add.
|