diff options
Diffstat (limited to 'test-suite/success/univers.v')
-rw-r--r-- | test-suite/success/univers.v | 21 |
1 files changed, 21 insertions, 0 deletions
diff --git a/test-suite/success/univers.v b/test-suite/success/univers.v index 0a4b284f..a619b8da 100644 --- a/test-suite/success/univers.v +++ b/test-suite/success/univers.v @@ -17,3 +17,24 @@ Lemma lem3 : (P:Prop)P. Intro P ; Pattern P. Apply lem2. Abort. + +(* Check managing of universe constraints in inversion *) +(* Bug report #855 *) + +Inductive dep_eq : (X:Type) X -> X -> Prop := + | intro_eq : (X:Type) (f:X)(dep_eq X f f) + | intro_feq : (A:Type) (B:A->Type) + let T = (x:A)(B x) in + (f, g:T) (x:A) + (dep_eq (B x) (f x) (g x)) -> + (dep_eq T f g). + +Require Import Relations. + +Theorem dep_eq_trans : (X:Type) (transitive X (dep_eq X)). +Proof. + Unfold transitive. + Intros X f g h H1 H2. + Inversion H1. +Abort. + |