src/HOL/Auth/NS_Shared.thy
changeset 80914 d97fdabd9e2b
parent 76299 0ad6f6508274
--- a/src/HOL/Auth/NS_Shared.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Auth/NS_Shared.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -17,7 +17,7 @@
  (* A is the true creator of X if she has sent X and X never appeared on
     the trace before this event. Recall that traces grow from head. *)
   Issues :: "[agent, agent, msg, event list] \<Rightarrow> bool"
-             ("_ Issues _ with _ on _") where
+             (\<open>_ Issues _ with _ on _\<close>) where
    "A Issues B with X on evs =
       (\<exists>Y. Says A B Y \<in> set evs \<and> X \<in> parts {Y} \<and>
         X \<notin> parts (spies (takeWhile (\<lambda>z. z  \<noteq> Says A B Y) (rev evs))))"