aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/isar/IllegalEscape.thy
blob: 3478830b66a44be34fdf99eeef66e1ca3e292273 (plain)
1
2
3
4
5
6
7
(* See http://proofgeneral.inf.ed.ac.uk/trac/ticket/166 *)

theory IllegalEscape imports Main begin

    lemma X: "a=b ==> b=a" by simp -- "Text with \illegal escape sequence"
      oops
end