src/HOL/Decision_Procs/MIR.thy
changeset 80914 d97fdabd9e2b
parent 80105 2fa018321400
--- a/src/HOL/Decision_Procs/MIR.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Decision_Procs/MIR.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -31,7 +31,7 @@
 lemmas dvd_period = zdvd_period
 
 (* The Divisibility relation between reals *)
-definition rdvd:: "real \<Rightarrow> real \<Rightarrow> bool" (infixl "rdvd" 50)
+definition rdvd:: "real \<Rightarrow> real \<Rightarrow> bool" (infixl \<open>rdvd\<close> 50)
   where "x rdvd y \<longleftrightarrow> (\<exists>k::int. y = x * real_of_int k)"
 
 lemma int_rdvd_real: