Skip to content
Snippets Groups Projects
  1. Nov 13, 2017
    • Robbert Krebbers's avatar
    • Robbert Krebbers's avatar
      Improved treatment of anonymous hypotheses in the proof mode. · bb3584e7
      Robbert Krebbers authored
      The proof mode now explicitly keeps track of anonymous hypotheses (i.e.
      hypotheses that are introduced by the introduction pattern `?`). Consider:
      
        Lemma foo {M} (P Q R : uPred M) : P -∗ (Q ∗ R) -∗ Q ∗ P.
        Proof. iIntros "? [H ?]". iFrame "H". iFrame. Qed.
      
      After the `iIntros`, the goal will be:
      
        _ : P
        "H" : Q
        _ : R
        --------------------------------------∗
        Q ∗ P
      
      Anonymous hypotheses are displayed in a special way (`_ : P`). An important
      property of the new anonymous hypotheses is that it is no longer possible to
      refer to them by name, whereas before, anonymous hypotheses were given some
      arbitrary fresh name (typically prefixed by `~`).
      
      Note tactics can still operate on these anonymous hypotheses. For example, both
      `iFrame` and `iAssumption`, as well as the symbolic execution tactics, will
      use them. The only thing that is not possible is to refer to them yourself,
      for example, in an introduction, specialization or selection pattern.
      
      Advantages of the new approach:
      
      - Proofs become more robust as one cannot accidentally refer to anonymous
        hypotheses by their fresh name.
      - Fresh name generation becomes considerably easier. Since anonymous hypotheses
        are internally represented by natural numbers (of type `N`), we can just fold
        over the hypotheses and take the max plus one. This thus solve issue #101.
      bb3584e7
  2. Nov 11, 2017
  3. Nov 01, 2017
    • Robbert Krebbers's avatar
      Hide the proof mode entailment behind a definition. · 8574d1ea
      Robbert Krebbers authored
      This solves issue #100: the proof mode notation is sometimes not printed. As
      Ralf discovered, the problem is that there are two overlapping notations:
      
      ```coq
      Notation "P ⊢ Q" := (uPred_entails P Q).
      ```
      
      And the "proof mode" notation:
      
      ```
      Notation "Γ '--------------------------------------' □ Δ '--------------------------------------' ∗ Q" :=
        (of_envs (Envs Γ Δ) ⊢ Q%I).
      ```
      
      These two notations overlap, so, when having a "proof mode" goal of the shape
      `of_envs (Envs Γ Δ) ⊢ Q%I`, how do we know which notation is Coq going to pick
      for pretty printing this goal? As we have seen, this choice depends on the
      import order (since both notations appear in different files), and as such, Coq
      sometimes (unintendedly) uses the first notation instead of the latter.
      
      The idea of this commit is to wrap `of_envs (Envs Γ Δ) ⊢ Q%I` into a definition
      so that there is no ambiguity for the pretty printer anymore.
      8574d1ea
  4. Oct 29, 2017
  5. Oct 28, 2017
  6. Oct 26, 2017
  7. Oct 25, 2017
  8. Sep 27, 2017
    • Robbert Krebbers's avatar
      Fix issue #99. · 7ed067a9
      Robbert Krebbers authored
      This causes a bit of backwards incompatibility: it may now succeed with
      later stripping below unlocked/TC transparent definitions. This problem
      actually occured for `wsat`.
      7ed067a9
  9. Sep 26, 2017
    • Robbert Krebbers's avatar
      Fix issue #98. · e17ac4ad
      Robbert Krebbers authored
      We used to normalize the goal, and then checked whether it was of
      a certain shape. Since `uPred_valid P` normalized to `True ⊢ P`,
      there was no way of making a distinction between the two, hence
      `True ⊢ P` was treated as `uPred_valid P`.
      
      In this commit, I use type classes to check whether the goal is of
      a certain shape. Since we declared `uPred_valid` as `Typeclasses
      Opaque`, we can now make a distinction between `True ⊢ P` and
      `uPred_valid P`.
      e17ac4ad
  10. Sep 21, 2017
  11. Sep 17, 2017
  12. Aug 20, 2017
  13. Aug 17, 2017
  14. Aug 07, 2017
  15. Jun 27, 2017
  16. Jun 12, 2017
  17. Jun 08, 2017
  18. May 12, 2017
  19. Apr 13, 2017
  20. Apr 11, 2017
  21. Apr 07, 2017
  22. Mar 27, 2017
  23. Mar 24, 2017
    • Robbert Krebbers's avatar
    • Robbert Krebbers's avatar
      Generic big operators that are no longer tied to CMRAs. · 6fbff46e
      Robbert Krebbers authored
      Instead, I have introduced a type class `Monoid` that is used by the big operators:
      
          Class Monoid {M : ofeT} (o : M → M → M) := {
            monoid_unit : M;
            monoid_ne : NonExpansive2 o;
            monoid_assoc : Assoc (≡) o;
            monoid_comm : Comm (≡) o;
            monoid_left_id : LeftId (≡) monoid_unit o;
            monoid_right_id : RightId (≡) monoid_unit o;
          }.
      
      Note that the operation is an argument because we want to have multiple monoids over
      the same type (for example, on `uPred`s we have monoids for `∗`, `∧`, and `∨`). However,
      we do bundle the unit because:
      
      - If we would not, the unit would appear explicitly in an implicit argument of the
        big operators, which confuses rewrite. By bundling the unit in the `Monoid` class
        it is hidden, and hence rewrite won't even see it.
      - The unit is unique.
      
      We could in principle have big ops over setoids instead of OFEs. However, since we do
      not have a canonical structure for bundled setoids, I did not go that way.
      6fbff46e
  24. Mar 22, 2017
  25. Mar 21, 2017
Loading