diff options
author | Enrico Tassi <Enrico.Tassi@inria.fr> | 2018-06-19 13:54:05 +0200 |
---|---|---|
committer | Enrico Tassi <Enrico.Tassi@inria.fr> | 2018-06-20 14:22:06 +0200 |
commit | fb825197d08554a208437ee31755a783ce48708b (patch) | |
tree | 6c8aae2d29535b210a9619ddbd59d372c6516880 /test-suite | |
parent | 6ba59cef7e143f1db6e272af165da5334e324e63 (diff) |
[ssr] test case for rewrite (setoid) making the goal illtyped
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/ssr/ssr_rew_illtyped.v | 9 |
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/ssr/ssr_rew_illtyped.v b/test-suite/ssr/ssr_rew_illtyped.v new file mode 100644 index 000000000..7358068c8 --- /dev/null +++ b/test-suite/ssr/ssr_rew_illtyped.v @@ -0,0 +1,9 @@ +From Coq Require Import ssreflect Setoid. + +Structure SEProp := {prop_of : Prop; _ : prop_of <-> True}. + +Fact anomaly: forall P : SEProp, prop_of P. +Proof. +move=> [P E]. +Fail rewrite E. +Abort. |