src/HOL/Nominal/Examples/Fsub.thy
changeset 80935 b5bdcdbf5ec1
parent 80914 d97fdabd9e2b
child 81125 ec121999a9cb
--- a/src/HOL/Nominal/Examples/Fsub.thy	Mon Sep 23 21:09:23 2024 +0200
+++ b/src/HOL/Nominal/Examples/Fsub.thy	Mon Sep 23 22:33:37 2024 +0200
@@ -17,7 +17,7 @@
 section \<open>Types for Names, Nominal Datatype Declaration for Types and Terms\<close>
 
 no_syntax
-  "_Map" :: "maplets => 'a \<rightharpoonup> 'b"  (\<open>(1[_])\<close>)
+  "_Map" :: "maplets => 'a \<rightharpoonup> 'b"  (\<open>(\<open>indent=1 notation=\<open>mixfix maplets\<close>\<close>[_])\<close>)
 
 text \<open>The main point of this solution is to use names everywhere (be they bound, 
   binding or free). In System \FSUB{} there are two kinds of names corresponding to