Skip to content
Snippets Groups Projects
Commit bde48e82 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Merge branch 'ralf/löb' into 'master'

prove a funny consequence of Löb induction

See merge request !538
parents 206d8842 9a6976e2
No related branches found
No related tags found
No related merge requests found
......@@ -165,6 +165,12 @@ Proof.
by rewrite -later_and impl_elim_r (comm _ R) wand_elim_r.
Qed.
(** A funny consequence of Löb induction.
This shows that Löb induction is incompatible with classical logic.
See [lib/counterexamples.v] for a fully worked-out proof of that fact. *)
Lemma not_not_later_False `{!BiLöb PROP} : ⊢@{PROP} ¬ ¬ False.
Proof. apply entails_impl, löb. Qed.
(* Iterated later modality *)
Global Instance laterN_ne m : NonExpansive (@bi_laterN PROP m).
Proof. induction m; simpl. by intros ???. solve_proper. Qed.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment