level: do not account for local theory blocks (relevant for document preparation);
authorwenzelm
Sat, 11 Nov 2006 21:13:12 +0100
changeset 21310 bfcc24fc7c46
parent 21309 367f4512e65c
child 21311 3556301c18cd
level: do not account for local theory blocks (relevant for document preparation);
src/Pure/Isar/toplevel.ML
--- a/src/Pure/Isar/toplevel.ML	Sat Nov 11 21:13:11 2006 +0100
+++ b/src/Pure/Isar/toplevel.ML	Sat Nov 11 21:13:12 2006 +0100
@@ -161,10 +161,9 @@
 fun level (State NONE) = 0
   | level (State (SOME (node, _))) =
       (case History.current node of
-        Theory (Context.Theory _, _) => 0
-      | Theory (Context.Proof _, _) => 1
-      | Proof (prf, _) => Proof.level (ProofHistory.current prf) + 1
-      | SkipProof (h, _) => History.current h + 2);   (*different notion of proof depth!*)
+        Theory _ => 0
+      | Proof (prf, _) => Proof.level (ProofHistory.current prf)
+      | SkipProof (h, _) => History.current h + 1);   (*different notion of proof depth!*)
 
 fun str_of_state (State NONE) = "at top level"
   | str_of_state (State (SOME (node, _))) =