aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorSimonBoulier2018-11-15 09:42:08 +0100
committerSimonBoulier2019-08-16 11:43:51 +0200
commit6414a2a96f6d9a237baf08b7b449a55ee5d34376 (patch)
tree1c8a24841e921cb46f5ba11fdeb228486f8b795a
parent889603e7a2ed41b890e43729aa0abf90bebd3ca6 (diff)
Add a file for typing_flags in the test-suite.
-rw-r--r--test-suite/success/typing_flags.v38
1 files changed, 38 insertions, 0 deletions
diff --git a/test-suite/success/typing_flags.v b/test-suite/success/typing_flags.v
new file mode 100644
index 0000000000..31550b45a6
--- /dev/null
+++ b/test-suite/success/typing_flags.v
@@ -0,0 +1,38 @@
+
+Print Typing Flags.
+Unset Guard Checking.
+Fixpoint f' (n : nat) : nat := f' n.
+
+Fixpoint f (n : nat) : nat.
+Proof.
+ exact (f n).
+Defined.
+
+Fixpoint bla (A:Type) (n:nat) := match n with 0 =>0 | S n => n end.
+
+Print Typing Flags.
+
+Set Guard Checking.
+
+Print Assumptions f.
+
+Unset Universes Checking.
+
+Definition T := Type.
+Fixpoint g (n : nat) : T := T.
+
+Print Typing Flags.
+Set Universes Checking.
+
+Fail Definition g2 (n : nat) : T := T.
+
+Fail Definition e := fix e (n : nat) : nat := e n.
+
+Unset Positivity Checking.
+
+Inductive Cor :=
+| Over : Cor
+| Next : ((Cor -> list nat) -> list nat) -> Cor.
+
+Set Positivity Checking.
+Print Assumptions Cor.