aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/AHundredProofs.thy
diff options
context:
space:
mode:
Diffstat (limited to 'etc/isar/AHundredProofs.thy')
-rw-r--r--etc/isar/AHundredProofs.thy7
1 files changed, 4 insertions, 3 deletions
diff --git a/etc/isar/AHundredProofs.thy b/etc/isar/AHundredProofs.thy
index 6f59f4e0..2687b306 100644
--- a/etc/isar/AHundredProofs.thy
+++ b/etc/isar/AHundredProofs.thy
@@ -1,7 +1,8 @@
-theory AHundredProofs imports Main
+theory AHundredProofs
+imports Main
begin
-ML {* val start = start_timing(); *}
+ML {* val start = Timing.start () *}
theorem and_comms1: "A & B --> B & A"
proof
@@ -1003,6 +1004,6 @@ proof
qed
qed
-ML {* Output.warning (#message (end_timing start)); *}
+ML {* warning (Timing.message (Timing.result start)) *}
end