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

Remove forgotten admit in f2c246c6.

Also, I removed the @ from lookup_weaken since the Coq bug we
experienced before somehow disappeared.
parent e06b1653
No related branches found
No related tags found
No related merge requests found
......@@ -123,13 +123,10 @@ Section gmap.
Lemma big_sepM_proper Φ Ψ m :
( k x, m !! k = Some x Φ k x ⊣⊢ Ψ k x)
([ map] k x m, Φ k x) ⊣⊢ ([ map] k x m, Ψ k x).
Proof. (*
(* FIXME: Coq bug since 8.5pl1. Without the @ in [@lookup_weaken] it gives
File "./algebra/upred_big_op.v", line 114, characters 4-131:
Anomaly: Uncaught exception Univ.AlreadyDeclared. Please report. *)
intros [??] ?; apply (anti_symm (⊢)); apply big_sepM_mono;
eauto using equiv_entails, equiv_entails_sym, @lookup_weaken.
Qed. *) Admitted.
Proof.
intros ?; apply (anti_symm ()); apply big_sepM_mono;
eauto using equiv_entails, equiv_entails_sym, lookup_weaken.
Qed.
Global Instance big_sepM_ne m n :
Proper (pointwise_relation _ (pointwise_relation _ (dist n)) ==> (dist n))
......
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