aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/romega
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-11 21:37:15 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-07-11 21:37:15 +0000
commit0c4965dd44ae43fc4fdae29854584281d1cf82cc (patch)
treed7eead5a23628f91ba1700388bdffadc8a190881 /contrib/romega
parent4a1f2e27312d8a6a97179d0f70378e057d214890 (diff)
Ajout de quelques Arguments Scope pour simuler la récursivité du scope romega_scope en compensation (et anticipation) d'une suppression de la récursivité des délimiteurs de scope (ici %term)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9041 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/romega')
-rw-r--r--contrib/romega/ReflOmegaCore.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/contrib/romega/ReflOmegaCore.v b/contrib/romega/ReflOmegaCore.v
index 2aa3516f1..83ea5b637 100644
--- a/contrib/romega/ReflOmegaCore.v
+++ b/contrib/romega/ReflOmegaCore.v
@@ -49,6 +49,11 @@ Inductive term : Set :=
| Tvar : nat -> term.
Delimit Scope romega_scope with term.
+Arguments Scope Tplus [romega_scope romega_scope].
+Arguments Scope Tmult [romega_scope romega_scope].
+Arguments Scope Tminus [romega_scope romega_scope].
+Arguments Scope Topp [romega_scope romega_scope].
+
Infix "+" := Tplus : romega_scope.
Infix "*" := Tmult : romega_scope.
Infix "-" := Tminus : romega_scope.