Skip to content

Commit

Permalink
adapt to mc#1300
Browse files Browse the repository at this point in the history
  • Loading branch information
Tragicus committed Nov 27, 2024
1 parent 1739214 commit 957fd92
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion theories/proof/coloring.v
Original file line number Diff line number Diff line change
Expand Up @@ -263,7 +263,7 @@ have oE_G'' w: order edge w = #|predD1 (cedge (h'' w)) unx|.
have [u_nx | nx'u] := altP eqP.
by apply/imageP => [[wu _ u_wu]]; case/eqP: (valP wu); rewrite -[RHS]u_nx.
set wu : G'' := Sub u nx'u; rewrite (mem_image Ih'' _ wu) /=.
apply: etrans (eq_fconnect (glink_fp_skip_edge _) w wu) _.
apply: etrans (@eq_fconnect _ _ _ (glink_fp_skip_edge _) w wu) _.
by rewrite /glink /= -!val_eqE /= nnx !eqxx /= orbT.
exact: (fconnect_skip edgeI w wu).
have [|k [kE kF]] := minimal_counter_example_is_minimal cexG _ ltG''G.
Expand Down
2 changes: 1 addition & 1 deletion theories/proof/discharge.v
Original file line number Diff line number Diff line change
Expand Up @@ -217,7 +217,7 @@ Qed.

Lemma dscore_mirror (x : G) : @dscore (mirror G) x = dscore x.
Proof.
rewrite /dscore arity_mirror (eq_bigl _ _ (cface_mirror x)); congr (_ + _).
rewrite /dscore arity_mirror (eq_bigl _ _ (@cface_mirror _ x)); congr (_ + _).
suffices{x} score1F (x : G): @dscore1 (mirror G) (face x) = dscore1 x.
rewrite (reindex_inj (@faceI G)) -(eq_bigl _ _ (fun y => cface1r y x)) /=.
by apply: eq_bigr => y _; rewrite /dscore2 2!{1}score1F (plain_eq' geoG).
Expand Down
2 changes: 1 addition & 1 deletion theories/proof/geometry.v
Original file line number Diff line number Diff line change
Expand Up @@ -158,7 +158,7 @@ Lemma iter_face_subn n x :
Proof. by move=> le_n_x; rewrite -iterD subnK ?iter_face_arity. Qed.

Lemma arity_mirror : @arity (mirror G) =1 @arity G.
Proof. by move=> x; apply/eq_card/(cface_mirror x). Qed.
Proof. by move=> x; apply/eq_card/(@cface_mirror _ x). Qed.

Section SimplePaths.

Expand Down

0 comments on commit 957fd92

Please sign in to comment.