aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-12-06 22:24:18 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-12-06 22:24:18 +0000
commit8e1c1ee13bbcab295a92928557515b4239e4bc46 (patch)
treeb382f4cef00c0cae68aed68e21f85250f663c7e8
parentb5d1aae31455d56e90424bb5c71d172a12df7240 (diff)
MAJ
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@218 85f007b7-540e-0410-9357-904b9bb8a0f7
-rwxr-xr-xsyntax/PPCommand.v21
-rw-r--r--syntax/PPTactic.v19
2 files changed, 13 insertions, 27 deletions
diff --git a/syntax/PPCommand.v b/syntax/PPCommand.v
index 4a39c94c1..0033807bd 100755
--- a/syntax/PPCommand.v
+++ b/syntax/PPCommand.v
@@ -31,7 +31,7 @@ Syntax constr
(* Things parsed in command0 *)
level 0:
prop [(PROP)] -> ["Prop"]
- | set [(SET)] -> ["Set"]
+ | set [(SET)] -> ["Set"]
| type [(TYPE)] -> ["Type"]
| type_sp [(TYPE ($PATH $sp) ($NUM $n))] -> ["Type"]
(* Note: Atomic constants (Nvar, CONST, MUTIND, MUTCONSTRUCT) are printed in
@@ -40,6 +40,7 @@ Syntax constr
| evar [<< ? >>] -> ["?"]
| meta [(META ($NUM $n))] -> [ "?" $n ]
| implicit [(IMPLICIT)] -> ["<Implicit>"]
+ | indice [(REL ($NUM $n))] -> ["<Unbound ref: " $n ">"]
;
(* Things parsed in command1 *)
@@ -103,7 +104,7 @@ Syntax constr
| prod_cons [(PRODBOX (BINDERS ($LIST $acc)) <<($x : $Dom)$body>>)]
-> [(PRODBOX (BINDERS ($LIST $acc) (BINDER $Dom $x)) $body)]
- | prodl_start [(PRODBOX $pbi (PRODLIST $Dom $Body))]
+ | prodl_start_cons [(PRODBOX $pbi (PRODLIST $Dom $Body))]
-> [(PRODLBOX $pbi $Dom (IDS) $Body)]
| prodl_end [(PRODLBOX (BINDERS ($LIST $acc)) $c (IDS ($LIST $ids)) $t)]
@@ -116,7 +117,7 @@ Syntax constr
| arrow [<< $A -> $B >>] -> [ [<hv 0> $A:L [0 0] "->" (ARROWBOX $B) ] ]
| arrow_stop [(ARROWBOX $c)] -> [ $c:E ]
- | arrow_again [(ARROWBOX << $A -> $B >>)] -> [ $A:L [0 0] "->" (ARROWBOX $B)]
+ | arrow_again [(ARROWBOX << $A -> $B >>)] -> [ $A:L [0 0] "->" (ARROWBOX $B) ]
;
(* Things parsed in command9 *)
@@ -126,13 +127,13 @@ Syntax constr
app_cons [(APPLIST $H ($LIST $T))]
-> [ [<hov 0> $H:E (APPTAIL ($LIST $T)):E ] ]
- | app_imp [(APPLIST (XTRA "!" $H) ($LIST $T))]
+ | app_imp [(APPLISTEXPL $H ($LIST $T))]
-> [ (APPLISTIMPL (ACC $H) ($LIST $T)):E ]
| app_imp_arg [(APPLISTIMPL (ACC ($LIST $AC)) $a ($LIST $T))]
-> [ (APPLISTIMPL (ACC ($LIST $AC) $a) ($LIST $T)):E ]
- | app_imp_imp_arg [ (APPLISTIMPL $AC (XTRA "!" $_ $_) ($LIST $T)) ]
+ | app_imp_imp_arg [ (APPLISTIMPL $AC (EXPL $_ $_) ($LIST $T)) ]
-> [ (APPLISTIMPL $AC ($LIST $T)):E ]
| app_imp_last [(APPLISTIMPL (ACC ($LIST $A)) $T)]
@@ -142,15 +143,15 @@ Syntax constr
| apptailcons
[ (APPTAIL $H ($LIST $T))] -> [ [1 1] $H:L (APPTAIL ($LIST $T)):E ]
| apptailnil [(APPTAIL)] -> [ ]
- | apptailcons1 [(APPTAIL (XTRA "!" $n $c1) ($LIST $T))]
- -> [ [1 1] (XTRA "!" $n $c1):L (APPTAIL ($LIST $T)):E ]
+ | apptailcons1 [(APPTAIL (EXPL "!" $n $c1) ($LIST $T))]
+ -> [ [1 1] (EXPL $n $c1):L (APPTAIL ($LIST $T)):E ]
;
(* Implicits *)
level 8:
- arg_implicit [(XTRA "!" ($NUM $n) $c1)] -> [ $n "!" $c1:L ]
- | arg_implicit1 [(XTRA "!" "EX" ($NUM $n) $c1)] -> [ $n "!" $c1:L ]
- | fun_explicit [(XTRA "!" $f)] -> [ $f ]
+ arg_implicit [(EXPL ($NUM $n) $c1)] -> [ $n "!" $c1:L ]
+ | arg_implicit1 [(EXPL "EX" ($NUM $n) $c1)] -> [ $n "!" $c1:L ]
+ | fun_explicit [(EXPL $f)] -> [ $f ]
;
diff --git a/syntax/PPTactic.v b/syntax/PPTactic.v
index e97df073f..62c3319a0 100644
--- a/syntax/PPTactic.v
+++ b/syntax/PPTactic.v
@@ -1,17 +1,5 @@
-(****************************************************************************)
-(* The Calculus of Inductive Constructions *)
-(* *)
-(* Projet Coq *)
-(* *)
-(* INRIA LRI-CNRS ENS-CNRS *)
-(* Rocquencourt Orsay Lyon *)
-(* *)
-(* Coq V6.3 *)
-(* July 1st 1999 *)
-(* *)
-(****************************************************************************)
-(* PPTactic.v *)
-(****************************************************************************)
+
+(* $Id$ *)
(* ======================================= *)
(* PP rules for basic elements *)
@@ -325,6 +313,3 @@ Syntax tactic
level 8:
command [(COMMAND $c)] -> [ (PPUNI$COMMAND $c):E ].
-
-
-(* $Id$ *)