aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/redexpr.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-01-02 08:46:18 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-01-02 08:46:18 +0000
commit6eff115a9094104eac9be09eb0e755f98366cf8d (patch)
tree62bb7fe5b47f0818cc5407c86cd4517b06f123b7 /proofs/redexpr.mli
parente4e04dfb5488330908ad14873f97d753821dd1ac (diff)
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@6544 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/redexpr.mli')
-rw-r--r--proofs/redexpr.mli31
1 files changed, 31 insertions, 0 deletions
diff --git a/proofs/redexpr.mli b/proofs/redexpr.mli
new file mode 100644
index 000000000..a0b7100b6
--- /dev/null
+++ b/proofs/redexpr.mli
@@ -0,0 +1,31 @@
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
+
+(* $Id$ *)
+
+open Names
+open Term
+open Closure
+open Rawterm
+open Reductionops
+
+(* Call by value strategy (uses virtual machine) *)
+val cbv_vm : reduction_function
+
+type red_expr = (constr, evaluable_global_reference) red_expr_gen
+
+val reduction_of_red_expr : red_expr -> reduction_function
+
+val declare_red_expr : string -> reduction_function -> unit
+
+(* Opaque and Transparent commands. *)
+val set_opaque_const : constant -> unit
+val set_transparent_const : constant -> unit
+
+val set_opaque_var : identifier -> unit
+val set_transparent_var : identifier -> unit