src/HOL/ex/Code_Lazy_Demo.thy
changeset 81090 843dba3d307a
parent 81019 dd59daa3c37a
child 81091 c007e6d9941d
--- a/src/HOL/ex/Code_Lazy_Demo.thy	Mon Sep 30 22:57:45 2024 +0200
+++ b/src/HOL/ex/Code_Lazy_Demo.thy	Mon Sep 30 23:32:26 2024 +0200
@@ -40,7 +40,7 @@
   | LCons (lhd: 'a) (ltl: "'a llist") (infixr \<open>###\<close> 65)
 
 syntax
-  "_llist" :: "args => 'a list"    (\<open>\<^bold>\<lbrakk>(\<open>notation=\<open>mixfix lazy list enumeration\<close>\<close>_)\<^bold>\<rbrakk>\<close>)
+  "_llist" :: "args => 'a list"  (\<open>(\<open>indent=1 notation=\<open>mixfix lazy list enumeration\<close>\<close>\<^bold>\<lbrakk>_\<^bold>\<rbrakk>)\<close>)
 syntax_consts
   LCons
 translations