diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Nominal/Examples/Weakening.thy --- a/src/HOL/Nominal/Examples/Weakening.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Nominal/Examples/Weakening.thy Fri Sep 20 19:51:08 2024 +0200 @@ -14,11 +14,11 @@ nominal_datatype lam = Var "name" | App "lam" "lam" - | Lam "\name\lam" ("Lam [_]._" [100,100] 100) + | Lam "\name\lam" (\Lam [_]._\ [100,100] 100) nominal_datatype ty = TVar "string" - | TArr "ty" "ty" ("_ \ _" [100,100] 100) + | TArr "ty" "ty" (\_ \ _\ [100,100] 100) lemma ty_fresh: fixes x::"name" @@ -42,7 +42,7 @@ text\Typing judgements\ inductive - typing :: "(name\ty) list\lam\ty\bool" ("_ \ _ : _" [60,60,60] 60) + typing :: "(name\ty) list\lam\ty\bool" (\_ \ _ : _\ [60,60,60] 60) where t_Var[intro]: "\valid \; (x,T)\set \\ \ \ \ Var x : T" | t_App[intro]: "\\ \ t1 : T1\T2; \ \ t2 : T1\ \ \ \ App t1 t2 : T2" @@ -60,7 +60,7 @@ text \Abbreviation for the notion of subcontexts.\ abbreviation - "sub_context" :: "(name\ty) list \ (name\ty) list \ bool" ("_ \ _" [60,60] 60) + "sub_context" :: "(name\ty) list \ (name\ty) list \ bool" (\_ \ _\ [60,60] 60) where "\1 \ \2 \ \x T. (x,T)\set \1 \ (x,T)\set \2"