Skip to content
GitLab
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
b0e11cff
Commit
b0e11cff
authored
Aug 17, 2017
by
Robbert Krebbers
Browse files
Bump coq-stdpp.
parent
9c189816
Changes
3
Hide whitespace changes
Inline
Side-by-side
opam.pins
View file @
b0e11cff
coq-stdpp https://gitlab.mpi-sws.org/robbertkrebbers/coq-stdpp
ee6200b4d74bfd06034f3cc36d1afdc309427e5c
coq-stdpp https://gitlab.mpi-sws.org/robbertkrebbers/coq-stdpp
24cc2e4786b2344e092e412f56e96c6971ab60d8
theories/algebra/auth.v
View file @
b0e11cff
...
...
@@ -279,7 +279,8 @@ Proof.
split
;
try
apply
_
.
-
intros
n
[[[
a
|]|]
b
]
;
rewrite
!
auth_validN_eq
;
try
naive_solver
eauto
using
cmra_morphism_monotoneN
,
cmra_morphism_validN
.
-
intros
[??].
apply
Some_proper
.
by
f_equiv
;
rewrite
/=
cmra_morphism_core
.
-
intros
[??].
apply
Some_proper
;
rewrite
/
auth_map
/=.
by
f_equiv
;
rewrite
/=
cmra_morphism_core
.
-
intros
[[?|]?]
[[?|]?]
;
try
apply
Auth_proper
=>//=
;
by
rewrite
cmra_morphism_op
.
Qed
.
Definition
authC_map
{
A
B
}
(
f
:
A
-
n
>
B
)
:
authC
A
-
n
>
authC
B
:
=
...
...
theories/algebra/ofe.v
View file @
b0e11cff
...
...
@@ -239,17 +239,18 @@ End contractive.
Ltac
f_contractive
:
=
match
goal
with
|
|-
?f
_
≡
{
_
}
≡
?f
_
=>
apply
(
_
:
Proper
(
dist_later
_
==>
_
)
f
)
|
|-
?f
_
_
≡
{
_
}
≡
?f
_
_
=>
apply
(
_
:
Proper
(
dist_later
_
==>
_
==>
_
)
f
)
|
|-
?f
_
_
≡
{
_
}
≡
?f
_
_
=>
apply
(
_
:
Proper
(
_
==>
dist_later
_
==>
_
)
f
)
|
|-
?f
_
≡
{
_
}
≡
?f
_
=>
simple
apply
(
_
:
Proper
(
dist_later
_
==>
_
)
f
)
|
|-
?f
_
_
≡
{
_
}
≡
?f
_
_
=>
simple
apply
(
_
:
Proper
(
dist_later
_
==>
_
==>
_
)
f
)
|
|-
?f
_
_
≡
{
_
}
≡
?f
_
_
=>
simple
apply
(
_
:
Proper
(
_
==>
dist_later
_
==>
_
)
f
)
end
;
try
match
goal
with
|
|-
@
dist_later
?A
_
?n
?x
?y
=>
destruct
n
as
[|
n
]
;
[
exact
I
|
change
(@
dist
A
_
n
x
y
)]
end
;
try
reflexivity
.
try
simple
apply
reflexivity
.
Ltac
solve_contractive
:
=
solve_proper_core
ltac
:
(
fun
_
=>
first
[
f_contractive
|
f_equiv
]).
Ltac
solve_contractive
:
=
solve_proper_core
ltac
:
(
fun
_
=>
first
[
f_contractive
|
f_equiv
]).
(** Limit preserving predicates *)
Class
LimitPreserving
`
{!
Cofe
A
}
(
P
:
A
→
Prop
)
:
Prop
:
=
...
...
Write
Preview
Supports
Markdown
0%
Try again
or
attach a new 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