Skip to content
GitLab
Menu
Projects
Groups
Snippets
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Menu
Open sidebar
George Pirlea
Iris
Commits
186ffb07
Commit
186ffb07
authored
Feb 21, 2018
by
Ralf Jung
Browse files
a BI is affine iff True |- emp
parent
47250f79
Changes
1
Hide whitespace changes
Inline
Side-by-side
theories/bi/derived_laws.v
View file @
186ffb07
...
...
@@ -673,6 +673,15 @@ Proof. apply (anti_symm _); auto using True_sep_2. Qed.
Lemma
sep_True
P
`
{!
Absorbing
P
}
:
P
∗
True
⊣
⊢
P
.
Proof
.
by
rewrite
comm
True_sep
.
Qed
.
Lemma
True_emp_iff_BiAffine
:
BiAffine
PROP
↔
(
True
⊢
emp
).
Proof
.
split
.
-
intros
?.
exact
:
affine
.
-
rewrite
/
BiAffine
/
Affine
=>
Hemp
?.
rewrite
-
Hemp
.
exact
:
True_intro
.
Qed
.
Section
bi_affine
.
Context
`
{
BiAffine
PROP
}.
...
...
Write
Preview
Supports
Markdown
0%
Try again
or
attach a new file
.
Attach a file
Cancel
You are about to add
0
people
to the discussion. Proceed with caution.
Finish editing this message first!
Cancel
Please
register
or
sign in
to comment