aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof.mli
diff options
context:
space:
mode:
authorGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-23 15:12:59 +0000
committerGravatar aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-23 15:12:59 +0000
commit0820caf877c5b74ebcca580d7872f1f69d19274f (patch)
tree276d5ead8da662eb0c16a47cfa710c207e2849de /proofs/proof.mli
parentce778df87e21dcbbf6885f1ccfc18556356794c6 (diff)
Enlevé les trucs commités au mauvais endroit
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10252 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/proof.mli')
-rw-r--r--proofs/proof.mli34
1 files changed, 0 insertions, 34 deletions
diff --git a/proofs/proof.mli b/proofs/proof.mli
deleted file mode 100644
index 4e30d8daf..000000000
--- a/proofs/proof.mli
+++ /dev/null
@@ -1,34 +0,0 @@
-(************************************************************************)
-(* 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: proof.mli aspiwack $ *)
-
-(* This module implements the actual proof datatype. It enforces strong
- invariants, and it is the only module that should access the module
- Subproof.
- Actually from outside the proofs/ subdirectory, this is the only module
- that should be used directly. *)
-
-open Term
-
-(* Type of a proof *)
-type 'a proof
-
-(* Type of the proof transformations *)
-type 'a transformation
-
-(* exception which represent a failure in a command.
- Opposed to anomalies and uncaught exceptions. *)
-exception Failure of Pp.std_ppcmds
-
-(* function to raise a failure less verbosely *)
-val fail : Pp.std_ppcmds -> 'a
-
-val do_command : 'a transformation -> 'a proof -> unit
-
-