From 889dcd22b3110279525af9fcb07d5de651c685d4 Mon Sep 17 00:00:00 2001 From: filliatr Date: Wed, 21 Jun 2000 17:27:03 +0000 Subject: - $BINDER -> BINDER dans g_constr.ml4 (=> erreur syntax Fix) - suite portage Ring git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@516 85f007b7-540e-0410-9357-904b9bb8a0f7 --- contrib/ring/Ring_normalize.v | 2 +- contrib/ring/Ring_theory.v | 2 ++ parsing/g_constr.ml4 | 2 +- 3 files changed, 4 insertions(+), 2 deletions(-) diff --git a/contrib/ring/Ring_normalize.v b/contrib/ring/Ring_normalize.v index 968ce7f6b..50c667499 100644 --- a/contrib/ring/Ring_normalize.v +++ b/contrib/ring/Ring_normalize.v @@ -8,7 +8,7 @@ Implicit Arguments On. Lemma index_eq_prop: (n,m:index)(Is_true (index_eq n m)) -> n=m. Proof. - Induction n; Induction m; Simpl; Try (Reflexivity Orelse Contradiction). + Induction n; Induction m; Simpl; Try '(Reflexivity Orelse Contradiction). Intros; Rewrite (H i0); Trivial. Intros; Rewrite (H i0); Trivial. Save. diff --git a/contrib/ring/Ring_theory.v b/contrib/ring/Ring_theory.v index 4b5fff53d..09b3e5b7b 100644 --- a/contrib/ring/Ring_theory.v +++ b/contrib/ring/Ring_theory.v @@ -371,6 +371,7 @@ End Theory_of_rings. Implicit Arguments Off. +(***TODO Definition Semi_Ring_Theory_of : (A:Type)(Aplus : A -> A -> A)(Amult : A -> A -> A)(Aone : A) (Azero : A)(Aopp : A -> A)(Aeq : A -> A -> bool) @@ -390,6 +391,7 @@ Defined. (* Every ring can be viewed as a semi-ring : this property will be used in Abstract_polynom. *) Coercion Semi_Ring_Theory_of : Ring_Theory >-> Semi_Ring_Theory. +***) Section product_ring. diff --git a/parsing/g_constr.ml4 b/parsing/g_constr.ml4 index 96be64616..e9ed83a54 100644 --- a/parsing/g_constr.ml4 +++ b/parsing/g_constr.ml4 @@ -141,7 +141,7 @@ GEXTEND Gram ; vardecls: [ [ id = ident; idl = ident_comma_list_tail; c = type_option -> - <:ast< ($BINDER $c $id ($LIST $idl)) >> + <:ast< (BINDER $c $id ($LIST $idl)) >> | id = ident; "="; c = constr -> <:ast< (ABST #Core#let.cci $c $id) >> ] ] ; -- cgit v1.2.3