Library prosa.util.unit_growth
From mathcomp Require Import ssreflect ssrbool eqtype ssrnat.
Require Import prosa.util.tactics prosa.util.notation.
Require Import prosa.util.tactics prosa.util.notation.
We say that a function f is a unit growth function iff for any
time instant t it holds that f (t + 1) ≤ f t + 1.
In this section, we prove a few useful lemmas about unit growth functions.
Let f be any unit growth function over natural numbers.
In the following section, we prove a result similar to the
intermediate value theorem for continuous functions.
Lemma exists_intermediate_point :
∃ x_mid, x1 ≤ x_mid < x2 ∧ f x_mid = y.
End ExistsIntermediateValue.
∃ x_mid, x1 ≤ x_mid < x2 ∧ f x_mid = y.
End ExistsIntermediateValue.
In this section, we, again, prove an analogue of the
intermediate value theorem, but for predicates over natural
numbers.
Let P be any predicate on natural numbers.
Consider a time interval
[t1,t2]
such that ...
... but holds for t2.