- May 11, 2020
-
-
Ralf Jung authored
-
- May 08, 2020
-
-
Ralf Jung authored
use new select tactic from std++ See merge request iris/iris!438
-
- May 07, 2020
- May 05, 2020
-
-
Ralf Jung authored
-
- May 01, 2020
-
-
Simon Friis Vindum authored
-
Simon Friis Vindum authored
-
Simon Friis Vindum authored
-
Simon Friis Vindum authored
-
Simon Friis Vindum authored
- Apr 28, 2020
-
-
Paolo G. Giarrusso authored
- Apr 26, 2020
-
- Apr 25, 2020
-
-
Abel Nieto authored
Here's one case this lemma might be useful. Suppose we want to programmatically generate namespaces for e.g. locks: ``` Definition lockN (l : loc) := nroot .@ "lock" .@ l. ``` Then to know that two such namespaces are disjoint, we need to know that the corresponding locations are distinct. For that we use the lemma here introduced. ``` Lemma ne l1 l2 v1 v2 : l1 ↦ v1 -∗ l2 ↦ v2 -∗ ⌜l1 ≠ l2⌝. Proof. iApply mapsto_mapsto_ne. (* goal ¬ ✓ 2%Qp *) by intros []. Qed. ```
-
- Apr 24, 2020
-
-
Robbert Krebbers authored
-
Robbert Krebbers authored
- Apr 23, 2020
-
-
Removes auth_both_op and renames auth_both_frac_op into auth_both_op.
-
Ralf Jung authored
- Apr 22, 2020
-
-
Ralf Jung authored
-
Paolo G. Giarrusso authored
-
- Apr 18, 2020
- Apr 16, 2020
-
- Apr 15, 2020
-
-
Robbert Krebbers authored
This works because there is already a `Reserved Notation`.
-
Robbert Krebbers authored
Fixed a spacing issue in metatheory.v See merge request !427
-
-
Paolo G. Giarrusso authored
Fix #302, including their ASCII variants. - Don't use quotes `'` that are not surrounded by spaces. - However, notation `'(⊢@{' PROP } )` prevents parsing `(⊢@{PROP} Q)` using the `⊢@{PROP} Q` notation. To fix that, we force left-factorization: we add a notation for `'(⊢@{' PROP } Q )`, defined to coincide with '⊢@{' PROP } Q but which can be left-factored with `( '⊢@{' PROP } )`. - Add left and right operator sections for (bi)entailment - Add tests. Also do all of the above also for ASCII notations, except for operator sections, which seem to require more discussion.
-
- Apr 14, 2020
-
-
Ralf Jung authored
-
Paolo G. Giarrusso authored
-
Paolo G. Giarrusso authored
-
Paolo G. Giarrusso authored
-
Paolo G. Giarrusso authored
-