src/HOL/Nominal/Examples/CR.thy
changeset 18269 3f36e2165e51
parent 18106 836135c8acb2
child 18303 b18fabea0fd0
--- a/src/HOL/Nominal/Examples/CR.thy	Mon Nov 28 00:25:43 2005 +0100
+++ b/src/HOL/Nominal/Examples/CR.thy	Mon Nov 28 05:03:00 2005 +0100
@@ -1,8 +1,11 @@
+(* $Id$ *)
 
 theory cr
 imports lam_substs
 begin
 
+text {* The Church-Rosser proof from Barendregt's book *}
+
 lemma forget[rule_format]: 
   shows "a\<sharp>t1 \<longrightarrow> t1[a::=t2] = t1"
 proof (nominal_induct t1 rule: lam_induct)