请输入您要查询的字词:

 

单词 ExamplesOfPrimitiveRecursivePredicates
释义

examples of primitive recursive predicates


In this entry, we give some examples of primitive recursive predicates. In particular, we will show that the predicateMathworldPlanetmathPlanetmath “x is a prime numberMathworldPlanetmath” is primitive recursive.

In the examples, we use Φ(𝒙) to indicate a predicate (over the natural numbersMathworldPlanetmath ). First, two very simple examples:

  1. 1.

    Φ(x) given by “x=n” for a fixed n is primitive recursive. To see this, note that the set associated with Φ is {n}, and its associated characteristic functionMathworldPlanetmathPlanetmath is primitive recursive by example 3(l) in this entry (http://planetmath.org/ExamplesOfPrimitiveRecursiveFunctions). As a result, Φ is primitive recursive.

  2. 2.

    Φ(x,y) given by “xy” is primitive recursive. The associated set is {(x,y)xy} whose characteristic function is sgn(s(y)-˙x), which is primitive recursive.

Before exhibiting more examples, we prove some basic facts about primitive recursive predicates:

Proposition 1.

If Φ and Θ are primitive recursive predicates, then so are ¬Φ (negationMathworldPlanetmath), ΦΘ (disjunctionMathworldPlanetmath), and ΦΘ (conjunctionMathworldPlanetmath).

Proof.

Let S,T be the sets associated with the predicates Φ and Θ. We may assume that S,Tk for some positive integer k. Let cS and cT be the associated characteristic functions.

First, 1-˙cS is the characteristic function of k-S, which is the associated set of the predicate ¬Φ. Since 1-˙cS is primitive recursive, so is ¬Φ.

Next, mult(CS,CT) is the characteristic function of ST, which is the associated set of the predicate ΦΘ. Since mult(CS,CT) is primitive recursive, so is ΦΘ.

Finally, the set associated with ΦΘ is ST, which is k-((k-S)(k-T)), which is primitive recursive. Hence ΦΘ is primitive recursive as well.∎

In short, primitive recursiveness is preserved under Boolean operations on predicates. By inductionMathworldPlanetmath, we also see primitive recursiveness is preserved under finite disjunction and finite conjunction.

Using this fact, we list three more examples:

  1. 3.

    the predicate “x=y” is primitive recursive, since it is the conjunction of primitive recursive predicates “xy” and “yx”.

  2. 4.

    the predicate “y<x” is primitive recursive, since it is the conjunction “yx” and “¬(x=y)”, both of which are primitive recursive.

  3. 5.

    the predicate “xS”, where S is a fixed finite setMathworldPlanetmath, is primitive recursive, as it is the disjunction of primitive predicates of the form “x=n”, where n ranges over S. Since the disjunction operationMathworldPlanetmath is finitary, “xS” is primitive recursive also.

Here’s another useful fact about primitive recursive predicates:

Proposition 2.

If Φ(x1,,xm) is primitive recursive, so is Θ(x1,,xn), defined by simultaneous substitution of the variables xi in Φ by n-ary primitive recursive functions fi:

Θ(x1,,xn):=Φ(f1(x1,,xn),,fm(x1,,xn)).
Proof.

Let cΦ be the characteristic function of (the set associated with) Φ, then

cΦ(f1(x1,,xn),,fm(x1,,xn))

is cΘ, the characteristic function of Θ. Since cΦ, fi are primitive recursive, cΘ, obtained by functionalMathworldPlanetmathPlanetmathPlanetmathPlanetmath composition, and hence Θ, are primitive recursive too.∎

Let us list two more examples:

  1. 6.

    the predicate “xyz” is primitive recursive.

  2. 7.

    the predicate “y<x!” is primitive recursive.

Finite disjunctions and finite conjunctions of predicates can be thought of as special cases of bounded quantification (http://planetmath.org/BoundedQuantifier) on predicates. In view of this, we have the following facts:

Proposition 3.

If Φ(𝐱,y) is primitive recursive, so are

Θ(𝒙,y):=zyΦ(𝒙,z)  𝑎𝑛𝑑  Ψ(𝒙,y):=zyΦ(𝒙,z).
Proof.

The set associated with Θ(𝒙,y) is {(𝒙,y) for all zy,Φ(𝒙,z)}, which is just

S:={(𝒙,y)Φ(𝒙,0)}{(𝒙,y)Φ(𝒙,1)}{(𝒙,y)Φ(𝒙,y)}

For each fixed i, let Φi(𝒙):=Φ(𝒙,i). Then by propositionPlanetmathPlanetmathPlanetmath 2, Φi is primitive recursive. Let ci be the characteristic function of Φi, and d the function such that d(𝒙,i) is ci(𝒙) if i{0,,n}, and 0 otherwise. So d is primitive recursive (see this entry (http://planetmath.org/ExamplesOfPrimitiveRecursiveFunctions)). Now, define function c by

c(𝒙,y):=i=0yd(𝒙,i).

So 1=d(𝒙,i)=ci(𝒙) iff Φi(𝒙) iff (𝒙,i){(𝒙,i)Φ(𝒙,i)} iff (𝒙,y){(𝒙,y)Φ(𝒙,i)}.

As a result, 1=c(𝒙,y) iff (𝒙,y){(𝒙,y)Φ(𝒙,i)} for all i{0,,y} iff (𝒙,y)S. In other words, c is the characteristic function of S. Since c is obtained from d by bounded product, c is primitive recursive. This shows that Θ is primitive recursive as well.

Next, since the characteristic function of Ψ(𝒙,y) is the same as the characteristic function of ¬zy(¬Φ(𝒙,z)), we conclude that Ψ is primitive recursive by proposition 1 and what we have just proved.∎

Our final example is the following:

  1. 8.

    Φ(x) given by “x is prime” is primitive recursive. One way to characterize Φ is the following: 1<x, and x can not be written as a productPlanetmathPlanetmath of two natural numbers, both greater than 1. In other words,

    Φ(x)(1<x)y(z¬(x=yz1<y1<z)),

    where means “can be characterized by” (they share the same characteristic function). Observe that since x=yz, both y and z are in fact boundedPlanetmathPlanetmath by x. Therefore,

    Φ(x)(1<x)yx(zx¬(x=yz1<y1<z)).

    As each of x=yz,1<y, and 1<z is primitive recursive, so are their conjunction:

    x=yz1<y1<z,

    the negation of which:

    ¬(x=yz1<y1<z),

    two successive applications of bounded universal quantifiersMathworldPlanetmath:

    yx(zx¬(x=yz1<y1<z)),

    and finally its conjunction with the primitive recursive predicate 1<x, which is just Φ(x). Therefore, Φ(x) is primitive recursive.

Remark. The empty setMathworldPlanetmath , corresponding to the predicate “x<x”, is clearly primitive recursive. However, as a function, is not primitive recursive.

随便看

 

数学辞典收录了18232条数学词条,基本涵盖了常用数学知识及数学英语单词词组的翻译及用法,是数学学习的有利工具。

 

Copyright © 2000-2023 Newdu.com.com All Rights Reserved
更新时间:2025/5/24 20:40:57