src/HOL/Library/Nat_Int_Bij.thy
changeset 30663 0b6aff7451b2
parent 29888 ab97183f1694
child 32338 e73eb2db4727
equal deleted inserted replaced
30662:396be15b95d5 30663:0b6aff7451b2
     1 (*  Title:      HOL/Nat_Int_Bij.thy
     1 (*  Title:      HOL/Nat_Int_Bij.thy
     2     ID:         $Id$
       
     3     Author:     Stefan Richter, Tobias Nipkow
     2     Author:     Stefan Richter, Tobias Nipkow
     4 *)
     3 *)
     5 
     4 
     6 header{* Bijections $\mathbb{N}\to\mathbb{N}^2$ and $\mathbb{N}\to\mathbb{Z}$*}
     5 header{* Bijections $\mathbb{N}\to\mathbb{N}^2$ and $\mathbb{N}\to\mathbb{Z}$*}
     7 
     6 
     8 theory Nat_Int_Bij
     7 theory Nat_Int_Bij
     9 imports Hilbert_Choice Presburger
     8 imports Main
    10 begin
     9 begin
    11 
    10 
    12 subsection{*  A bijection between @{text "\<nat>"} and @{text "\<nat>\<twosuperior>"} *}
    11 subsection{*  A bijection between @{text "\<nat>"} and @{text "\<nat>\<twosuperior>"} *}
    13 
    12 
    14 text{* Definition and proofs are from \cite[page 85]{Oberschelp:1993}. *}
    13 text{* Definition and proofs are from \cite[page 85]{Oberschelp:1993}. *}