diff options
author | Jason Gross <jgross@mit.edu> | 2017-04-25 14:41:36 -0400 |
---|---|---|
committer | Jason Gross <jgross@mit.edu> | 2017-05-28 09:38:36 -0400 |
commit | 0a2362cd8547bc073d60470c2a49174dd15634d0 (patch) | |
tree | abdfe61d8b69ef174bc5a0137896fcd3e286310c /theories/Init | |
parent | 97480f826658043204d41a9454f96a355a608853 (diff) |
Remove motive argument from [rew dependent]
Diffstat (limited to 'theories/Init')
-rw-r--r-- | theories/Init/Specif.v | 18 |
1 files changed, 9 insertions, 9 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v index 2b4cc745f..fc7250e2f 100644 --- a/theories/Init/Specif.v +++ b/theories/Init/Specif.v @@ -220,12 +220,12 @@ Qed. (** Equality of sigma types *) Import EqNotations. -Local Notation "'rew' 'dependent' [ Q ] H 'in' H'" - := (match H as p in (_ = y) return Q y (rew p in _) with +Local Notation "'rew' 'dependent' H 'in' H'" + := (match H with | eq_refl => H' end) (at level 10, H' at level 10, - format "'[' 'rew' 'dependent' [ Q ] '/ ' H in '/' H' ']'"). + format "'[' 'rew' 'dependent' '/ ' H in '/' H' ']'"). (** Equality for [sigT] *) Section sigT. @@ -309,7 +309,7 @@ Section sigT. = existT (Q y) (rew H in projT1 u) - (rew dependent [Q] H in (projT2 u)). + (rew dependent H in (projT2 u)). Proof. destruct H, u; reflexivity. Defined. @@ -380,7 +380,7 @@ Section sig. = exist (Q y) (rew H in proj1_sig u) - (rew dependent [Q] H in proj2_sig u). + (rew dependent H in proj2_sig u). Proof. destruct H, u; reflexivity. Defined. @@ -494,8 +494,8 @@ Section sigT2. (Q y) (R y) (rew H in projT1 u) - (rew dependent [Q] H in projT2 u) - (rew dependent [R] H in projT3 u). + (rew dependent H in projT2 u) + (rew dependent H in projT3 u). Proof. destruct H, u; reflexivity. Defined. @@ -609,8 +609,8 @@ Section sig2. (Q y) (R y) (rew H in proj1_sig u) - (rew dependent [Q] H in proj2_sig u) - (rew dependent [R] H in proj3_sig u). + (rew dependent H in proj2_sig u) + (rew dependent H in proj3_sig u). Proof. destruct H, u; reflexivity. Defined. |