src/HOL/GCD.thy
changeset 80760 be8c0e039a5e
parent 80084 173548e4d5d0
child 80764 47c0aa388621
--- a/src/HOL/GCD.thy	Sun Aug 25 12:43:43 2024 +0200
+++ b/src/HOL/GCD.thy	Sun Aug 25 15:02:19 2024 +0200
@@ -153,6 +153,10 @@
   "_LCM1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3LCM _./ _)" [0, 10] 10)
   "_LCM"      :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"  ("(3LCM _\<in>_./ _)" [0, 0, 10] 10)
 
+syntax_consts
+  "_GCD1" "_GCD" \<rightleftharpoons> Gcd and
+  "_LCM1" "_LCM" \<rightleftharpoons> Lcm
+
 translations
   "GCD x y. f"   \<rightleftharpoons> "GCD x. GCD y. f"
   "GCD x. f"     \<rightleftharpoons> "CONST Gcd (CONST range (\<lambda>x. f))"
@@ -2933,6 +2937,8 @@
 
 syntax "_type_char" :: "type => nat" ("(1CHAR/(1'(_')))")
 
+syntax_consts "_type_char" == semiring_char
+
 translations "CHAR('t)" => "CONST semiring_char (CONST Pure.type :: 't itself)"
 
 print_translation \<open>