aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/NamesInStrings.thy
diff options
context:
space:
mode:
authorGravatar David Aspinall <da@inf.ed.ac.uk>2004-06-17 21:40:20 +0000
committerGravatar David Aspinall <da@inf.ed.ac.uk>2004-06-17 21:40:20 +0000
commit05f5c056220fcf555b2b9a64a8657f580f07a4e7 (patch)
treefab14055299ed817681b8b54c5c7fbc7117681b5 /etc/isar/NamesInStrings.thy
parent3af94770dad3d79ab3b2fe6b5138fdd1b98bd9c4 (diff)
Make theory name match file name
Diffstat (limited to 'etc/isar/NamesInStrings.thy')
-rw-r--r--etc/isar/NamesInStrings.thy2
1 files changed, 1 insertions, 1 deletions
diff --git a/etc/isar/NamesInStrings.thy b/etc/isar/NamesInStrings.thy
index b71e2dfc..3d56e8c8 100644
--- a/etc/isar/NamesInStrings.thy
+++ b/etc/isar/NamesInStrings.thy
@@ -1,4 +1,4 @@
-theory "a b" = Main: (* NB: must also check case without quotes! *)
+theory "Names In Strings" = Main: (* NB: must also check case without quotes! *)
lemma foo: "B --> B" by auto