adapted to History changes;
authorwenzelm
Fri, 21 May 1999 11:39:47 +0200
changeset 6684 4f859545bd92
parent 6683 b7293047b0f4
child 6685 e33ae2af0d36
adapted to History changes;
src/Pure/Isar/proof_history.ML
--- a/src/Pure/Isar/proof_history.ML	Fri May 21 11:38:57 1999 +0200
+++ b/src/Pure/Isar/proof_history.ML	Fri May 21 11:39:47 1999 +0200
@@ -9,13 +9,12 @@
 sig
   type T
   exception FAIL of string
-  val init: Proof.state -> T
+  val init: int option -> Proof.state -> T
+  val is_initial: T -> bool
   val current: T -> Proof.state
   val clear: T -> T
   val undo: T -> T
   val redo: T -> T
-  val undos: int -> T -> T
-  val redos: int -> T -> T
   val position: T -> int
   val nesting: T -> int
   val prev: T -> T
@@ -54,15 +53,13 @@
 
 (* generic history operations *)
 
-fun init st = ProofHistory (History.init (((st, Seq.empty), 0), []));
+fun init lim st = ProofHistory (History.init lim (((st, Seq.empty), 0), []));
+fun is_initial (ProofHistory prf) = History.is_initial prf;
 fun current (ProofHistory prf) = fst (fst (fst (History.current prf)));
 val clear = app History.clear;
 val undo = app History.undo;
 val redo = app History.redo;
 
-fun undos n = funpow n undo;
-fun redos n = funpow n redo;
-
 
 (* navigate *)