Theory Chinese

(*  Author:     Ning Zhang and Christian Urban

Example theory involving Unicode characters (UTF-8 encoding) -- both
formal and informal ones.
*)

section ‹A Chinese theory›

theory Chinese imports Main begin

text‹数学家能把咖啡变成理论,如今中国的数学家也可
       以在伊莎贝拉的帮助下把茶变成理论.  

       伊莎贝拉-世界数学家的新宠,现今能识别中文,成为
       中国数学家理论推导的得力助手.

›

datatype shuzi =
    One   ("")
  | Two   ("")
  | Three ("") 
  | Four  ("")
  | Five  ("")
  | Six   ("")
  | Seven ("")
  | Eight ("")
  | Nine  ("")
  | Ten   ("")

primrec translate :: "shuzi  nat" ("|_|" [100] 100) where
 "|| = 1"
|"|| = 2"
|"|| = 3"
|"|| = 4"
|"|| = 5"
|"|| = 6"
|"|| = 7"
|"|| = 8"
|"|| = 9"
|"|| = 10"

thm translate.simps

lemma "|| + || = ||"
  by simp 

end