src/HOL/Proofs/Lambda/ListBeta.thy
changeset 80914 d97fdabd9e2b
parent 62390 842917225d56
--- a/src/HOL/Proofs/Lambda/ListBeta.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Proofs/Lambda/ListBeta.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -12,7 +12,7 @@
 \<close>
 
 abbreviation
-  list_beta :: "dB list => dB list => bool"  (infixl "=>" 50) where
+  list_beta :: "dB list => dB list => bool"  (infixl \<open>=>\<close> 50) where
   "rs => ss == step1 beta rs ss"
 
 lemma head_Var_reduction: