--- a/Quot/Examples/LamEx.thy Tue Dec 08 16:36:01 2009 +0100
+++ b/Quot/Examples/LamEx.thy Tue Dec 08 17:30:00 2009 +0100
@@ -128,7 +128,7 @@
unfolding fresh_def supp_def
sorry
-lemma perm_rsp[quotient_rsp]:
+lemma perm_rsp[quot_respect]:
"(op = ===> alpha ===> alpha) op \<bullet> op \<bullet>"
apply(auto)
(* this is propably true if some type conditions are imposed ;o) *)
@@ -140,14 +140,14 @@
(* this is probably only true if some type conditions are imposed *)
sorry
-lemma rVar_rsp[quotient_rsp]:
+lemma rVar_rsp[quot_respect]:
"(op = ===> alpha) rVar rVar"
by (auto intro:a1)
-lemma rApp_rsp[quotient_rsp]: "(alpha ===> alpha ===> alpha) rApp rApp"
+lemma rApp_rsp[quot_respect]: "(alpha ===> alpha ===> alpha) rApp rApp"
by (auto intro:a2)
-lemma rLam_rsp[quotient_rsp]: "(op = ===> alpha ===> alpha) rLam rLam"
+lemma rLam_rsp[quot_respect]: "(op = ===> alpha ===> alpha) rLam rLam"
apply(auto)
apply(rule a3)
apply(rule_tac t="[(x,x)]\<bullet>y" and s="y" in subst)
@@ -160,7 +160,7 @@
apply(simp add: abs_fresh)
done
-lemma rfv_rsp[quotient_rsp]: "(alpha ===> op =) rfv rfv"
+lemma rfv_rsp[quot_respect]: "(alpha ===> op =) rfv rfv"
sorry
lemma rvar_inject: "rVar a \<approx> rVar b = (a = b)"