aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-10-13 13:09:41 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-10-13 13:09:41 +0000
commit3690735581c7995e4be17c3a3029e66ddf2d3e49 (patch)
tree68dde8eac50aa60d99cbe93cf1679af55edc8dea /contrib
parent6272fe2c65ccace5982515ec58398505a22855dc (diff)
Mise en place de 'Scope' pour gérer des ensembles de notations - phase 1; hack temporaire autour du printer
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3120 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib')
-rw-r--r--contrib/interface/xlate.ml17
-rw-r--r--contrib/romega/ReflOmegaCore.v2
2 files changed, 13 insertions, 6 deletions
diff --git a/contrib/interface/xlate.ml b/contrib/interface/xlate.ml
index 4e4b51833..d8663f09d 100644
--- a/contrib/interface/xlate.ml
+++ b/contrib/interface/xlate.ml
@@ -311,8 +311,8 @@ let ident_or_meta_to_ct_ID = function
let xlate_qualid_list l = CT_id_list (List.map loc_qualid_to_ct_ID l)
let reference_to_ct_ID = function
- | RIdent (_,id) -> CT_ident (Names.string_of_id id)
- | RQualid (_,qid) -> CT_ident (Libnames.string_of_qualid qid)
+ | Coqast.RIdent (_,id) -> CT_ident (Names.string_of_id id)
+ | Coqast.RQualid (_,qid) -> CT_ident (Libnames.string_of_qualid qid)
let xlate_class = function
| FunClass -> CT_ident "FUNCLASS"
@@ -986,7 +986,7 @@ and (xlate_call_or_tacarg:raw_tactic_arg -> ct_TACTIC_COM) =
(reference_to_ct_ID r,
CT_tactic_arg_list(xlate_tacarg a,List.map xlate_tacarg l))
| TacCall (_,_,_) -> xlate_error ""
- | Reference (RIdent (_,s)) -> ident_tac s
+ | Reference (Coqast.RIdent (_,s)) -> ident_tac s
| t -> xlate_error "TODO: result other than tactic or constr"
and xlate_red_tactic =
@@ -1906,7 +1906,14 @@ let xlate_vernac =
| ("SYNTAX", [Varg_ident phy; Varg_ident s; spatarg; unparg]) ->
(syntaxop phy s spatarg unparg
coerce_ID_OPT_to_FORMULA_OPT(CT_coerce_NONE_to_ID_OPT(CT_none)))*)
- | VernacInfix (str_assoc, n, str, id) ->
+ | VernacOpenScope sc -> xlate_error "TODO: open scope"
+
+ | VernacDelimiters _ -> xlate_error "TODO: Delimiters"
+
+ | VernacNotation _ -> xlate_error "TODO: Notation"
+
+ | VernacInfix (str_assoc, n, str, id, sc) ->
+ (* TODO: handle scopes *)
CT_infix (
(match str_assoc with
| Some Gramext.LeftA -> CT_lefta
@@ -1949,7 +1956,7 @@ let xlate_vernac =
VernacSetOption (_, _)|VernacUnsetOption _|VernacDeclareImplicits (_, _)|
VernacHintDestruct (_, _, _, _, _)|VernacBack _|VernacRestoreState _|
VernacWriteState _|VernacSolveExistential (_, _)|VernacCanonical _|
- VernacImport (_, _)|VernacExactProof _|VernacDistfix (_, _, _, _)|
+ VernacImport (_, _)|VernacExactProof _|VernacDistfix (_, _, _, _, _)|
VernacTacticGrammar _|VernacVar _|VernacTime _|VernacNop|VernacComments _)
-> xlate_error "TODO: vernac"
diff --git a/contrib/romega/ReflOmegaCore.v b/contrib/romega/ReflOmegaCore.v
index f0ccfb886..0df34f422 100644
--- a/contrib/romega/ReflOmegaCore.v
+++ b/contrib/romega/ReflOmegaCore.v
@@ -1622,7 +1622,7 @@ Theorem exact_divide_valid :
Unfold valid1 exact_divide; Intros k1 k2 t e p1; (Simplify ());Simpl; Auto;
(Elim_eq_term '(scalar_norm t (Tmult k2 (Tint k1))) 't1); Simpl; Auto;
-(Elim_eq_Z 'k1 'ZERO); Simpl; Auto; Intros H1 H2; Elim H2;
+(Elim_eq_Z 'k1 '(ZERO)); Simpl; Auto; Intros H1 H2; Elim H2;
Elim scalar_norm_stable; Simpl; Generalize H1; Case (interp_term e k2);
Try Trivial; (Case k1; Simpl; [
Intros; Absurd `0 = 0`; Assumption