diff options
author | Xavier Clerc <xavier.clerc@inria.fr> | 2015-01-28 14:26:19 +0100 |
---|---|---|
committer | Xavier Clerc <xavier.clerc@inria.fr> | 2015-01-28 14:26:19 +0100 |
commit | 51b15993cb4a9cc2521b6107b7f4195b21040087 (patch) | |
tree | 88770fda6bf2cac9ecee156f9869f9974a0bf2dd /test-suite/bugs/opened/3944.v | |
parent | 754e66eb2878eb964e0369226ae809ecadb1b376 (diff) |
Several reproduction cases for the test suite.
Diffstat (limited to 'test-suite/bugs/opened/3944.v')
-rw-r--r-- | test-suite/bugs/opened/3944.v | 4 |
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/3944.v b/test-suite/bugs/opened/3944.v new file mode 100644 index 000000000..3d0deb4c5 --- /dev/null +++ b/test-suite/bugs/opened/3944.v @@ -0,0 +1,4 @@ +Require Import Setoid. +Class C (T : Type) := c : T. +Goal forall T (i : C T) (v : T), True. +setoid_rewrite plus_n_Sm. |