aboutsummaryrefslogtreecommitdiff
path: root/proofs/tactic_debug.mli
diff options
context:
space:
mode:
authordelahaye2000-10-30 16:56:19 +0000
committerdelahaye2000-10-30 16:56:19 +0000
commit2c13632cd7296072ab5271fc047cda720f23686c (patch)
treebd6ed3886cee140c56ffdf88e83cab3d6208909e /proofs/tactic_debug.mli
parentcae025c40c270a23ffef489d855346dd86944aa6 (diff)
Tactiques utilisateur + debugger
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@786 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs/tactic_debug.mli')
-rw-r--r--proofs/tactic_debug.mli21
1 files changed, 21 insertions, 0 deletions
diff --git a/proofs/tactic_debug.mli b/proofs/tactic_debug.mli
new file mode 100644
index 0000000000..26ab1a9470
--- /dev/null
+++ b/proofs/tactic_debug.mli
@@ -0,0 +1,21 @@
+open Proof_type
+open Term
+
+(* This module intends to be a beginning of debugger for tactic expressions.
+ Currently, it is quite simple and we can hope to have, in the future, a more
+ complete panel of commands dedicated to a proof assistant framework *)
+
+(* Debug information *)
+type debug_info =
+ | DebugOn
+ | DebugOff
+ | Exit
+
+(* Prints the state and waits *)
+val debug_prompt : goal sigma option -> Coqast.t -> debug_info
+
+(* Prints a matched hypothesis *)
+val db_matched_hyp : debug_info -> Environ.env -> string * constr -> unit
+
+(* Prints the matched conclusion *)
+val db_matched_concl : debug_info -> Environ.env -> constr -> unit