aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Amin Timany <amintimany@gmail.com>2017-04-28 11:12:26 +0200
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-06-16 04:51:16 +0200
commit9903b47cdccc2fe98a905ab085cb24ca36de1aed (patch)
tree37249aac01e0dcdb8c3c9c9e6c65391f5ee6804f
parent9468e4b49bd2f397b5e1bd2b7994cc84929fb6ac (diff)
Disable debug printing
Fix a mistake in record declaration
-rw-r--r--kernel/subtyping.ml4
-rw-r--r--test-suite/bugs/closed/3330.v6
-rw-r--r--test-suite/success/polymorphism.v2
-rw-r--r--vernac/record.ml2
4 files changed, 4 insertions, 10 deletions
diff --git a/kernel/subtyping.ml b/kernel/subtyping.ml
index 60cd77f40..60e630a6d 100644
--- a/kernel/subtyping.ml
+++ b/kernel/subtyping.ml
@@ -303,10 +303,6 @@ let check_constant cst env mp1 l info1 cb2 spec2 subst1 subst2 =
let ctx2 = Univ.instantiate_univ_context cb2.const_universes in
let inst1, ctx1 = Univ.UContext.dest ctx1 in
let inst2, ctx2 = Univ.UContext.dest ctx2 in
- output_string stderr "\ninst1:\n";
- output_string stderr (Pp.string_of_ppcmds (Univ.Instance.pr Univ.Level.pr inst1));
- output_string stderr "\ninst2:\n";
- output_string stderr (Pp.string_of_ppcmds (Univ.Instance.pr Univ.Level.pr inst2)); flush stderr;
if not (Univ.Instance.length inst1 == Univ.Instance.length inst2) then
error IncompatibleInstances
else
diff --git a/test-suite/bugs/closed/3330.v b/test-suite/bugs/closed/3330.v
index a497e7a98..672fb3f13 100644
--- a/test-suite/bugs/closed/3330.v
+++ b/test-suite/bugs/closed/3330.v
@@ -1072,10 +1072,8 @@ Section Adjunction.
Variable F : Functor C D.
Variable G : Functor D C.
-(* Let Adjunction_Type :=
- Eval simpl in (hom_functor D) o (F^op, 1) <~=~> (hom_functor C) o (1, G).*)
-
- Set Printing All. Set Printing Universes.
+ Let Adjunction_Type :=
+ Eval simpl in (hom_functor D) o (F^op, 1) <~=~> (hom_functor C) o (1, G).
Record AdjunctionHom :=
{
diff --git a/test-suite/success/polymorphism.v b/test-suite/success/polymorphism.v
index f57cbcc2b..ecc988507 100644
--- a/test-suite/success/polymorphism.v
+++ b/test-suite/success/polymorphism.v
@@ -360,7 +360,7 @@ End F.
Set Universe Polymorphism.
-Record box (X : Type) (T := Type) : Type := wrap { unwrap : T }.
+Cumulative Record box (X : Type) (T := Type) : Type := wrap { unwrap : T }.
Section test_letin_subtyping.
Universe i j k i' j' k'.
diff --git a/vernac/record.ml b/vernac/record.ml
index 8a83dceef..b95131b72 100644
--- a/vernac/record.ml
+++ b/vernac/record.ml
@@ -584,7 +584,7 @@ let definition_structure (kind,cum,poly,finite,(is_coe,((loc,idstruc),pl)),ps,cf
let implfs = List.map
(fun impls -> implpars @ Impargs.lift_implicits
(succ (List.length params)) impls) implfs in
- let ind = declare_structure Finite cum poly (Universes.univ_inf_ind_from_universe_context ctx) idstruc
+ let ind = declare_structure finite cum poly (Universes.univ_inf_ind_from_universe_context ctx) idstruc
idbuild implpars params arity template implfs
fields is_coe (List.map (fun coe -> not (Option.is_empty coe)) coers) sign in
IndRef ind