diff options
Diffstat (limited to 'test-suite/bugs/closed/3815.v')
-rw-r--r-- | test-suite/bugs/closed/3815.v | 9 |
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3815.v b/test-suite/bugs/closed/3815.v new file mode 100644 index 00000000..5fb48398 --- /dev/null +++ b/test-suite/bugs/closed/3815.v @@ -0,0 +1,9 @@ +Require Import Setoid Coq.Program.Basics. +Global Open Scope program_scope. +Axiom foo : forall A (f : A -> A), f ∘ f = f. +Require Import Coq.Program.Combinators. +Hint Rewrite foo. +Theorem t {A B C D} (f : A -> A) (g : B -> C) (h : C -> D) +: f ∘ f = f. +Proof. + rewrite_strat topdown (hints core). |