Skip to content

Commit

Permalink
removing troublesome lemma
Browse files Browse the repository at this point in the history
  • Loading branch information
zstone1 authored and proux01 committed Oct 2, 2024
1 parent bab1cb0 commit 881be66
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 21 deletions.
3 changes: 1 addition & 2 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -37,8 +37,7 @@
`big_lexi_le_reflexive`, `big_lexi_le_anti`, `big_lexi_le_trans`,
`big_lexi_le_total`, `start_with_prefix`, `leEbig_lexi_order`,
`big_lexi_order_prefix_lt`, `big_lexi_order_prefix_gt`,
`big_lexi_order_between`, `big_lexi_order_interval_prefix`, and
`big_lexi_order_prefix_closed_itv`.
`big_lexi_order_between`, and `big_lexi_order_interval_prefix`.

### Changed

Expand Down
19 changes: 0 additions & 19 deletions classical/classical_orders.v
Original file line number Diff line number Diff line change
Expand Up @@ -356,22 +356,3 @@ move: i; case=> [][[]l|[]] [[]r|[]] [][]; rewrite ?in_itv /= ?andbT.
by move=> _; exists 0 => ? ?; rewrite set_itvE.
Qed.
End big_lexi_intervals.

(** TODO: generalize to tbOrderType when that's available in mathcomp *)
Lemma big_lexi_order_prefix_closed_itv {d} {K : nat -> finOrderType d} n
(x : big_lexi_order K) :
same_prefix n x = `[
(start_with n x (fun=>\bot):big_lexi_order K)%O,
(start_with n x (fun=>\top))%O].
Proof.
rewrite eqEsubset; split=> [z pfxz|z]; first last.
rewrite set_itvE /= => xbt; apply: same_prefix_trans.
exact: (start_with_prefix _ (fun=> \bot)%O).
apply/same_prefix_sym/(big_lexi_order_between xbt).
apply: same_prefix_trans (start_with_prefix _ _).
exact/same_prefix_sym/start_with_prefix.
rewrite set_itvE /= !leEbig_lexi_order; apply/andP; split;
case E : (first_diff _ _) => [m|] //; rewrite /start_with /=.
- by case: ifPn => [/pfxz -> //|]; rewrite le0x.
- by case: ifPn => [/pfxz -> //|]; rewrite lex1.
Qed.

0 comments on commit 881be66

Please sign in to comment.