Skip to content

Commit

Permalink
Merge pull request #24 from coq-community/remove-floor
Browse files Browse the repository at this point in the history
Remove floor.v
  • Loading branch information
pi8027 committed Jul 15, 2024
2 parents 037b40c + 05e8b85 commit 3b24987
Show file tree
Hide file tree
Showing 4 changed files with 6 additions and 111 deletions.
1 change: 0 additions & 1 deletion _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -42,7 +42,6 @@ theories/z3irrational.v
theories/z3seq_props.v
theories/rho_computations.v
theories/multinomial.v
theories/floor.v
theories/hanson_elem_arith.v
theories/hanson_elem_analysis.v
theories/hanson.v
101 changes: 0 additions & 101 deletions theories/floor.v

This file was deleted.

13 changes: 5 additions & 8 deletions theories/hanson.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
Require Import ZArith.
From mathcomp Require Import all_ssreflect all_algebra all_field.
Require Import extra_mathcomp tactics binomialz floor arithmetics posnum.
From mathcomp Require Import all_ssreflect all_algebra all_field archimedean.
Require Import extra_mathcomp tactics binomialz arithmetics posnum.
Require Import rat_of_Z hanson_elem_arith hanson_elem_analysis.

Set Implicit Arguments.
Expand Down Expand Up @@ -522,13 +522,10 @@ suff [K [Kpos KP]] : exists K : nat,
exists K; split => // -[| n]; first by rewrite expn0 muln1 iter_lcmn0.
case: n => [| n]; first by rewrite iter_lcmn1 muln_gt0 Kpos.
by apply/leq_trans/KP/n_between_a => //; apply/lcm_leq_Cnk.
suff [K [Kpos KP]] : exists K : rat,
suff [K [/ltW/trunc_itv/andP[_ Kpos] KP]] : exists K : rat,
(0 < K) /\ forall n k, cond n k -> (C n k.+1)%:R <= K * 3%:R ^ n.
move: (floorQ K) (floorQ_ge0 (ltW Kpos)) (floorQ_spec K).
case=> // k _ /andP [_ leKSn]; exists k.+1; split=> // n m {}/KP KP.
suff: (C n m.+1)%:R <= (k%:Q + 1) * 3%:R ^ n.
by rewrite -[_ + 1%:R]natrD -[_ ^ n]natrX -natrM ler_nat addn1.
exact/le_trans/ler_wpM2r/ltW/leKSn/exprz_ge0.
exists (Num.trunc K).+1; split=> // n m {}/KP.
by rewrite -(ler_nat rat) natrM natrX => /le_trans-> //; apply/ler_wpM2r/ltW.
move mE: 10%N%:Q => m. (* FIXME *)
have lt0m : 0 < m by rewrite -mE.
have le0m : 0 <= m by exact: ltW.
Expand Down
2 changes: 1 addition & 1 deletion theories/hanson_elem_arith.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
From mathcomp Require Import all_ssreflect all_algebra.
Require Import extra_mathcomp tactics floor arithmetics multinomial.
Require Import extra_mathcomp tactics arithmetics multinomial.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down

0 comments on commit 3b24987

Please sign in to comment.