Skip to content
Snippets Groups Projects
counter_examples.v 2.21 KiB
Newer Older
From iris.algebra Require Import upred.
From iris.proofmode Require Import tactics.

(** This proves that we need the ▷ in a "Saved Proposition" construction with
Section savedprop.
  Context (M : ucmraT).
  Notation iProp := (uPred M).
  Notation "¬ P" := ( (P  False))%I : uPred_scope.
  Implicit Types P : iProp.
  (* Saved Propositions and view shifts. *)
  Context (sprop : Type) (saved : sprop  iProp  iProp).
  Hypothesis sprop_persistent :  i P, PersistentP (saved i P).
     (P : sprop  iProp), True =r=> ( i, saved i (P i)).
  Hypothesis sprop_agree :  i P Q, saved i P  saved i Q  P  Q.

  (* Self-contradicting assertions are inconsistent *)
  Lemma no_self_contradiction P `{!PersistentP P} :  (P  ¬ P)  False.
Robbert Krebbers's avatar
Robbert Krebbers committed
  Proof.
    iIntros "#[H1 H2]".
    { iApply "H2". iIntros "! #HP". by iApply ("H1" with "[#]"). }
    by iApply ("H1" with "[#]").
  Qed.

  (* "Assertion with name [i]" is equivalent to any assertion P s.t. [saved i P] *)
  Definition A (i : sprop) : iProp :=  P, saved i P   P.
  Lemma saved_is_A i P `{!PersistentP P} : saved i P   (A i  P).
Robbert Krebbers's avatar
Robbert Krebbers committed
    iIntros "#HS !". iSplit.
    - iDestruct 1 as (Q) "[#HSQ HQ]".
      iApply (sprop_agree i P Q with "[]"); eauto.
    - iIntros "#HP". iExists P. by iSplit.
  Qed.

  (* Define [Q i] to be "negated assertion with name [i]". Show that this
     implies that assertion with name [i] is equivalent to its own negation. *)
  Definition Q i := saved i (¬ A i).
  Lemma Q_self_contradiction i : Q i   (A i  ¬ A i).
  Proof. iIntros "#HQ !". by iApply (saved_is_A i (¬A i)). Qed.

  (* We can obtain such a [Q i]. *)
  Lemma make_Q : True =r=>  i, Q i.
  Proof. apply sprop_alloc_dep. Qed.

  (* Put together all the pieces to derive a contradiction. *)
  Lemma rvs_false : (True : uPred M) =r=> False.
    rewrite make_Q. apply uPred.rvs_mono. iDestruct 1 as (i) "HQ".
    iApply (no_self_contradiction (A i)). by iApply Q_self_contradiction.

  Lemma contradiction : False.
  Proof.
    apply (@uPred.adequacy M False 1); simpl.
    rewrite -uPred.later_intro. apply rvs_false.
  Qed.