aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coq.mli
diff options
context:
space:
mode:
authorGravatar vgross <vgross@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-26 19:31:28 +0000
committerGravatar vgross <vgross@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-26 19:31:28 +0000
commit0a6175c36e3b4185e5b6a3c6f019dff108ef5cfe (patch)
treea775f6ab570b0b03a9c6a5dc6768d54d047fa4d2 /ide/coq.mli
parent9731a6e86bac7206a2a52c4a47d51c5c439f3bb5 (diff)
New API for backtracking.
Aside the command stack, the only parameter is the number of step to go back. Went back and forth without sync losses on tests-suite/ide/undo.v. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12821 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'ide/coq.mli')
-rw-r--r--ide/coq.mli5
1 files changed, 1 insertions, 4 deletions
diff --git a/ide/coq.mli b/ide/coq.mli
index 27a0dfe45..e863288cd 100644
--- a/ide/coq.mli
+++ b/ide/coq.mli
@@ -54,10 +54,7 @@ val interp_and_replace : string ->
val push_phrase : ('a * reset_info) Stack.t -> reset_info -> 'a -> unit
-type undo_cmds
-val init_undo_cmds : unit -> undo_cmds
-val pop_command : ('a * reset_info) Stack.t -> undo_cmds -> undo_cmds
-val apply_undos : ('a * reset_info) Stack.t -> undo_cmds -> unit
+val old_rewind : int -> ('a * reset_info) Stack.t -> unit
val is_vernac_tactic_command : Vernacexpr.vernac_expr -> bool
val is_vernac_state_preserving_command : Vernacexpr.vernac_expr -> bool