src/HOL/Induct/LList.thy
changeset 15413 901d1bfedf09
parent 13585 db4005b40cc6
child 15481 fc075ae929e4
--- a/src/HOL/Induct/LList.thy	Wed Dec 15 10:19:19 2004 +0100
+++ b/src/HOL/Induct/LList.thy	Wed Dec 15 17:32:40 2004 +0100
@@ -443,12 +443,6 @@
 
 subsection{* Isomorphisms *}
 
-lemma inj_Rep_LList: "inj Rep_LList"
-apply (rule inj_on_inverseI)
-apply (rule Rep_LList_inverse)
-done
-
-
 lemma LListI: "x \<in> llist (range Leaf) ==> x \<in> LList"
 by (unfold LList_def, simp)