Skip to content

Commit

Permalink
Fixes 20231117 (math-comp#1106)
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist committed Dec 7, 2023
1 parent 480ca05 commit 1b4404e
Show file tree
Hide file tree
Showing 6 changed files with 12 additions and 7 deletions.
3 changes: 3 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -26,6 +26,9 @@

### Renamed

- in `exp.v`:
+ `lnX` -> `lnXn`

### Generalized

### Deprecated
Expand Down
1 change: 1 addition & 0 deletions theories/Make
Original file line number Diff line number Diff line change
Expand Up @@ -13,6 +13,7 @@ reals.v
landau.v
Rstruct.v
topology.v
cantor.v
prodnormedzmodule.v
normedtype.v
realfun.v
Expand Down
9 changes: 5 additions & 4 deletions theories/cantor.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,9 @@
(* mathcomp analysis (c) 2017 Inria and AIST. License: CeCILL-C. *)
From mathcomp Require Import all_ssreflect ssralg ssrint ssrnum.
From mathcomp Require Import interval rat fintype finmap.
Require Import mathcomp_extra boolp classical_sets signed functions cardinality.
Require Import reals topology.
From mathcomp Require Import all_ssreflect ssralg ssrint ssrnum interval rat.
From mathcomp Require Import finmap.
From mathcomp Require Import mathcomp_extra boolp classical_sets functions.
From mathcomp Require Import cardinality.
Require Import reals signed topology.
From HB Require Import structures.

(******************************************************************************)
Expand Down
2 changes: 1 addition & 1 deletion theories/constructive_ereal.v
Original file line number Diff line number Diff line change
Expand Up @@ -624,7 +624,7 @@ Context {R : numDomainType}.
Implicit Type (x : \bar R).

Definition fin_num := [qualify a x : \bar R | (x != -oo) && (x != +oo)].
Fact fin_num_key : pred_key fin_num. by []. Qed.
Fact fin_num_key : pred_key fin_num. Proof. by []. Qed.
Canonical fin_num_keyd := KeyedQualifier fin_num_key.

Lemma fin_numE x : (x \is a fin_num) = (x != -oo) && (x != +oo).
Expand Down
2 changes: 1 addition & 1 deletion theories/exp.v
Original file line number Diff line number Diff line change
Expand Up @@ -631,7 +631,7 @@ Proof. by move=> x y x_gt0 y_gt0; rewrite -ltr_expR !lnK. Qed.
Lemma ler_ln : {in Num.pos &, {mono ln : x y / x <= y}}.
Proof. by move=> x y x_gt0 y_gt0; rewrite -ler_expR !lnK. Qed.

Lemma lnX n x : 0 < x -> ln(x ^+ n) = ln x *+ n.
Lemma lnXn n x : 0 < x -> ln (x ^+ n) = ln x *+ n.
Proof.
move=> x_gt0; elim: n => [|n ih] /=; first by rewrite expr0 ln1 mulr0n.
by rewrite !exprS lnM ?qualifE//= ?exprn_gt0// mulrS ih.
Expand Down
2 changes: 1 addition & 1 deletion theories/topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -2520,7 +2520,7 @@ HB.instance Definition _ :=

End Product_Topology.

(** dnbhs *)
(** deleted neighborhood *)

Definition dnbhs {T : topologicalType} (x : T) :=
within (fun y => y != x) (nbhs x).
Expand Down

0 comments on commit 1b4404e

Please sign in to comment.