aboutsummaryrefslogtreecommitdiff
path: root/test-suite/failure
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2020-02-07 18:13:25 +0100
committerPierre-Marie Pédrot2020-02-09 16:38:14 +0100
commitb6264bb2df9b73b905af126ede49cd31abf0e7da (patch)
tree6eddb39c2870eb12be6d6cdb5cfe15f9eaf55513 /test-suite/failure
parent1820f40590ec358b40e3a9c444f80c5283e55292 (diff)
Remove the Template Check option.
Diffstat (limited to 'test-suite/failure')
-rw-r--r--test-suite/failure/Template.v28
1 files changed, 0 insertions, 28 deletions
diff --git a/test-suite/failure/Template.v b/test-suite/failure/Template.v
deleted file mode 100644
index fbd9c8bcba..0000000000
--- a/test-suite/failure/Template.v
+++ /dev/null
@@ -1,28 +0,0 @@
-
-Module TestUnsetTemplateCheck.
- Unset Template Check.
-
- Section Foo.
-
- Context (A : Type).
-
- Definition cstr := nat : ltac:(let ty := type of A in exact ty).
-
- Inductive myind :=
- | cons : A -> myind.
- End Foo.
-
- (* Can only succeed if no template check is performed *)
- Check myind True : Prop.
-
- About myind.
-
- (* test discharge puts things in the right order (by using the
- checker on the result) *)
- Section S.
-
- Variables (A:Type) (a:A).
- Inductive bb (B:Type) := BB : forall a', a = a' -> B -> bb B.
- End S.
-
-End TestUnsetTemplateCheck.