Quot/Nominal/LamEx2.thy
changeset 1139 c4001cda9da3
parent 1129 9a86f0ef6503
child 1210 10a0e3578507
--- a/Quot/Nominal/LamEx2.thy	Fri Feb 12 15:50:43 2010 +0100
+++ b/Quot/Nominal/LamEx2.thy	Fri Feb 12 16:04:10 2010 +0100
@@ -175,22 +175,22 @@
 
 quotient_definition
   "Var :: name \<Rightarrow> lam"
-as
+is
   "rVar"
 
 quotient_definition
    "App :: lam \<Rightarrow> lam \<Rightarrow> lam"
-as
+is
   "rApp"
 
 quotient_definition
   "Lam :: name \<Rightarrow> lam \<Rightarrow> lam"
-as
+is
   "rLam"
 
 quotient_definition
   "fv :: lam \<Rightarrow> atom set"
-as
+is
   "rfv"
 
 lemma perm_rsp[quot_respect]:
@@ -239,7 +239,7 @@
 
 quotient_definition
   "permute_lam :: perm \<Rightarrow> lam \<Rightarrow> lam"
-as
+is
   "permute :: perm \<Rightarrow> rlam \<Rightarrow> rlam"
 
 lemma permute_lam [simp]: