src/HOL/HOLCF/IOA/Seq.thy
changeset 80914 d97fdabd9e2b
parent 66453 cc19f7ca2ed6
--- a/src/HOL/HOLCF/IOA/Seq.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/HOLCF/IOA/Seq.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -10,7 +10,7 @@
 
 default_sort pcpo
 
-domain (unsafe) 'a seq = nil  ("nil") | cons (HD :: 'a) (lazy TL :: "'a seq")  (infixr "##" 65)
+domain (unsafe) 'a seq = nil  (\<open>nil\<close>) | cons (HD :: 'a) (lazy TL :: "'a seq")  (infixr \<open>##\<close> 65)
 
 inductive Finite :: "'a seq \<Rightarrow> bool"
 where
@@ -108,7 +108,7 @@
   sconc_nil: "sconc \<cdot> nil \<cdot> y = y"
 | sconc_cons': "x \<noteq> UU \<Longrightarrow> sconc \<cdot> (x ## xs) \<cdot> y = x ## (sconc \<cdot> xs \<cdot> y)"
 
-abbreviation sconc_syn :: "'a seq \<Rightarrow> 'a seq \<Rightarrow> 'a seq"  (infixr "@@" 65)
+abbreviation sconc_syn :: "'a seq \<Rightarrow> 'a seq \<Rightarrow> 'a seq"  (infixr \<open>@@\<close> 65)
   where "xs @@ ys \<equiv> sconc \<cdot> xs \<cdot> ys"
 
 lemma sconc_UU [simp]: "UU @@ y = UU"