Skip to content
GitLab
Projects
Groups
Snippets
Help
Loading...
Help
What's new
7
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Open sidebar
David Swasey
coq-stdpp
Commits
62389c82
Commit
62389c82
authored
Oct 04, 2016
by
Zhen Zhang
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
tweak the Qp lemmas
parent
f9c54965
Changes
1
Hide whitespace changes
Inline
Side-by-side
Showing
1 changed file
with
5 additions
and
2 deletions
+5
-2
theories/numbers.v
theories/numbers.v
+5
-2
No files found.
theories/numbers.v
View file @
62389c82
...
...
@@ -567,9 +567,12 @@ Proof.
apply
Qp_eq
;
simpl
.
ring
.
Qed
.
Lemma
Qp_ge_1
(
q
:
Qp
)
:
¬
((
1
+
q
)%
Qp
≤
1
%
Qp
)%
Qc
.
Lemma
Qp_
not_plus_q_
ge_1
(
q
:
Qp
)
:
¬
((
1
+
q
)%
Qp
≤
1
%
Qp
)%
Qc
.
Proof
.
intros
Hle
.
apply
(
Qcplus_le_mono_l
q
0
1
)
in
Hle
.
apply
Qcle_ngt
in
Hle
.
by
destruct
q
.
apply
Qcle_ngt
in
Hle
.
apply
Hle
,
Qp_prf
.
Qed
.
Lemma
Qp_ge_0
(
q
:
Qp
)
:
(
0
≤
q
)%
Qc
.
Proof
.
apply
Qclt_le_weak
,
Qp_prf
.
Qed
.
Write
Preview
Markdown
is supported
0%
Try again
or
attach a new file
.
Attach a file
Cancel
You are about to add
0
people
to the discussion. Proceed with caution.
Finish editing this message first!
Cancel
Please
register
or
sign in
to comment