more inner-syntax markup;
authorwenzelm
Sun, 20 Oct 2024 21:51:47 +0200
changeset 81215 c9235a0cde83
parent 81214 7c2745efec69
child 81216 2fccbfca1361
more inner-syntax markup;
src/HOL/ex/Antiquote.thy
--- a/src/HOL/ex/Antiquote.thy	Sun Oct 20 21:48:38 2024 +0200
+++ b/src/HOL/ex/Antiquote.thy	Sun Oct 20 21:51:47 2024 +0200
@@ -14,8 +14,11 @@
   where "Expr exp env = exp env"
 
 syntax
-  "_Expr" :: "'a \<Rightarrow> 'a"  (\<open>EXPR _\<close> [1000] 999)
-  "_Var" :: "'a \<Rightarrow> ('a \<Rightarrow> nat) \<Rightarrow> nat"  (\<open>VAR _\<close> [1000] 999)
+  "_Expr" :: "'a \<Rightarrow> 'a"  (\<open>(\<open>notation=\<open>prefix EXPR\<close>\<close>EXPR _)\<close> [1000] 999)
+  "_Var" :: "'a \<Rightarrow> ('a \<Rightarrow> nat) \<Rightarrow> nat"  (\<open>(\<open>notation=\<open>prefix VAR\<close>\<close>VAR _)\<close> [1000] 999)
+
+syntax_consts
+  "_Expr" \<rightleftharpoons> Expr
 
 parse_translation
   \<open>[Syntax_Trans.quote_antiquote_tr