- Jun 12, 2017
-
-
Robbert Krebbers authored
-
- Jun 08, 2017
-
-
Robbert Krebbers authored
-
Robbert Krebbers authored
when using iCombine.
-
- May 12, 2017
-
-
Robbert Krebbers authored
-
- Apr 27, 2017
-
-
Robbert Krebbers authored
-
- Apr 13, 2017
-
-
Robbert Krebbers authored
This enables things like `iSpecialize ("H2" with "H1") in the below: "H1" : P ---------□ "H2" : □ P -∗ Q ---------∗ R
-
- Apr 07, 2017
-
-
Robbert Krebbers authored
For example, when having `H : ▷ P → Q` and `HP : P`, we can now do `iSpecialize ("H" with "HP")`. This is achieved by putting a `FromAssumption` premise in the base instance for `IntoWand`.
-
- Mar 24, 2017
-
-
Robbert Krebbers authored
This commit fixes the issues that refolding of big operators did not work nicely in the proof mode, e.g., given: Goal forall M (P : nat → uPred M) l, ([∗ list] x ∈ 10 :: l, P x) -∗ True. Proof. iIntros (M P l) "[H1 H2]". We got: "H1" : P 10 "H2" : (fix big_opL (M0 : ofeT) (o : M0 → M0 → M0) (H : Monoid o) (A : Type) (f : nat → A → M0) (xs : list A) {struct xs} : M0 := match xs with | [] => monoid_unit | x :: xs0 => o (f 0 x) (big_opL M0 o H A (λ n : nat, f (S n)) xs0) end) (uPredC M) uPred_sep uPred.uPred_sep_monoid nat (λ _ x : nat, P x) l --------------------------------------∗ True The problem here is that proof mode looked for an instance of `IntoAnd` for `[∗ list] x ∈ 10 :: l, P x` and then applies the instance for separating conjunction without folding back the fixpoint. This problem is not specific to the Iris proof mode, but more of a general problem of Coq's `apply`, for example: Goal forall x l, Forall (fun _ => True) (map S (x :: l)). Proof. intros x l. constructor. Gives: Forall (λ _ : nat, True) ((fix map (l0 : list nat) : list nat := match l0 with | [] => [] | a :: t => S a :: map t end) l) This commit fixes this issue by making the big operators type class opaque and instead handle them solely via corresponding type classes instances for the proof mode tactics. Furthermore, note that we already had instances for persistence and timelessness. Those were really needed; computation did not help to establish persistence when the list in question was not a ground term. In fact, the sitation was worse, to establish persistence of `[∗ list] x ∈ 10 :: l, P x` it could either use the persistence instance of big ops directly, or use the persistency instance for `∗` first. Worst case, this can lead to an exponential blow up because of back tracking.
-
Robbert Krebbers authored
-
Robbert Krebbers authored
Big ops over list with a cons reduce, hence these just follow immediately from conversion.
-
Robbert Krebbers authored
-
- Mar 21, 2017
-
-
Robbert Krebbers authored
This way, iSplit will work when one side is persistent.
-
Robbert Krebbers authored
-
Robbert Krebbers authored
This could lead to awkward loops, for example, when having: - As goal `own γ c` with `c` persistent, one could keep on `iSplit`ting the goal. Especially in (semi-)automated proof scripts this is annoying as it easily leads to loops. - When having a hypothesis `own γ c` with `c` persistent, one could keep on `iDestruct`ing it. To that end, this commit removes the `IntoOp` and `FromOp` instances for persistent CMRA elements. Instead, we changed the instances for pairs, so that one, for example, can still split `(a ⋅ b, c)` with `c` persistent.
-
- Mar 20, 2017
-
-
Robbert Krebbers authored
-
- Mar 16, 2017
-
-
Robbert Krebbers authored
-
- Mar 15, 2017
-
-
Robbert Krebbers authored
The instances frame_big_sepL_cons and frame_big_sepL_app could be applied repeatedly often when framing in [∗ list] k ↦ x ∈ ?e, Φ k x when ?e an evar. This commit fixes this bug.
-
Robbert Krebbers authored
- Allow framing of persistent hypotheses below the always modality. - Allow framing of persistent hypotheses in just one branch of a disjunction.
-
Robbert Krebbers authored
-
Robbert Krebbers authored
-
- Mar 11, 2017
-
-
Robbert Krebbers authored
-
- Mar 09, 2017
-
-
Robbert Krebbers authored
Also, make the setup of IntoLaterN more consistent with that of WandWeaken. Maybe, we should do something similar for other proof mode classes too.
-
- Feb 22, 2017
-
-
Robbert Krebbers authored
There is no need to restrict the type class using Hint Mode, we have a default instance that will always be used first. In case of evars, the default instance should apply. The reason for this change is that `iAssumption` should be able to prove `H : ?e |- P` and `H : P |- ?e`. The former Hint Mode prevented it from doing that.
-
- Feb 15, 2017
- Feb 13, 2017
-
-
Robbert Krebbers authored
-
- Feb 11, 2017
-
-
Robbert Krebbers authored
Instead of doing all the instantiations by invoking a single type class search, it now performs the instantiations by invoking individual type class searches. This a.) gives better error messages and b.) works when `xj` depends on `xi`.
-
- Feb 06, 2017
-
-
Ralf Jung authored
-
- Jan 26, 2017
-
-
Robbert Krebbers authored
TODO: document the setup of the IntoWand and WandWeaken type classes and the tricks using Hint Mode.
-
- Jan 24, 2017
-
-
Robbert Krebbers authored
-
- Jan 23, 2017
-
-
Robbert Krebbers authored
-
- Jan 22, 2017
-
-
Robbert Krebbers authored
This fixes issue #62.
-
- Jan 05, 2017
-
-
Ralf Jung authored
-
- Jan 03, 2017
-
-
Ralf Jung authored
This patch was created using find -name *.v | xargs -L 1 awk -i inplace '{from = 0} /^From/{ from = 1; ever_from = 1} { if (from == 0 && seen == 0 && ever_from == 1) { print "Set Default Proof Using \"Type*\"."; seen = 1 } }1 ' and some minor manual editing
-
- Dec 28, 2016
-
-
Robbert Krebbers authored
This fixes issue #55.
-
- Dec 14, 2016
-
-
Ralf Jung authored
-
- Dec 09, 2016
-
-
Ralf Jung authored
-