diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Nominal/Examples/VC_Condition.thy --- a/src/HOL/Nominal/Examples/VC_Condition.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Nominal/Examples/VC_Condition.thy Fri Sep 20 19:51:08 2024 +0200 @@ -16,7 +16,7 @@ nominal_datatype lam = Var "name" | App "lam" "lam" - | Lam "\name\lam" ("Lam [_]._" [100,100] 100) + | Lam "\name\lam" (\Lam [_]._\ [100,100] 100) text \ The inductive relation 'unbind' unbinds the top-most @@ -27,7 +27,7 @@ of the algorithm W.\ inductive - unbind :: "lam \ name list \ lam \ bool" ("_ \ _,_" [60,60,60] 60) + unbind :: "lam \ name list \ lam \ bool" (\_ \ _,_\ [60,60,60] 60) where u_var: "(Var a) \ [],(Var a)" | u_app: "(App t1 t2) \ [],(App t1 t2)" @@ -143,7 +143,7 @@ strips off the top-most binders from lambdas.\ inductive - strip :: "lam \ lam \ bool" ("_ \ _" [60,60] 60) + strip :: "lam \ lam \ bool" (\_ \ _\ [60,60] 60) where s_var: "(Var a) \ (Var a)" | s_app: "(App t1 t2) \ (App t1 t2)"