src/HOL/Hyperreal/NatStar.thy
changeset 21404 eb85850d3eb7
parent 20740 5a103b43da5a
child 21847 59a68ed9f2f2
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
   184 
   184 
   185 
   185 
   186 subsection{*Nonstandard Characterization of Induction*}
   186 subsection{*Nonstandard Characterization of Induction*}
   187 
   187 
   188 definition
   188 definition
   189   hSuc :: "hypnat => hypnat"
   189   hSuc :: "hypnat => hypnat" where
   190   "hSuc n = n + 1"
   190   "hSuc n = n + 1"
   191 
   191 
   192 lemma starP: "(( *p* P) (star_n X)) = ({n. P (X n)} \<in> FreeUltrafilterNat)"
   192 lemma starP: "(( *p* P) (star_n X)) = ({n. P (X n)} \<in> FreeUltrafilterNat)"
   193 by (rule starP_star_n)
   193 by (rule starP_star_n)
   194 
   194