src/HOL/Nominal/Examples/SN.thy
changeset 18269 3f36e2165e51
parent 18263 7f75925498da
child 18313 e61d2424863d
--- a/src/HOL/Nominal/Examples/SN.thy	Mon Nov 28 00:25:43 2005 +0100
+++ b/src/HOL/Nominal/Examples/SN.thy	Mon Nov 28 05:03:00 2005 +0100
@@ -1,10 +1,12 @@
 (* $Id$ *)
 
+
+
 theory sn
 imports lam_substs  Accessible_Part
 begin
 
-(* Strong normalisation according to the P&T book by Girard et al *)
+text {* Strong Normalisation proof from the Proofs and Types book *}
 
 section {* Beta Reduction *}