changeset 22501 | cb41c397a699 |
parent 22494 | b61306c7987a |
child 22531 | 1cbfb4066e47 |
--- a/src/HOL/Nominal/Examples/Crary.thy Thu Mar 22 14:26:05 2007 +0100 +++ b/src/HOL/Nominal/Examples/Crary.thy Thu Mar 22 16:34:03 2007 +0100 @@ -64,7 +64,7 @@ lookup :: "Subst \<Rightarrow> name \<Rightarrow> trm" where "lookup [] x = Var x" - "lookup ((y,T)#\<theta>) x = (if x=y then T else lookup \<theta> x)" +| "lookup ((y,T)#\<theta>) x = (if x=y then T else lookup \<theta> x)" lemma lookup_eqvt[eqvt]: fixes pi::"name prm"