Skip to content
Snippets Groups Projects
Commit 8bfac1ad authored by Ralf Jung's avatar Ralf Jung
Browse files

Merge branch 'master' of gitlab.mpi-sws.org:FP/iris-coq

parents 6c6f5755 126d54c3
No related branches found
No related tags found
No related merge requests found
......@@ -3,7 +3,7 @@ From iris.heap_lang Require Export lang.
From iris.algebra Require Import excl agree csum.
From iris.heap_lang.lib.barrier Require Import proof specification.
From iris.heap_lang Require Import notation par proofmode.
From iris.proofmode Require Import invariants.
From iris.proofmode Require Import tactics.
Definition one_shotR (Σ : gFunctors) (F : cFunctor) :=
csumR (exclR unitC) (agreeR $ laterC $ F (iPreProp Σ)).
......
......@@ -2,7 +2,7 @@ From iris.program_logic Require Export weakestpre hoare.
From iris.heap_lang Require Export lang.
From iris.algebra Require Import excl dec_agree csum.
From iris.heap_lang Require Import assert proofmode notation.
From iris.proofmode Require Import invariants.
From iris.proofmode Require Import tactics.
Definition one_shot_example : val := λ: <>,
let: "x" := ref NONE in (
......
From iris.proofmode Require Import tactics.
From iris.proofmode Require Import pviewshifts invariants.
From iris.program_logic Require Import invariants.
Lemma demo_0 {M : ucmraT} (P Q : uPred M) :
(P Q) ( x, x = 0 x = 1) (Q P).
......
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