diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Nominal/Examples/Compile.thy --- a/src/HOL/Nominal/Examples/Compile.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Nominal/Examples/Compile.thy Fri Sep 20 19:51:08 2024 +0200 @@ -13,11 +13,11 @@ nominal_datatype ty = Data "data" - | Arrow "ty" "ty" ("_\_" [100,100] 100) + | Arrow "ty" "ty" (\_\_\ [100,100] 100) nominal_datatype trm = Var "name" - | Lam "\name\trm" ("Lam [_]._" [100,100] 100) + | Lam "\name\trm" (\Lam [_]._\ [100,100] 100) | App "trm" "trm" | Const "nat" | Pr "trm" "trm" @@ -26,24 +26,24 @@ | InL "trm" | InR "trm" | Case "trm" "\name\trm" "\name\trm" - ("Case _ of inl _ \ _ | inr _ \ _" [100,100,100,100,100] 100) + (\Case _ of inl _ \ _ | inr _ \ _\ [100,100,100,100,100] 100) nominal_datatype dataI = OneI | NatI nominal_datatype tyI = DataI "dataI" - | ArrowI "tyI" "tyI" ("_\_" [100,100] 100) + | ArrowI "tyI" "tyI" (\_\_\ [100,100] 100) nominal_datatype trmI = IVar "name" - | ILam "\name\trmI" ("ILam [_]._" [100,100] 100) + | ILam "\name\trmI" (\ILam [_]._\ [100,100] 100) | IApp "trmI" "trmI" | IUnit | INat "nat" | ISucc "trmI" - | IAss "trmI" "trmI" ("_\_" [100,100] 100) + | IAss "trmI" "trmI" (\_\_\ [100,100] 100) | IRef "trmI" - | ISeq "trmI" "trmI" ("_;;_" [100,100] 100) + | ISeq "trmI" "trmI" (\_;;_\ [100,100] 100) | Iif "trmI" "trmI" "trmI" text \valid contexts\ @@ -57,7 +57,7 @@ text \typing judgements for trms\ inductive - typing :: "(name\ty) list\trm\ty\bool" (" _ \ _ : _ " [80,80,80] 80) + typing :: "(name\ty) list\trm\ty\bool" (\ _ \ _ : _ \ [80,80,80] 80) where t0[intro]: "\valid \; (x,\)\set \\\ \ \ Var x : \" | t1[intro]: "\\ \ e1 : \1\\2; \ \ e2 : \1\\ \ \ App e1 e2 : \2" @@ -75,7 +75,7 @@ text \typing judgements for Itrms\ inductive - Ityping :: "(name\tyI) list\trmI\tyI\bool" (" _ I\ _ : _ " [80,80,80] 80) + Ityping :: "(name\tyI) list\trmI\tyI\bool" (\ _ I\ _ : _ \ [80,80,80] 80) where t0[intro]: "\valid \; (x,\)\set \\\ \ I\ IVar x : \" | t1[intro]: "\\ I\ e1 : \1\\2; \ I\ e2 : \1\\ \ I\ IApp e1 e2 : \2" @@ -91,7 +91,7 @@ text \capture-avoiding substitution\ class subst = - fixes subst :: "'a \ name \ 'a \ 'a" ("_[_::=_]" [100,100,100] 100) + fixes subst :: "'a \ name \ 'a \ 'a" (\_[_::=_]\ [100,100,100] 100) instantiation trm :: subst begin @@ -169,7 +169,7 @@ text \big-step evaluation for trms\ inductive - big :: "trm\trm\bool" ("_ \ _" [80,80] 80) + big :: "trm\trm\bool" (\_ \ _\ [80,80] 80) where b0[intro]: "Lam [x].e \ Lam [x].e" | b1[intro]: "\e1\Lam [x].e; e2\e2'; e[x::=e2']\e'\ \ App e1 e2 \ e'" @@ -183,7 +183,7 @@ | b9[intro]: "\e\InR e'; e2[x::=e']\e''\ \ Case e of inl x1 \ e1 | inr x2 \ e2 \ e''" inductive - Ibig :: "((nat\nat)\trmI)\((nat\nat)\trmI)\bool" ("_ I\ _" [80,80] 80) + Ibig :: "((nat\nat)\trmI)\((nat\nat)\trmI)\bool" (\_ I\ _\ [80,80] 80) where m0[intro]: "(m,ILam [x].e) I\ (m,ILam [x].e)" | m1[intro]: "\(m,e1)I\(m',ILam [x].e); (m',e2)I\(m'',e3); (m'',e[x::=e3])I\(m''',e4)\