aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Matej Kosik <m4tej.kosik@gmail.com>2015-11-04 19:31:05 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-12-10 09:35:14 +0100
commit5edfac63b6feb0b8d6ddad47a4ca9c8b5905b03a (patch)
tree49e82e45f7b00b4a813bb56c30e2f336e8edf834
parent2b7368ae43fefb6f151b7032b351f0da796f6cc3 (diff)
COMMENT: questions
-rw-r--r--doc/refman/RefMan-cic.tex29
1 files changed, 29 insertions, 0 deletions
diff --git a/doc/refman/RefMan-cic.tex b/doc/refman/RefMan-cic.tex
index ddd9f075e..b862db320 100644
--- a/doc/refman/RefMan-cic.tex
+++ b/doc/refman/RefMan-cic.tex
@@ -1910,7 +1910,36 @@ impredicative system for sort \Set{} become:
{\compat{I:\Set}{I\ra s}}}
\end{description}
+% QUESTION: Why, when I add this definition:
+%
+% Inductive foo : Type := .
+%
+% Coq claims that the type of 'foo' is 'Prop'?
+
+% QUESTION: If I add this definition:
+%
+% Inductive bar (A:Type) : Type := .
+%
+% then Coq claims that 'bar' has type 'Type → Prop' where I would expect 'Type → Type' with appropriate constraint.
+% QUESTION: If I add this definition:
+%
+% Inductive foo (A:Type) : Type :=
+% | foo1 : foo A
+% | foo2 : foo A.
+%
+% then Coq claims that 'foo' has type 'Type → Set'.
+% Why?
+
+% NOTE: If I add this definition:
+%
+% Inductive foo (A:Type) : Type :=
+% | foo1 : foo A
+% | foo2 : A → foo A.
+%
+% then Coq claims, as expected, that:
+%
+% foo : Type → Type.
%%% Local Variables:
%%% mode: latex