slightly tuned
authorurbanc
Thu, 19 Jun 2008 15:47:26 +0200
changeset 27272 75b251e9cdb7
parent 27271 ba2a00d35df1
child 27273 d54ae0bdad80
slightly tuned
src/HOL/Nominal/Examples/SN.thy
--- a/src/HOL/Nominal/Examples/SN.thy	Thu Jun 19 11:46:14 2008 +0200
+++ b/src/HOL/Nominal/Examples/SN.thy	Thu Jun 19 15:47:26 2008 +0200
@@ -180,12 +180,6 @@
 where
   SN_intro: "(\<And>t'. t \<longrightarrow>\<^isub>\<beta> t' \<Longrightarrow> SN t') \<Longrightarrow> SN t"
 
-lemma SN_elim:
-  assumes a: "SN M"
-  shows "(\<forall>M. (\<forall>N. M \<longrightarrow>\<^isub>\<beta> N \<longrightarrow> P N)\<longrightarrow> P M) \<longrightarrow> P M"
-using a
-by (induct rule: SN.SN.induct) (blast)
-
 lemma SN_preserved: 
   assumes a: "SN t1" "t1\<longrightarrow>\<^isub>\<beta> t2"
   shows "SN t2"