Skip to content
Snippets Groups Projects
Commit 5657f5ca authored by Jacques-Henri Jourdan's avatar Jacques-Henri Jourdan
Browse files

sig_equivI

parent 42ecd0a6
No related branches found
No related tags found
No related merge requests found
......@@ -592,5 +592,10 @@ Lemma cofe_funC_equivI {A B} (f g : A -c> B) : f ≡ g ⊣⊢ ∀ x, f x ≡ g x
Proof. by unseal. Qed.
Lemma cofe_morC_equivI {A B : ofeT} (f g : A -n> B) : f g ⊣⊢ x, f x g x.
Proof. by unseal. Qed.
(* Sig ofes *)
Lemma sig_equivI {A : ofeT} (P : A Prop) (x y : sigC P) :
x y ⊣⊢ proj1_sig x proj1_sig y.
Proof. by unseal. Qed.
End primitive.
End uPred.
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