Markov’s principle

Content created by Fredrik Bakke.

Created on 2025-01-07.
Last modified on 2025-01-07.

module logic.markovs-principle where
Imports
open import elementary-number-theory.natural-numbers

open import foundation.booleans
open import foundation.decidable-subtypes
open import foundation.dependent-pair-types
open import foundation.disjunction
open import foundation.existential-quantification
open import foundation.function-types
open import foundation.inhabited-types
open import foundation.negation
open import foundation.universal-quantification
open import foundation.universe-levels

open import foundation-core.identity-types
open import foundation-core.propositions
open import foundation-core.sets

open import logic.markovian-types

open import univalent-combinatorics.standard-finite-types

Idea

Markov’s principle asserts that if a decidable subtype 𝒫 of the natural numbers is not full, then there is a natural number n that is not in 𝒫.

Markov’s principle is an example of a constructive taboo. It is a consequence of the law of excluded middle that is not provable generally in constructive mathematics.

Definitions

Markov’s principle

Markov's-Principle : UU lzero
Markov's-Principle = is-markovian 

Properties

Markov’s principle is constructively valid for ascending chains of decidable propositions

Proof. Assume given an ascending chain of decidable propositions Pᵢ ⇒ Pᵢ₊₁ indexed by the natural numbers . This gives a decidable subtype 𝒫 of given by i ∈ 𝒫 iff Pᵢ is true. Observe that if i ∈ 𝒫 then every j ≥ i is also in 𝒫, and there must exist a least such i ∈ 𝒫. Therefore, 𝒫 = Σ (m ∈ ℕ) (m ≥ k) for some k. So, if ¬ (∀ᵢ Pᵢ) it is necessarily the case that ¬ P₀.

markovs-principle-ascending-chains :
  {l : Level} (P :   UU l)
  (H : (n : )  P n  P (succ-ℕ n))  ¬ ((n : )  P n)  Σ  (¬_  P)
markovs-principle-ascending-chains P H q = (0 , λ x  q (ind-ℕ x H))

See also

Recent changes