MathIsimple

Poisson Processes

Master the mathematical foundations of Poisson processes: definitions, properties, and applications to counting processes

Advanced TheoryMathematical RigorPractical Applications
📊Poisson Process Definition

Two Equivalent Characterizations

A Poisson process is a continuous-time counting process that describes the occurrence of rare events. Let N(t)N(t) denote the number of events in the interval (0,t](0, t], with state space I={0,1,2,}I = \{0, 1, 2, \ldots\}.

Definition 1: Based on Increment Probability

  1. Initial condition: N(0)=0N(0) = 0
  2. Independent increments: For any 0=t0<t1<<tn0 = t_0 < t_1 < \cdots < t_n, the increments N(t1)N(t0),,N(tn)N(tn1)N(t_1) - N(t_0), \ldots, N(t_n) - N(t_{n-1}) are independent
  3. Rarity: For any t0t \geq 0, as h0+h \to 0^+:
    • P{N(t+h)N(t)=1}=λh+o(h)P\{N(t+h) - N(t) = 1\} = \lambda h + o(h) (intensity λ>0\lambda > 0)
    • P{N(t+h)N(t)2}=o(h)P\{N(t+h) - N(t) \geq 2\} = o(h) (almost no multiple events)

Definition 2: Based on Increment Distribution

  1. Initial condition: N(0)=0N(0) = 0
  2. Independent increments: Same as Definition 1
  3. Increment distribution: For any t>s0t > s \geq 0,N(t)N(s)Poisson(λ(ts))N(t) - N(s) \sim \text{Poisson}(\lambda(t-s))

Equivalence Proof Sketch

Divide (s,t](s, t] into nn subintervals of length h=(ts)/nh = (t-s)/n. By rarity, each subinterval has approximately λh\lambda h probability of one event. The total increment N(t)N(s)N(t) - N(s) approximately follows B(n,λh)B(n, \lambda h). As nn \to \infty, this converges to Poisson(λ(ts))\text{Poisson}(\lambda(t-s)).

🔍Core Properties

Mean and Variance

E[N(t)]=λt,D[N(t)]=λtE[N(t)] = \lambda t, \quad D[N(t)] = \lambda t

Both the mean and variance grow linearly with time. For intensity λ=2\lambda = 2 events per minute, in 10 minutes we expect 20 events with variance 20.

Covariance and Autocorrelation

Cov[N(s),N(t)]=λmin(s,t)\text{Cov}[N(s), N(t)] = \lambda \min(s, t)
RN(s,t)=λmin(s,t)+λ2stR_N(s, t) = \lambda \min(s, t) + \lambda^2 st

The correlation between two time points depends only on the shorter time interval. For s=3,t=5s = 3, t = 5, correlation = λ×3\lambda \times 3.

Conditional Distribution 1

Given total events N(t)=nN(t) = n, the distribution of events in (0,s](0, s]:

P{N(s)=mN(t)=n}=(nm)(st)m(1st)nmP\{N(s) = m \mid N(t) = n\} = \binom{n}{m}\left(\frac{s}{t}\right)^m\left(1-\frac{s}{t}\right)^{n-m}

This follows a binomial distribution, indicating events are uniformly distributed in time.

📈Key Distributions: Event Timing and Time Intervals

Event Occurrence Times WnW_n

The nn-th event occurs at time WnW_n:

WnΓ(n,λ)W_n \sim \Gamma(n, \lambda)

Properties: E[Wn]=nλE[W_n] = \frac{n}{\lambda}, D[Wn]=nλ2D[W_n] = \frac{n}{\lambda^2}

Application: Find probability that 5th customer arrives within 10 minutes.

Time Intervals TnT_n

Time between consecutive events:

TnExp(λ)T_n \sim \text{Exp}(\lambda)

Properties: Independent and identically distributed, memoryless property

Application: Find probability that time between customers ≤ 2 minutes.

Conditional Uniform Distribution

Given exactly one event in (0,t](0, t], the event time W1W_1 is uniformly distributed:

P{W1sN(t)=1}=st,0stP\{W_1 \leq s \mid N(t) = 1\} = \frac{s}{t}, \quad 0 \leq s \leq t

Meaning: Rare events are uniformly distributed in time intervals.

🔄Synthesis and Decomposition

Synthesis (Superposition)

If {N1(t)}\{N_1(t)\} (intensity λ1\lambda_1) and {N2(t)}\{N_2(t)\} (intensity λ2\lambda_2) are independent Poisson processes, then:

N(t)=N1(t)+N2(t)Poisson(λ1+λ2)N(t) = N_1(t) + N_2(t) \sim \text{Poisson}(\lambda_1 + \lambda_2)

Example: Two service windows with intensities 2 and 3 customers/hour create a combined process with intensity 5 customers/hour.

Decomposition (Thinning)

If {N(t)}\{N(t)\} has intensity λ\lambda, and each event is independently classified as type 1 with probability pp, then:

N1(t)Poisson(λp),N2(t)Poisson(λ(1p))N_1(t) \sim \text{Poisson}(\lambda p), \quad N_2(t) \sim \text{Poisson}(\lambda(1-p))

Example: SMS process with intensity 10/day, 20% spam probability, creates independent spam (2/day) and useful (8/day) processes.

Non-Homogeneous Poisson Processes

Time-Varying Intensity

When the event rate varies with time (e.g., rush hour traffic, business hour phone calls), we use a non-homogeneous Poisson process with intensity function λ(t)\lambda(t).

Key Properties

  • Increment distribution: N(t)N(s)Poisson(Λ(s,t))N(t) - N(s) \sim \text{Poisson}(\Lambda(s,t)), where Λ(s,t)=stλ(u)du\Lambda(s,t) = \int_s^t \lambda(u) du is the cumulative intensity
  • Mean function: E[N(t)]=Λ(0,t)=0tλ(u)duE[N(t)] = \Lambda(0,t) = \int_0^t \lambda(u) du
  • Variance: D[N(t)]=Λ(0,t)D[N(t)] = \Lambda(0,t) (still equal to mean)

Example: Linear Growth

For intensity function λ(t)=2t\lambda(t) = 2t, the increment N(3)N(1)N(3) - N(1)follows Poisson(4)\text{Poisson}(4), since Λ(1,3)=132udu=4\Lambda(1,3) = \int_1^3 2u du = 4.

🎯Typical Applications

Service System Counting

Bank with 2 windows, each with service completion rate λ=3\lambda = 3 customers/hour. Total service completions follow Poisson(6)\text{Poisson}(6). Probability of 10 completions in 1 hour: P{N(1)=10}=61010!e6P\{N(1) = 10\} = \frac{6^{10}}{10!}e^{-6}.

Communication Systems

SMS reception with intensity λ=10\lambda = 10 per day, spam probability p=0.2p = 0.2. Spam messages follow Poisson(2)\text{Poisson}(2) per day. Probability of no spam in a day: P{N1(1)=0}=e2P\{N_1(1) = 0\} = e^{-2}.

Traffic Flow Statistics

Rush hour (7:00-9:00) with intensity function λ(t)=100+50(t7)\lambda(t) = 100 + 50(t-7). Cumulative intensity 7:00-8:00: Λ(7,8)=78(100+50(t7))dt=125\Lambda(7,8) = \int_7^8 (100 + 50(t-7)) dt = 125. Traffic flow N(8)N(7)Poisson(125)N(8) - N(7) \sim \text{Poisson}(125).

Ready to Practice?

Test your understanding with interactive problems and use our specialized calculators