Skip to content
Snippets Groups Projects
Commit d9cad5bf authored by Janno's avatar Janno
Browse files

Add IntoPure instances for ∗, ∧, and ∨.

parent 84d78426
No related branches found
No related tags found
No related merge requests found
...@@ -55,6 +55,15 @@ Global Instance into_pure_forall {X : Type} (Φ : X → uPred M) φ : ...@@ -55,6 +55,15 @@ Global Instance into_pure_forall {X : Type} (Φ : X → uPred M) φ :
Proof. Proof.
rewrite /IntoPure=>Hx. rewrite -pure_forall_2. by setoid_rewrite Hx. rewrite /IntoPure=>Hx. rewrite -pure_forall_2. by setoid_rewrite Hx.
Qed. Qed.
Global Instance into_pure_pure_conj (φ1 φ2 : uPred M) P1 P2 :
IntoPure φ1 P1 -> IntoPure φ2 P2 -> IntoPure (φ1 φ2) (P1 P2).
Proof. rewrite /IntoPure pure_and. by intros -> ->. Qed.
Global Instance into_pure_pure_sep (φ1 φ2 : uPred M) P1 P2 :
IntoPure φ1 P1 -> IntoPure φ2 P2 -> IntoPure (φ1 φ2) (P1 P2).
Proof. rewrite /IntoPure sep_and pure_and. by intros -> ->. Qed.
Global Instance into_pure_pure_disj (φ1 φ2 : uPred M) P1 P2 :
IntoPure φ1 P1 -> IntoPure φ2 P2 -> IntoPure (φ1 φ2) (P1 P2).
Proof. rewrite /IntoPure pure_or. by intros -> ->. Qed.
(* FromPure *) (* FromPure *)
Global Instance from_pure_pure φ : @FromPure M φ φ. Global Instance from_pure_pure φ : @FromPure M φ φ.
......
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