aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/command.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-01-02 08:48:46 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-01-02 08:48:46 +0000
commit38f06f8024d3f338983105ffdb323ccd7c0db935 (patch)
treed499a88f2f92f3ec0444c69d6c51d32334d43041 /toplevel/command.ml
parent6684253c156d0a8c775bcf534ed602060d65c234 (diff)
Renommage symbols.ml{,i} en notation.ml{,i} pour permettre le chargement de printers dans ocamldebug; partie reduction_of_red_expr de tacred.ml qui dépend de la vm maintenant dans redexpr.ml
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6550 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel/command.ml')
-rw-r--r--toplevel/command.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/toplevel/command.ml b/toplevel/command.ml
index a7f39f053..42e18fadc 100644
--- a/toplevel/command.ml
+++ b/toplevel/command.ml
@@ -18,7 +18,7 @@ open Entries
open Inductive
open Environ
open Reduction
-open Tacred
+open Redexpr
open Declare
open Nametab
open Names
@@ -37,7 +37,7 @@ open Indtypes
open Vernacexpr
open Decl_kinds
open Pretyping
-open Symbols
+open Notation
let mkLambdaCit = List.fold_right (fun (x,a) b -> mkLambdaC(x,a,b))
let mkProdCit = List.fold_right (fun (x,a) b -> mkProdC(x,a,b))
@@ -124,7 +124,7 @@ let red_constant_entry bl ce = function
| Some red ->
let body = ce.const_entry_body in
{ ce with const_entry_body =
- under_binders (Global.env()) (reduction_of_redexp red)
+ under_binders (Global.env()) (reduction_of_red_expr red)
(length_of_raw_binders bl)
body }