diff options
author | Jason Gross <jgross@mit.edu> | 2017-05-24 16:51:37 -0400 |
---|---|---|
committer | Jason Gross <jgross@mit.edu> | 2017-05-28 09:38:36 -0400 |
commit | 08751d1328c11a6e1a8427a12970587b12b9878a (patch) | |
tree | ef1f4f5c7339b1f35363cdd72b9bb48b74ee62cb /theories/Init | |
parent | c6a05d73fc195cc7d5ffb62f2109617701d4791c (diff) |
Use the rew dependent notation in ex, ex2 proofs
Diffstat (limited to 'theories/Init')
-rw-r--r-- | theories/Init/Logic.v | 19 |
1 files changed, 10 insertions, 9 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v index 1cd2f4cde..4db11ae77 100644 --- a/theories/Init/Logic.v +++ b/theories/Init/Logic.v @@ -650,6 +650,13 @@ Qed. Declare Left Step iff_stepl. Declare Right Step iff_trans. +Local Notation "'rew' 'dependent' H 'in' H'" + := (match H with + | eq_refl => H' + end) + (at level 10, H' at level 10, + format "'[' 'rew' 'dependent' '/ ' H in '/' H' ']'"). + (** Equality for [ex] *) Section ex. Local Unset Implicit Arguments. @@ -680,9 +687,7 @@ Section ex. => ex_intro (Q y) (rew H in u1) - match H in (_ = y) return Q y (rew H in u1) with - | eq_refl => u2 - end + (rew dependent H in u2) end. Proof. destruct H, u; reflexivity. @@ -731,12 +736,8 @@ Section ex2. (Q y) (R y) (rew H in u1) - match H in (_ = y) return Q y (rew H in u1) with - | eq_refl => u2 - end - match H in (_ = y) return R y (rew H in u1) with - | eq_refl => u3 - end + (rew dependent H in u2) + (rew dependent H in u3) end. Proof. destruct H, u; reflexivity. |