From 5b8e645b675b6b2efac8e13c29da5e984248e507 Mon Sep 17 00:00:00 2001 From: barras Date: Fri, 27 Oct 2006 21:21:17 +0000 Subject: simplif de la partie ML de ring/field git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9302 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Reals/RIneq.v | 30 ------------------------------ 1 file changed, 30 deletions(-) (limited to 'theories/Reals/RIneq.v') diff --git a/theories/Reals/RIneq.v b/theories/Reals/RIneq.v index 1996eaa97..daebd9178 100644 --- a/theories/Reals/RIneq.v +++ b/theories/Reals/RIneq.v @@ -16,42 +16,12 @@ Require Export Raxioms. Require Export ZArithRing. Require Import Omega. Require Export RealField. -Require Export LegacyField. Open Local Scope Z_scope. Open Local Scope R_scope. Implicit Type r : R. -(***************************************************************************) -(** * Instantiating Field tactic on reals *) -(***************************************************************************) - -(* Legacy Field *) -Require Export LegacyField. -Import LegacyRing_theory. - -Lemma RLegacyTheory : Ring_Theory Rplus Rmult 1 0 Ropp (fun x y:R => false). - split. - exact Rplus_comm. - symmetry in |- *; apply Rplus_assoc. - exact Rmult_comm. - symmetry in |- *; apply Rmult_assoc. - intro; apply Rplus_0_l. - intro; apply Rmult_1_l. - exact Rplus_opp_r. - intros. - rewrite Rmult_comm. - rewrite (Rmult_comm n p). - rewrite (Rmult_comm m p). - apply Rmult_plus_distr_l. - intros; contradiction. -Defined. - -Add Legacy Field -R Rplus Rmult 1 0 Ropp (fun x y:R => false) Rinv RLegacyTheory Rinv_l - with minus := Rminus div := Rdiv. - (**************************************************************************) (** * Relation between orders and equality *) (**************************************************************************) -- cgit v1.2.3