src/HOL/Lambda/Eta.thy
changeset 22422 ee19cdb07528
parent 22272 aac2ac7c32fd
child 23750 a1db5f819d00
--- a/src/HOL/Lambda/Eta.thy	Tue Mar 06 16:40:32 2007 +0100
+++ b/src/HOL/Lambda/Eta.thy	Fri Mar 09 08:45:50 2007 +0100
@@ -163,7 +163,7 @@
     iff del: dB.distinct simp: dB.distinct)    (*23 seconds?*)
   done
 
-lemma confluent_beta_eta: "confluent (join beta eta)"
+lemma confluent_beta_eta: "confluent (sup beta eta)"
   apply (assumption |
     rule square_rtrancl_reflcl_commute confluent_Un
       beta_confluent eta_confluent square_beta_eta)+
@@ -366,7 +366,7 @@
 qed
 
 theorem eta_postponement:
-  assumes st: "(join beta eta)\<^sup>*\<^sup>* s t"
+  assumes st: "(sup beta eta)\<^sup>*\<^sup>* s t"
   shows "(eta\<^sup>*\<^sup>* OO beta\<^sup>*\<^sup>*) s t" using st
 proof induct
   case 1