author | paulson |
Thu, 01 Oct 2009 16:43:19 +0100 | |
changeset 32823 | b13e04329012 |
parent 32821 | 99843bbfaeb2 (current diff) |
parent 32822 | 45fa9254ddc8 (diff) |
child 32826 | f7f94bb9ac94 |
child 32851 | d6956d589f96 |
--- a/src/HOL/Library/Nat_Int_Bij.thy Thu Oct 01 15:54:55 2009 +0200 +++ b/src/HOL/Library/Nat_Int_Bij.thy Thu Oct 01 16:43:19 2009 +0100 @@ -128,6 +128,9 @@ thus "\<forall>y. \<exists>x. y = nat2_to_nat x" by fast qed +lemma nat_to_nat2_inj: "inj nat_to_nat2" + by (simp add: nat_to_nat2_def surj_imp_inj_inv nat2_to_nat_surj) + subsection{* A bijection between @{text "\<nat>"} and @{text "\<int>"} *}