src/HOL/ex/Tarski.thy
changeset 80914 d97fdabd9e2b
parent 70202 373eb0aa97e3
child 82248 e8c96013ea8a
--- a/src/HOL/ex/Tarski.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/ex/Tarski.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -80,7 +80,7 @@
     (SIGMA cl : CompleteLattice.
       {S. S \<subseteq> pset cl \<and> \<lparr>pset = S, order = induced S (order cl)\<rparr> \<in> CompleteLattice})"
 
-abbreviation sublat :: "['a set, 'a potype] \<Rightarrow> bool"  ("_ <<= _" [51, 50] 50)
+abbreviation sublat :: "['a set, 'a potype] \<Rightarrow> bool"  (\<open>_ <<= _\<close> [51, 50] 50)
   where "S <<= cl \<equiv> S \<in> sublattice `` {cl}"
 
 definition dual :: "'a potype \<Rightarrow> 'a potype"