Skip to content

Commit

Permalink
Redefine \min and \max in function_scope
Browse files Browse the repository at this point in the history
  • Loading branch information
pi8027 authored and proux01 committed Jan 15, 2024
1 parent bedcf0c commit 8bc854a
Showing 1 changed file with 3 additions and 8 deletions.
11 changes: 3 additions & 8 deletions classical/mathcomp_extra.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,8 +15,6 @@ From mathcomp Require Import finset interval.
(* This files contains lemmas and definitions missing from MathComp. *)
(* *)
(* ``` *)
(* f \max g := fun x => Num.max (f x) (g x) *)
(* f \min g := fun x => Num.min (f x) (g x) *)
(* oflit f := Some \o f *)
(* pred_oapp T D := [pred x | oapp (mem D) false x] *)
(* f \* g := fun x => f x * g x *)
Expand Down Expand Up @@ -49,6 +47,9 @@ Reserved Notation "\- f" (at level 35, f at level 35).

Number Notation positive Pos.of_num_int Pos.to_num_uint : AC_scope.

Notation "f \min g" := (Order.min_fun f g) : function_scope.
Notation "f \max g" := (Order.max_fun f g) : function_scope.

Lemma all_sig2_cond {I : Type} {T : Type} (D : pred I)
(P Q : I -> T -> Prop) : T ->
(forall x : I, D x -> {y : T | P x y & Q x y}) ->
Expand Down Expand Up @@ -1384,12 +1385,6 @@ rewrite horner_poly !big_ord_recr !big_ord0/= !Monoid.simpm/= expr1.
by rewrite -mulrA -expr2 addrC addrA addrAC.
Qed.

Reserved Notation "f \min g" (at level 50, left associativity).

Definition min_fun T (R : numDomainType) (f g : T -> R) x := Num.min (f x) (g x).
Notation "f \min g" := (min_fun f g) : ring_scope.
Arguments min_fun {T R} _ _ _ /.

(* NB: Coq 8.17.0 generalizes dependent_choice from Set to Type
making the following lemma redundant *)
Section dependent_choice_Type.
Expand Down

0 comments on commit 8bc854a

Please sign in to comment.