You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
(** Note that the Coq standard library has a [rapply], but it is like our [rapply'] with many-holes first. We prefer fewer-holes first, for instance so that a theorem producing an equivalence will by preference be used to produce an equivalence rather than to apply the coercion of that equivalence to a function. *)
322
322
TacticNotation "rapply" uconstr(term)
323
-
:= do_with_holes ltac:(fun x => refine x) term.
323
+
:= do_with_holes ltac:(fun x => try (try (nrefine x || fail 2); fail); refine x) term.
Copy file name to clipboardExpand all lines: theories/Homotopy/Join/JoinAssoc.v
+3-3
Original file line number
Diff line number
Diff line change
@@ -80,7 +80,7 @@ Definition trijoinrecdata_fun_twist (A B C : Type)
80
80
Definition equiv_trijoin_twist' (A B C : Type)
81
81
: TriJoin A B C <~> TriJoin B A C.
82
82
Proof.
83
-
rapply (opyon_equiv_0gpd (A:=Type)).
83
+
refine (opyon_equiv_0gpd (A:=Type) _).
84
84
apply trijoinrecdata_fun_twist.
85
85
Defined.
86
86
@@ -122,7 +122,7 @@ Definition trijoin_twist_homotopic (A B C : Type)
122
122
Proof.
123
123
symmetry.
124
124
(** Both sides are [trijoin_rec] applied to [TriJoinRecData]: *)
125
-
rapply (fmap trijoin_rec).
125
+
refine (fmap trijoin_rec _).
126
126
bundle_trijoinrecpath; intros; cbn.
127
127
1: refine (ap inverse _).
128
128
1, 2, 3: apply ap_idmap.
@@ -375,7 +375,7 @@ Definition hexagon_join_twist_sym A B C
375
375
== trijoin_twist B C A o trijoin_id_sym B A C o trijoin_twist A B C.
376
376
Proof.
377
377
(* It's enough to show that both sides induces the same natural transformation under the covariant Yoneda embedding, i.e., after postcomposing with a general function [f]. *)
378
-
rapply (opyon_faithful_0gpd (A:=Type)).
378
+
refine (opyon_faithful_0gpd (A:=Type) _ _ _ _ _).
379
379
intros P f.
380
380
(* We replace [f] by [trijoin_rec t] for generic [t]. This will allow induction later. *)
0 commit comments