aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/typeops.ml
diff options
context:
space:
mode:
Diffstat (limited to 'kernel/typeops.ml')
-rw-r--r--kernel/typeops.ml18
1 files changed, 9 insertions, 9 deletions
diff --git a/kernel/typeops.ml b/kernel/typeops.ml
index 46ee8d97e..46cf163bf 100644
--- a/kernel/typeops.ml
+++ b/kernel/typeops.ml
@@ -1,10 +1,10 @@
-(***********************************************************************)
-(* v * The Coq Proof Assistant / The Coq Development Team *)
-(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
-(* \VV/ *************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(***********************************************************************)
+(************************************************************************)
+(* v * The Coq Proof Assistant / The Coq Development Team *)
+(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
+(* \VV/ **************************************************************)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(************************************************************************)
(* $Id$ *)
@@ -319,8 +319,8 @@ let type_fixpoint env lna lar vdefj =
with NotConvertibleVect i ->
error_ill_typed_rec_body env i lna vdefj lar
-(***********************************************************************)
-(***********************************************************************)
+(************************************************************************)
+(************************************************************************)
(* This combinator adds the universe constraints both in the local
graph and in the universes of the environment. This is to ensure