Skip to content

Commit a779b65

Browse files
author
Patrick Nicodemus
committed
using Jason's first definition
1 parent 1cb4677 commit a779b65

File tree

19 files changed

+29
-36
lines changed

19 files changed

+29
-36
lines changed

theories/Algebra/AbGroups/Abelianization.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -248,7 +248,7 @@ Section AbelGroup.
248248
intros x y z; cbn beta.
249249
lhs nrapply ap.
250250
2: rhs nrapply ap.
251-
1,3: lhs rapply inverse_sg_op; nrapply (ap (.* _)); rapply inverse_sg_op.
251+
1,3: lhs tapply inverse_sg_op; nrapply (ap (.* _)); tapply inverse_sg_op.
252252
change (abel_in z^ * abel_in y^ * abel_in x^
253253
= abel_in y^ * abel_in z^ * abel_in x^).
254254
apply (ap (.* _)).

theories/Algebra/AbGroups/TensorProduct.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -251,7 +251,7 @@ Definition ab_tensor_prod_ind_hprop_triple {A B C : AbGroup}
251251
Proof.
252252
rapply (ab_tensor_prod_ind_hprop P).
253253
- intros a.
254-
rapply (ab_tensor_prod_ind_hprop (fun x => P (tensor _ x))).
254+
rapply (ab_tensor_prod_ind_hprop (fun x => P (tensor _ x))); cbv beta.
255255
+ nrapply Hin.
256256
+ intros x y Hx Hy.
257257
rewrite tensor_dist_l.
@@ -781,15 +781,15 @@ Proof.
781781
- snrapply ab_tensor_prod_ind_homotopy.
782782
intros x.
783783
change (f $o g $o grp_homo_tensor_l x $== grp_homo_tensor_l x).
784-
rapply Abel_ind_hprop.
784+
rapply Abel_ind_hprop; cbv beta.
785785
change (@abel_in ?G) with (grp_homo_map (@abel_unit G)).
786786
repeat change (cat_comp (A:=AbGroup) ?f ?g) with (cat_comp (A:=Group) f g).
787787
change (forall y, grp_homo_map ?f (abel_unit y) = grp_homo_map ?g (abel_unit y))
788788
with (cat_comp (A:=Group) f abel_unit $== cat_comp (A:=Group) g abel_unit).
789789
rapply FreeGroup_ind_homotopy.
790790
intros y; revert x.
791791
change (f $o g $o grp_homo_tensor_r (freeabgroup_in y) $== grp_homo_tensor_r (freeabgroup_in y)).
792-
rapply Abel_ind_hprop.
792+
rapply Abel_ind_hprop; cbv beta.
793793
change (@abel_in ?G) with (grp_homo_map (@abel_unit G)).
794794
repeat change (cat_comp (A:=AbGroup) ?f ?g) with (cat_comp (A:=Group) f g).
795795
change (forall y, grp_homo_map ?f (abel_unit y) = grp_homo_map ?g (abel_unit y))

theories/Algebra/AbSES/Core.v

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -713,8 +713,6 @@ Lemma abses_from_surjection {E B : AbGroup@{u}} (p : E $-> B) `{IsSurjection p}
713713
: AbSES B (ab_kernel p).
714714
Proof.
715715
srapply (Build_AbSES E _ p).
716-
1: exact (subgroup_incl _).
717-
1: exact _.
718716
snrapply Build_IsExact.
719717
- apply phomotopy_homotopy_hset.
720718
intros [e q]; cbn.
@@ -734,7 +732,7 @@ Proof.
734732
refine (ap _ p^ @ _).
735733
tapply cx_isexact.
736734
- apply isequiv_surj_emb.
737-
1: rapply cancelR_conn_map.
735+
1: tapply cancelR_conn_map.
738736
apply isembedding_isinj_hset.
739737
srapply Quotient_ind2_hprop; intros x y.
740738
intro p.

theories/Algebra/Groups/Subgroup.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1122,7 +1122,7 @@ Proof.
11221122
snrapply subgroup_image_rec.
11231123
intros x Jx.
11241124
change (subgroup_image f J ((grp_conj y $o f) x)).
1125-
revert y; rapply (conn_map_elim (Tr (-1)) f); intros y.
1125+
revert y; rapply (conn_map_elim (Tr (-1)) f); intros y; cbv beta.
11261126
rewrite <- grp_homo_conj.
11271127
nrapply subgroup_image_in.
11281128
by rapply isnormal_conj.

theories/Algebra/Rings/CRing.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -29,7 +29,7 @@ Definition Build_CRing' (R : AbGroup) `(!One R, !Mult R)
2929
: CRing.
3030
Proof.
3131
snrapply Build_CRing.
32-
- rapply (Build_Ring R); only 1,2,4: exact _.
32+
- rapply (Build_Ring R).
3333
+ intros x y z.
3434
lhs nrapply comm.
3535
lhs rapply dist_l.

theories/Basics/Tactics.v

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -322,15 +322,15 @@ Tactic Notation "snrefine" uconstr(term) := simple notypeclasses refine term; gl
322322
(** This tactic is weaker than [tapply], and equivalent in strength to [nrapply], i.e., it should succeed iff [nrapply] succeeds, but it solves all possible typeclasses afterward. The implementation is: try [nrefine t, t _, t _ _], ... until success; upon success, revert the last (successful) application of [nrefine] and call [refine (t _ _ _)]. *)
323323
(** TODO: Find a nicer implementation of this tactic. *)
324324
Tactic Notation "rapply" uconstr(term)
325-
:= do_with_holes ltac:(fun x => assert_succeeds (nrefine x); refine x) term.
325+
:= do_with_holes ltac:(fun x => simple notypeclasses refine x) term; try typeclasses eauto; shelve_unifiable.
326326
Tactic Notation "rapply'" uconstr(term)
327-
:= do_with_holes' ltac:(fun x => assert_succeeds (nrefine x); refine x) term.
327+
:= do_with_holes' ltac:(fun x => simple notypeclasses refine x) term; try typeclasses eauto; shelve_unifiable.
328328

329329
(** See comment for [rapply]. This cannot be simplified to [snrefine x] because we don't want the [global_axiom] tactic to run here. *)
330330
Tactic Notation "srapply" uconstr(term)
331-
:= do_with_holes ltac:(fun x => assert_succeeds (simple notypeclasses refine x); srefine x) term.
331+
:= do_with_holes ltac:(fun x => simple notypeclasses refine x) term; try typeclasses eauto.
332332
Tactic Notation "srapply'" uconstr(term)
333-
:= do_with_holes' ltac:(fun x => assert_succeeds (simple notypeclasses refine x); srefine x) term.
333+
:= do_with_holes' ltac:(fun x => simple notypeclasses refine x) term; try typeclasses eauto.
334334

335335
Tactic Notation "nrapply" uconstr(term)
336336
:= do_with_holes ltac:(fun x => nrefine x) term.

theories/Classes/theory/rings.v

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -254,7 +254,8 @@ Section ring_props.
254254
Lemma negate_swap_r : forall x y, x - y = -(y - x).
255255
Proof.
256256
intros; symmetry.
257-
lhs rapply groups.inverse_sg_op.
257+
Set Printing All.
258+
lhs tapply groups.inverse_sg_op.
258259
f_ap.
259260
apply involutive.
260261
Defined.
@@ -465,7 +466,7 @@ Section ringmor_props.
465466

466467
Definition preserves_negate x : f (- x) = - f x.
467468
Proof.
468-
rapply preserves_inverse.
469+
tapply preserves_inverse.
469470
Defined.
470471

471472
Lemma preserves_minus x y : f (x - y) = f x - f y.

theories/Colimits/Colimit_Coequalizer.v

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -80,8 +80,7 @@ Section Coequalizer.
8080
: Coeq f g <~> Coequalizer f g.
8181
Proof.
8282
srapply colimit_unicity.
83-
3: eapply iscoequalizer_Coeq.
84-
eapply iscolimit_colimit.
83+
eapply iscoequalizer_Coeq.
8584
Defined.
8685

8786
End Coequalizer.

theories/Colimits/Colimit_Flattening.v

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -224,9 +224,7 @@ Section Flattening.
224224
Definition flattening_lemma : Colimit (diagram_sigma E) <~> sig E'.
225225
Proof.
226226
srapply colimit_unicity.
227-
3: apply iscolimit_colimit.
228227
rapply Build_IsColimit.
229-
apply unicocone_cocone_E'.
230228
Defined.
231229

232230
End Flattening.

theories/Colimits/Colimit_Pushout.v

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -161,7 +161,8 @@ Section is_PO_pushout.
161161

162162
Definition is_PO_pushout : is_PO f g (Pushout f g).
163163
Proof.
164-
srapply Build_IsColimit.
164+
unfold is_PO.
165+
unshelve eapply Build_IsColimit.
165166
- srapply Build_span_cocone.
166167
+ exact (push o inl).
167168
+ exact (push o inr).
@@ -201,8 +202,7 @@ Section is_PO_pushout.
201202
Definition equiv_pushout_PO : Pushout f g <~> PO f g.
202203
Proof.
203204
srapply colimit_unicity.
204-
3: eapply is_PO_pushout.
205-
eapply iscolimit_colimit.
205+
eapply is_PO_pushout.
206206
Defined.
207207

208208
Definition equiv_pushout_PO_beta_pglue (a : A)

0 commit comments

Comments
 (0)