aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Wellfounded/Lexicographic_Product.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-11-24 23:08:09 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-11-24 23:08:09 +0000
commita2669e5c949d39cb4c05549cbcf405db65249285 (patch)
tree4bc1159ef1f1dbb55d9bfbfcc565472e2bada4a7 /theories/Wellfounded/Lexicographic_Product.v
parente3038e0822548b90792903ccb460a0e61f1cadaf (diff)
Remplacement de Syntactic Definition par Notation
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3267 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Wellfounded/Lexicographic_Product.v')
-rw-r--r--theories/Wellfounded/Lexicographic_Product.v7
1 files changed, 3 insertions, 4 deletions
diff --git a/theories/Wellfounded/Lexicographic_Product.v b/theories/Wellfounded/Lexicographic_Product.v
index 3e8ba318a..39b00e676 100644
--- a/theories/Wellfounded/Lexicographic_Product.v
+++ b/theories/Wellfounded/Lexicographic_Product.v
@@ -23,8 +23,7 @@ Variable B:A->Set.
Variable leA: A->A->Prop.
Variable leB: (x:A)(B x)->(B x)->Prop.
-
-Syntactic Definition LexProd := (lexprod A B leA leB).
+Notation LexProd := (lexprod A B leA leB).
Hints Resolve t_step Acc_clos_trans wf_clos_trans.
@@ -86,7 +85,7 @@ Section Wf_Symmetric_Product.
Variable leA: A->A->Prop.
Variable leB: B->B->Prop.
- Syntactic Definition Symprod := (symprod A B leA leB).
+ Notation Symprod := (symprod A B leA leB).
(*i
Local sig_prod:=
@@ -135,7 +134,7 @@ Section Swap.
Variable A:Set.
Variable R:A->A->Prop.
- Syntactic Definition SwapProd :=(swapprod A R).
+ Notation SwapProd :=(swapprod A R).
Lemma swap_Acc: (x,y:A)(Acc A*A SwapProd (x,y))->(Acc A*A SwapProd (y,x)).