src/HOL/Library/Numeral_Type.thy
changeset 29025 8c8859c0d734
parent 28920 4ed4b8b1988d
child 29629 5111ce425e7a
--- a/src/HOL/Library/Numeral_Type.thy	Tue Dec 09 12:53:25 2008 -0800
+++ b/src/HOL/Library/Numeral_Type.thy	Tue Dec 09 15:31:38 2008 -0800
@@ -14,23 +14,6 @@
 subsection {* Preliminary lemmas *}
 (* These should be moved elsewhere *)
 
-lemma inj_Inl [simp]: "inj_on Inl A"
-  by (rule inj_onI, simp)
-
-lemma inj_Inr [simp]: "inj_on Inr A"
-  by (rule inj_onI, simp)
-
-lemma inj_Some [simp]: "inj_on Some A"
-  by (rule inj_onI, simp)
-
-lemma card_Plus:
-  "[| finite A; finite B |] ==> card (A <+> B) = card A + card B"
-  unfolding Plus_def
-  apply (subgoal_tac "Inl ` A \<inter> Inr ` B = {}")
-  apply (simp add: card_Un_disjoint card_image)
-  apply fast
-  done
-
 lemma (in type_definition) univ:
   "UNIV = Abs ` A"
 proof