aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-19 14:31:51 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-19 14:31:51 +0000
commitcff24d313545efba6bd14116b83bd3fa0b7f44ff (patch)
treea1c77555098c23f0a7271c0d668bad6aee20b97b /parsing
parent26f2ff64a641f1767abb1a0d3da3e7449a5835d3 (diff)
Distinction entre 'as _' qui cache le terme filtre (si variable) et rien dans case_item
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4949 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'parsing')
-rw-r--r--parsing/g_cases.ml48
-rw-r--r--parsing/g_constrnew.ml45
2 files changed, 5 insertions, 8 deletions
diff --git a/parsing/g_cases.ml4 b/parsing/g_cases.ml4
index 2c5640d18..56c522948 100644
--- a/parsing/g_cases.ml4
+++ b/parsing/g_cases.ml4
@@ -57,17 +57,17 @@ GEXTEND Gram
operconstr: LEVEL "1"
[ [ "<"; p = annot; ">"; "Cases"; lc = LIST1 constr; "of";
OPT "|"; eqs = ne_eqn_list; "end" ->
- let lc = List.map (fun c -> c,(Names.Anonymous,None)) lc in
+ let lc = List.map (fun c -> c,(None,None)) lc in
CCases (loc, (Some p,None), lc, eqs)
| "Cases"; lc = LIST1 constr; "of";
OPT "|"; eqs = ne_eqn_list; "end" ->
- let lc = List.map (fun c -> c,(Names.Anonymous,None)) lc in
+ let lc = List.map (fun c -> c,(None,None)) lc in
CCases (loc, (None,None), lc, eqs)
| "<"; p = annot; ">"; "Cases"; lc = LIST1 constr; "of"; "end" ->
- let lc = List.map (fun c -> c,(Names.Anonymous,None)) lc in
+ let lc = List.map (fun c -> c,(None,None)) lc in
CCases (loc, (Some p,None), lc, [])
| "Cases"; lc = LIST1 constr; "of"; "end" ->
- let lc = List.map (fun c -> c,(Names.Anonymous,None)) lc in
+ let lc = List.map (fun c -> c,(None,None)) lc in
CCases (loc, (None,None), lc, []) ] ]
;
END;
diff --git a/parsing/g_constrnew.ml4 b/parsing/g_constrnew.ml4
index 8aebc87bb..cf7dafb47 100644
--- a/parsing/g_constrnew.ml4
+++ b/parsing/g_constrnew.ml4
@@ -257,10 +257,7 @@ GEXTEND Gram
br=branches; "end" -> mk_match (loc,ci,ty,br) ] ]
;
case_item:
- [ [ c=operconstr LEVEL "100"; p=pred_pattern ->
- match p with
- | (None,indp) -> (c,(Anonymous,indp))
- | (Some na,indp) -> (c,(na,indp)) ] ]
+ [ [ c=operconstr LEVEL "100"; p=pred_pattern -> (c,p) ] ]
;
pred_pattern:
[ [ ona = OPT ["as"; id=name -> snd id];