aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib
diff options
context:
space:
mode:
authorGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-18 15:43:17 +0000
committerGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-18 15:43:17 +0000
commit7f69511216f0ef262e89e3711a93230e2103be4d (patch)
tree474100cba9f0ffc7aaba72a3a930c28773ac0679 /contrib
parent7cee3c25f72c6ad8350e129c4dd39f38abd9805a (diff)
Correcting a problem of s that appears behind a Let when there are
several variables introduced (showproof.ml) Added CASTEDOPENCOMMAND, QUALIDCONSTARG as variants in several places (xlate.ml) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1604 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib')
-rw-r--r--contrib/interface/showproof.ml1
-rw-r--r--contrib/interface/xlate.ml6
2 files changed, 4 insertions, 3 deletions
diff --git a/contrib/interface/showproof.ml b/contrib/interface/showproof.ml
index ad6544a0b..56d395e44 100644
--- a/contrib/interface/showproof.ml
+++ b/contrib/interface/showproof.ml
@@ -365,6 +365,7 @@ let txtn n s =
|"an" -> ""
|"une" -> "des"
|"Soit" -> "Soient"
+ |"Let" -> "Let"
| s -> s^"s"
;;
diff --git a/contrib/interface/xlate.ml b/contrib/interface/xlate.ml
index a616d2190..0d15dc58e 100644
--- a/contrib/interface/xlate.ml
+++ b/contrib/interface/xlate.ml
@@ -291,7 +291,7 @@ let make_casec casety =
let qualid_to_ct_ID =
function
Nvar(_, s) -> Some(CT_ident s)
- | Node(_, ("QUALID"|"QUALIDARG"), l) ->
+ | Node(_, ("QUALID"|"QUALIDARG"|"QUALIDCONSTARG"), l) ->
(* // to be modified when qualified identifiers are introducted. *)
let rec f =
function
@@ -992,7 +992,7 @@ let rec cvt_arg =
Targ_unfold_ne_list(
CT_unfold_ne_list(mk_unfold_occ fst, List.map mk_unfold_occ l))
| Node (_, "COMMAND", (c :: [])) -> Targ_command (xlate_formula c)
- | Node (_, "CASTEDCOMMAND", (c :: [])) -> Targ_command (xlate_formula c)
+ | Node (_, ("CASTEDCOMMAND"|"CASTEDOPENCOMMAND"), (c :: [])) -> Targ_command (xlate_formula c)
| Node (_, "BINDINGS", bl) ->
Targ_spec_list (filter_binding_or_command_list (List.map cvt_arg bl))
| Node (_, "BINDING", ((Node (_, "COMMAND", (c :: []))) :: [])) ->
@@ -1533,7 +1533,7 @@ let rec cvt_varg =
Varg_call (CT_ident na, List.map cvt_varg l)
| Node (_, "VERNACCALL", ((Id (_, na)) :: l)) ->
Varg_call (CT_ident na, List.map cvt_varg l)
- | Node (_, "QUALIDARG", _) as it ->
+ | Node (_, ("QUALIDARG"|"QUALIDCONSTARG"), _) as it ->
(match qualid_to_ct_ID it with
Some x -> Varg_ident x
| None -> assert false)