aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/program.mli
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-06-25 13:15:46 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-06-25 13:15:46 +0000
commit94a8d080d4a802ffb092fa19b84d3cd470f1e444 (patch)
tree0fa24739f4acc3fc88f1452996c8729f009075e8 /pretyping/program.mli
parent505c7b0881d68670af24fd8fe0e3c28157b2c90d (diff)
Added a .mli to pretyping/program.ml
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15490 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/program.mli')
-rw-r--r--pretyping/program.mli35
1 files changed, 35 insertions, 0 deletions
diff --git a/pretyping/program.mli b/pretyping/program.mli
new file mode 100644
index 000000000..ddb28e5a5
--- /dev/null
+++ b/pretyping/program.mli
@@ -0,0 +1,35 @@
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2010 *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
+
+open Term
+
+(** A bunch of Coq constants used by Progam *)
+
+val sig_typ : unit -> constr
+val sig_intro : unit -> constr
+val sig_proj1 : unit -> constr
+val sigT_typ : unit -> constr
+val sigT_intro : unit -> constr
+val sigT_proj1 : unit -> constr
+val sigT_proj2 : unit -> constr
+
+val prod_typ : unit -> constr
+val prod_intro : unit -> constr
+val prod_proj1 : unit -> constr
+val prod_proj2 : unit -> constr
+
+val coq_eq_ind : unit -> constr
+val coq_eq_refl : unit -> constr
+val coq_eq_refl_ref : unit -> Globnames.global_reference
+val coq_eq_rect : unit -> constr
+
+val coq_JMeq_ind : unit -> constr
+val coq_JMeq_refl : unit -> constr
+
+val mk_coq_and : constr list -> constr
+val mk_coq_not : constr -> constr