Skip to content
Snippets Groups Projects
Commit b0e11cff authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Bump coq-stdpp.

parent 9c189816
No related branches found
No related tags found
No related merge requests found
coq-stdpp https://gitlab.mpi-sws.org/robbertkrebbers/coq-stdpp ee6200b4d74bfd06034f3cc36d1afdc309427e5c
coq-stdpp https://gitlab.mpi-sws.org/robbertkrebbers/coq-stdpp 24cc2e4786b2344e092e412f56e96c6971ab60d8
......@@ -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 :=
......
......@@ -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 :=
......
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