Skip to content
Snippets Groups Projects
Forked from Iris / Iris
5571 commits behind the upstream repository.
deprecated.v 498 B
From iris.base_logic Require Import primitive.

(* Deprecated 2016-11-22. Use ⌜φ⌝ instead. *)
Notation "■ φ" := (uPred_pure φ%C%type)
    (at level 20, right associativity, only parsing) : uPred_scope.

(* Deprecated 2016-11-22. Use ⌜x = y⌝ instead. *)
Notation "x = y" := (uPred_pure (x%C%type = y%C%type)) (only parsing) : uPred_scope.

(* Deprecated 2016-11-22. Use ⌜x ⊥ y ⌝ instead. *)
Notation "x ⊥ y" := (uPred_pure (x%C%type ⊥ y%C%type)) (only parsing) : uPred_scope.