Skip to content

Commit

Permalink
fix a few warnings
Browse files Browse the repository at this point in the history
  • Loading branch information
Casteran committed Jan 3, 2024
1 parent 5ee6c80 commit 45e65f5
Show file tree
Hide file tree
Showing 2 changed files with 11 additions and 7 deletions.
15 changes: 9 additions & 6 deletions theories/ordinals/Prelude/Merge_Sort.v
Original file line number Diff line number Diff line change
Expand Up @@ -244,15 +244,18 @@ Section Generic.
- rewrite <- (LocallySorted_cons' A le).
split.
+ apply (merge_Forall (le a1) l0 (a2::l3)).
* rewrite <- LocallySorted_cons' in H1; intuition.
* rewrite <- LocallySorted_cons' in H2; intuition.
* rewrite <- LocallySorted_cons' in H1.
now destruct H1.
apply le_total.
* rewrite <- LocallySorted_cons' in H2.
intuition.
apply forall_weak with a2 ...
apply le_total. intuition.
apply le_total.
now constructor.
+ eapply H0 ...
rewrite <- LocallySorted_cons' in H1; intuition.
+ apply le_total.
- rewrite <- LocallySorted_cons'.
- rewrite <- LocallySorted_cons'.
split.
+ apply (merge_Forall (le a2) (a1::l0) l3).
* rewrite <- LocallySorted_cons' in H1; intuition.
Expand All @@ -264,8 +267,8 @@ Section Generic.
* rewrite <- LocallySorted_cons' in H2; intuition.
+ eapply H0 ...
rewrite <- LocallySorted_cons' in H2; intuition.
+ apply le_total.
Qed.
+ apply le_total.
Qed.

Lemma merge_permutation:
forall l1 l2, Permutation (l1++l2) (merge (fun x y => bool_decide (x <= y)) l1 l2).
Expand Down
3 changes: 2 additions & 1 deletion theories/ordinals/Schutte/Schutte_basics.v
Original file line number Diff line number Diff line change
Expand Up @@ -475,7 +475,8 @@ Proof. (* .no-out *)
(*| .. coq:: no-out |*)
destruct (@AX3 (Singleton alpha)).
- apply countable_singleton.
- unfold succ_spec; apply the_least_unicity; exists x; intuition.
- unfold succ_spec; apply the_least_unicity; exists x.
apply H; split.
Qed.
(*||*)
(* end snippet succOkb *)
Expand Down

0 comments on commit 45e65f5

Please sign in to comment.