aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/AHundredTheorems.thy
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-04 16:35:49 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2009-09-04 16:35:49 +0000
commite516288796182bb3a7cd6d10ecbee34a902d78b5 (patch)
tree38e3390b1387ef5cd0bbb8e53db83f0e56a7005c /etc/isar/AHundredTheorems.thy
parenta0351c6691d7892cc3dbd047280719041b903701 (diff)
Add Elisp timings
Diffstat (limited to 'etc/isar/AHundredTheorems.thy')
-rw-r--r--etc/isar/AHundredTheorems.thy10
1 files changed, 9 insertions, 1 deletions
diff --git a/etc/isar/AHundredTheorems.thy b/etc/isar/AHundredTheorems.thy
index 08e4c03a..cc2aebe7 100644
--- a/etc/isar/AHundredTheorems.thy
+++ b/etc/isar/AHundredTheorems.thy
@@ -1,8 +1,9 @@
theory AHundredTheorems imports Main
begin
-ML {* val start = start_timing(); *}
+(* ELISP: -- (setq start (current-time)) -- *)
+ML {* val start = start_timing(); *}
lemma foo: "P --> P" by auto
lemma foo2: "P --> P" by auto
@@ -105,6 +106,13 @@ lemma foo98: "P --> P" by auto
lemma foo99: "P --> P" by auto
lemma foo100: "P --> P" by auto
+
+(* NB: this doesn't work because of comment aggregation *)
+(* ELISP: -- (message "Time taken: %f seconds" (time-to-seconds (time-since start))) -- *)
ML {* Output.warning (#message (end_timing start)); *}
end
+
+
+
+