From 86503800a77326db19412ea1c3e534f79dc5d6d1 Mon Sep 17 00:00:00 2001 From: filliatr Date: Fri, 19 Apr 2002 08:12:51 +0000 Subject: un thm de plus dans Zdiv; un retour chariot apres un message de la tactique FourierR git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2659 85f007b7-540e-0410-9357-904b9bb8a0f7 --- contrib/fourier/fourierR.ml | 2 +- theories/ZArith/Zdiv.v | 8 ++++++++ 2 files changed, 9 insertions(+), 1 deletion(-) 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 *) -- cgit v1.2.3