aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-01-11 18:55:05 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-01-11 18:55:05 +0000
commit07602743dd112779f29f17add9c318929276ccbe (patch)
tree3d20ba661400ef0632ae4b7ce46dac3d99ff3624
parent9a820584d6797b98d9ff183aef301e291c33a3b9 (diff)
Ajout d'une option de débogage pour expliciter l'instance des evars
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9479 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--interp/constrextern.ml19
-rw-r--r--interp/constrextern.mli1
2 files changed, 8 insertions, 12 deletions
diff --git a/interp/constrextern.ml b/interp/constrextern.ml
index 85ca1fac4..d38662294 100644
--- a/interp/constrextern.ml
+++ b/interp/constrextern.ml
@@ -63,9 +63,6 @@ let print_projections = ref false
let print_meta_as_hole = ref false
-(* This forces printing of evar instances *)
-let print_instances = ref false
-
let with_arguments f = Options.with_option print_arguments f
let with_implicits f = Options.with_option print_implicits f
let with_coercions f = Options.with_option print_coercions f
@@ -104,7 +101,13 @@ let idopt_of_name = function
| Name id -> Some id
| Anonymous -> None
-let extern_evar loc n = CEvar (loc,n)
+let extern_evar loc n =
+(*
+ msgerrnl (str
+ "Warning: existential variable turned into meta-variable during externalization");
+ CPatVar (loc,(false,make_ident "META" (Some n)))
+*)
+ CEvar (loc,n)
let raw_string_of_ref = function
| ConstRef kn ->
@@ -638,13 +641,7 @@ let rec extern inctx scopes vars r =
| REvar (loc,n,None) when !print_meta_as_hole -> CHole loc
- | REvar (loc,n,args) ->
- if !print_instances & args <> None then
- explicitize loc false [] (None,extern_evar loc n)
- (List.map (sub_extern true scopes vars) (out_some args))
- else
- (* we drop args *)
- extern_evar loc n
+ | REvar (loc,n,_) -> (* we drop args *) extern_evar loc n
| RPatVar (loc,n) -> if !print_meta_as_hole then CHole loc else CPatVar (loc,n)
diff --git a/interp/constrextern.mli b/interp/constrextern.mli
index f4843756e..0ffb8c333 100644
--- a/interp/constrextern.mli
+++ b/interp/constrextern.mli
@@ -51,7 +51,6 @@ val print_coercions : bool ref
val print_universes : bool ref
val print_no_symbol : bool ref
val print_projections : bool ref
-val print_instances : bool ref
(* This governs printing of implicit arguments. If [with_implicits] is
on and not [with_arguments] then implicit args are printed prefixed