aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/NamesInStrings.thy
blob: 366b9a2a5e2f48fa7c9bf4a42e19c900cc7b7209 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
theory "Names In Strings" imports Main begin   (* NB: must also check case without quotes! *)

lemma foo: "B --> B" by auto

lemma "foo bar": "B --> B" by auto

lemma "foo-wiggle-bar": "B --> B" by auto

theorem "x b": "B --> B" by auto

(* NB: various other regexps and settings based on them are sensitive
   to grouping in isar-name-regexp: should check function menu, imenu,
   as well as undo behaviour. *)

end


(*

I noticed the following minor problem with Isabelle and 
ProofGeneral:


>>   theory "a" = Main:
>>   Proof General -> Use -> Retract:
>>   *** Outer syntax error: end of input expected,
>>   *** but identifier "a" was found

Regards,
Tjark

*)