Skip to content
Snippets Groups Projects
Commit ae69f50b authored by Yusuke Matsushita's avatar Yusuke Matsushita
Browse files

fix typos

parent 524fbf52
No related branches found
No related tags found
No related merge requests found
...@@ -91,7 +91,7 @@ borrows" in the Coq development. ...@@ -91,7 +91,7 @@ borrows" in the Coq development.
| F-endlft | programs.v | type_endlft | | F-endlft | programs.v | type_endlft |
| F-call | function.v | type_call' | | F-call | function.v | type_call' |
Some of these lemmas are called `something'` because the version without the `'` is a derived, more speicalized form used together with our eauto-based `solve_typing` tactic. You can see this tactic in action in the [examples](theories/typing/examples) subfolder. Some of these lemmas are called `something'` because the version without the `'` is a derived, more specialized form used together with our eauto-based `solve_typing` tactic. You can see this tactic in action in the [examples](theories/typing/examples) subfolder.
### Lifetime Logic Rules ### Lifetime Logic Rules
......
...@@ -16,7 +16,7 @@ Section own. ...@@ -16,7 +16,7 @@ Section own.
end%I. end%I.
Next Obligation. intros _ _ _ sz0 ? n ?. by apply Qcmult_pos_pos. Qed. Next Obligation. intros _ _ _ sz0 ? n ?. by apply Qcmult_pos_pos. Qed.
Arguments freeable_sz : simpl never. Arguments freeable_sz : simpl never.
Global Instance freable_sz_timeless n sz l : Timeless (freeable_sz n sz l). Global Instance freeable_sz_timeless n sz l : Timeless (freeable_sz n sz l).
Proof. destruct sz, n; apply _. Qed. Proof. destruct sz, n; apply _. Qed.
Lemma freeable_sz_full n l : freeable_sz n n l ⊣⊢ {1}ln Z.of_nat n = 0⌝. Lemma freeable_sz_full n l : freeable_sz n n l ⊣⊢ {1}ln Z.of_nat n = 0⌝.
......
...@@ -7,7 +7,7 @@ Set Default Proof Using "Type". ...@@ -7,7 +7,7 @@ Set Default Proof Using "Type".
Section case. Section case.
Context `{!typeG Σ}. Context `{!typeG Σ}.
(* FIXME : have a iris version of Forall2. *) (* FIXME : have an Iris version of Forall2. *)
Lemma type_case_own' E L C T p n tyl el : Lemma type_case_own' E L C T p n tyl el :
Forall2 (λ ty e, Forall2 (λ ty e,
( typed_body E L C ((p + #0 own_ptr n (uninit 1)) :: (p + #1 own_ptr n ty) :: ( typed_body E L C ((p + #0 own_ptr n (uninit 1)) :: (p + #1 own_ptr n ty) ::
......
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