Skip to content
GitLab
Menu
Projects
Groups
Snippets
Help
Help
Support
Community forum
Keyboard shortcuts
?
Submit feedback
Contribute to GitLab
Sign in / Register
Toggle navigation
Menu
Open sidebar
Janno
iris-coq
Commits
fda80965
Commit
fda80965
authored
Sep 29, 2017
by
Robbert Krebbers
Browse files
Fix regression caused by
e17ac4ad
and another similar bug.
parent
c0253c3e
Changes
2
Hide whitespace changes
Inline
Side-by-side
theories/proofmode/tactics.v
View file @
fda80965
...
...
@@ -535,16 +535,17 @@ a goal [P] for non-dependent arguments [x_i : P]. *)
Tactic
Notation
"iIntoValid"
open_constr
(
t
)
:
=
let
rec
go
t
:
=
let
tT
:
=
type
of
t
in
first
[
apply
(
proj1
(
_
:
AsValid
tT
_
)
t
)
|
lazymatch
eval
hnf
in
tT
with
|
?P
→
?Q
=>
let
H
:
=
fresh
in
assert
P
as
H
;
[|
go
uconstr
:
(
t
H
)
;
clear
H
]
|
∀
_
:
?T
,
_
=>
(* Put [T] inside an [id] to avoid TC inference from being invoked. *)
(* This is a workarround for Coq bug #4969. *)
let
e
:
=
fresh
in
evar
(
e
:
id
T
)
;
let
e'
:
=
eval
unfold
e
in
e
in
clear
e
;
go
(
t
e'
)
end
]
in
lazymatch
eval
hnf
in
tT
with
|
?P
→
?Q
=>
let
H
:
=
fresh
in
assert
P
as
H
;
[|
go
uconstr
:
(
t
H
)
;
clear
H
]
|
∀
_
:
?T
,
_
=>
(* Put [T] inside an [id] to avoid TC inference from being invoked. *)
(* This is a workarround for Coq bug #4969. *)
let
e
:
=
fresh
in
evar
(
e
:
id
T
)
;
let
e'
:
=
eval
unfold
e
in
e
in
clear
e
;
go
(
t
e'
)
|
_
=>
let
tT'
:
=
eval
cbv
zeta
in
tT
in
apply
(
proj1
(
_
:
AsValid
tT'
_
)
t
)
||
fail
"iPoseProof: not a uPred"
end
in
go
t
.
(* The tactic [tac] is called with a temporary fresh name [H]. The argument
...
...
theories/tests/proofmode.v
View file @
fda80965
...
...
@@ -201,6 +201,18 @@ Lemma test_True_intros : (True : uPred M) -∗ True.
Proof
.
iIntros
"?"
.
done
.
Qed
.
Lemma
test_iPoseProof_let
P
Q
:
(
let
R
:
=
True
%
I
in
R
∗
P
⊢
Q
)
→
P
⊢
Q
.
Proof
.
iIntros
(
help
)
"HP"
.
iPoseProof
(
help
with
"[$HP]"
)
as
"?"
.
done
.
Qed
.
Lemma
test_iIntros_let
P
:
∀
Q
,
let
R
:
=
True
%
I
in
P
-
∗
R
-
∗
Q
-
∗
P
∗
Q
.
Proof
.
iIntros
(
Q
R
)
"$ HR $"
.
Qed
.
End
tests
.
Section
more_tests
.
...
...
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