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

Make arguments for sig and sigT constructors and projections maximally implicit.

Some were already maximally implicit, some were not. Now it is consistent.
parent c1687739
No related branches found
No related tags found
No related merge requests found
......@@ -551,7 +551,12 @@ Instance option_inhabited {A} : Inhabited (option A) := populate None.
(** ** Sigma types *)
Arguments existT {_ _} _ _.
Arguments projT1 {_ _} _.
Arguments projT2 {_ _} _.
Arguments exist {_} _ _ _.
Arguments proj1_sig {_ _} _.
Arguments proj2_sig {_ _} _.
Notation "x ↾ p" := (exist _ x p) (at level 20) : C_scope.
Notation "` x" := (proj1_sig x) (at level 10, format "` x") : C_scope.
......
......@@ -186,7 +186,7 @@ Qed.
Instance coPset_leibniz : LeibnizEquiv coPset.
Proof.
intros X Y; rewrite elem_of_equiv; intros HXY.
apply (sig_eq_pi _), coPset_eq; try apply proj2_sig.
apply (sig_eq_pi _), coPset_eq; try apply @proj2_sig.
intros p; apply eq_bool_prop_intro, (HXY p).
Qed.
......
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