Skip to content
GitLab
Projects
Groups
Snippets
Help
Loading...
Help
What's new
10
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Open sidebar
Janno
iris-coq
Commits
94768d56
Commit
94768d56
authored
Feb 20, 2016
by
Ralf Jung
Browse files
Options
Browse Files
Download
Email Patches
Plain Diff
fix transitivity change
parent
08b69a69
Changes
2
Hide whitespace changes
Inline
Side-by-side
Showing
2 changed files
with
2 additions
and
2 deletions
+2
-2
prelude/lexico.v
prelude/lexico.v
+1
-1
prelude/list.v
prelude/list.v
+1
-1
No files found.
prelude/lexico.v
View file @
94768d56
...
...
@@ -52,7 +52,7 @@ Proof.
-
intros
[
x
y
].
apply
prod_lexico_irreflexive
.
by
apply
(
irreflexivity
lexico
y
).
-
intros
[??]
[??]
[??]
??.
eapply
prod_lexico_transitive
;
eauto
.
apply
trans
.
eapply
prod_lexico_transitive
;
eauto
.
apply
trans
itivity
.
Qed
.
Instance
prod_lexico_trichotomyT
`
{
Lexico
A
,
tA
:
!
TrichotomyT
(@
lexico
A
_
)}
`
{
Lexico
B
,
tB
:
!
TrichotomyT
(@
lexico
B
_
)}
:
TrichotomyT
(@
lexico
(
A
*
B
)
_
).
...
...
prelude/list.v
View file @
94768d56
...
...
@@ -2493,7 +2493,7 @@ Section Forall2_order.
Global Instance: Symmetric R → Symmetric (Forall2 R).
Proof. intros. induction 1; constructor; auto. Qed.
Global Instance: Transitive R → Transitive (Forall2 R).
Proof. intros ????. apply Forall2_transitive. by apply @trans. Qed.
Proof. intros ????. apply Forall2_transitive. by apply @trans
itivity
. Qed.
Global Instance: Equivalence R → Equivalence (Forall2 R).
Proof. split; apply _. Qed.
Global Instance: PreOrder R → PreOrder (Forall2 R).
...
...
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