aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--contrib/fourier/fourierR.ml2
-rw-r--r--theories/ZArith/Zdiv.v8
2 files changed, 9 insertions, 1 deletions
diff --git a/contrib/fourier/fourierR.ml b/contrib/fourier/fourierR.ml
index b3e141822..74a58b11d 100644
--- a/contrib/fourier/fourierR.ml
+++ b/contrib/fourier/fourierR.ml
@@ -436,7 +436,7 @@ let rec fourier gl=
let res=fourier_lineq (!lineq) in
let tac=ref tclIDTAC in
if res=[]
- then (print_string "Tactic Fourier fails.";
+ then (print_string "Tactic Fourier fails.\n";
flush stdout)
(* l'algorithme de Fourier a réussi: on va en tirer une preuve Coq *)
else (match res with
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index d3aa637bb..b7876f340 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -181,6 +181,14 @@ Intros.
Absurd `(NEG p)>0`; [ Generalize (NEG_lt_ZERO p); Omega | Omega ].
Qed.
+Theorem Z_div_mod_eq : (a,b:Z)`b > 0` -> `a = b * (Zdiv a b) + (Zmod a b)`.
+Proof.
+Unfold Zdiv Zmod.
+Intros a b Hb.
+Generalize (Z_div_mod a b Hb).
+Pattern (Zdiv_eucl a b).
+Case (Zdiv_eucl); Tauto.
+Save.
(** Existence theorems *)