src/HOL/ex/Chinese.thy
changeset 80914 d97fdabd9e2b
parent 61343 5b5656a63bd6
--- a/src/HOL/ex/Chinese.thy	Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/ex/Chinese.thy	Fri Sep 20 19:51:08 2024 +0200
@@ -17,18 +17,18 @@
 \<close>
 
 datatype shuzi =
-    One   ("一")
-  | Two   ("二")
-  | Three ("三") 
-  | Four  ("四")
-  | Five  ("五")
-  | Six   ("六")
-  | Seven ("七")
-  | Eight ("八")
-  | Nine  ("九")
-  | Ten   ("十")
+    One   (\<open>一\<close>)
+  | Two   (\<open>二\<close>)
+  | Three (\<open>三\<close>) 
+  | Four  (\<open>四\<close>)
+  | Five  (\<open>五\<close>)
+  | Six   (\<open>六\<close>)
+  | Seven (\<open>七\<close>)
+  | Eight (\<open>八\<close>)
+  | Nine  (\<open>九\<close>)
+  | Ten   (\<open>十\<close>)
 
-primrec translate :: "shuzi \<Rightarrow> nat" ("|_|" [100] 100) where
+primrec translate :: "shuzi \<Rightarrow> nat" (\<open>|_|\<close> [100] 100) where
  "|一| = 1"
 |"|二| = 2"
 |"|三| = 3"