fixed function syntax
authorkrauss
Thu, 22 Mar 2007 16:53:37 +0100
changeset 22502 baee64dbe8ea
parent 22501 cb41c397a699
child 22503 d53664118418
fixed function syntax
src/HOL/Nominal/Examples/SOS.thy
--- a/src/HOL/Nominal/Examples/SOS.thy	Thu Mar 22 16:34:03 2007 +0100
+++ b/src/HOL/Nominal/Examples/SOS.thy	Thu Mar 22 16:53:37 2007 +0100
@@ -66,7 +66,7 @@
   lookup :: "(name\<times>trm) list \<Rightarrow> name \<Rightarrow> trm"   
 where
   "lookup [] x        = Var x"
-  "lookup ((y,e)#\<theta>) x = (if x=y then e else lookup \<theta> x)"
+| "lookup ((y,e)#\<theta>) x = (if x=y then e else lookup \<theta> x)"
 
 lemma lookup_eqvt:
   fixes pi::"name prm"