Skip to content

Commit

Permalink
Merge branch 'beforepoly' of /Users/mat/research/coq/git into trunk
Browse files Browse the repository at this point in the history
  • Loading branch information
mattam82 committed Dec 19, 2012
2 parents e615099 + 883da1e commit 3d84c09
Show file tree
Hide file tree
Showing 4 changed files with 3 additions and 7 deletions.
3 changes: 0 additions & 3 deletions test-suite/success/indelim.v
Expand Up @@ -11,9 +11,6 @@ Inductive False : Prop :=.


Inductive Empty_set : Set :=. Inductive Empty_set : Set :=.


Fail Inductive Large_set : Set :=
large_constr : forall A : Set, A -> Large_set.

Fail Inductive Large_set : Set := Fail Inductive Large_set : Set :=
large_constr : forall A : Set, A -> Large_set. large_constr : forall A : Set, A -> Large_set.


Expand Down
3 changes: 1 addition & 2 deletions toplevel/record.ml
Expand Up @@ -407,8 +407,7 @@ open Autoinstance
(* [fs] corresponds to fields and [ps] to parameters; [coers] is a (* [fs] corresponds to fields and [ps] to parameters; [coers] is a
list telling if the corresponding fields must me declared as coercions list telling if the corresponding fields must me declared as coercions
or subinstances *) or subinstances *)
let definition_structure (kind,finite,infer,(is_coe,(loc,idstruc)),ps,cfs,idbuild,s) = let definition_structure (kind,poly,finite,infer,(is_coe,(loc,idstruc)),ps,cfs,idbuild,s) =
let poly = Flags.use_polymorphic_flag () in
let cfs,notations = List.split cfs in let cfs,notations = List.split cfs in
let cfs,priorities = List.split cfs in let cfs,priorities = List.split cfs in
let coers,fs = List.split cfs in let coers,fs = List.split cfs in
Expand Down
2 changes: 1 addition & 1 deletion toplevel/record.mli
Expand Up @@ -35,6 +35,6 @@ val declare_structure : Decl_kinds.recursivity_kind ->
inductive inductive


val definition_structure : val definition_structure :
inductive_kind * Decl_kinds.recursivity_kind * bool(**infer?*)* lident with_coercion * local_binder list * inductive_kind * Decl_kinds.polymorphic * Decl_kinds.recursivity_kind * bool(**infer?*)* lident with_coercion * local_binder list *
(local_decl_expr with_instance with_priority with_notation) list * (local_decl_expr with_instance with_priority with_notation) list *
identifier * constr_expr option -> global_reference identifier * constr_expr option -> global_reference
2 changes: 1 addition & 1 deletion toplevel/vernacentries.ml
Expand Up @@ -525,7 +525,7 @@ let vernac_record k poly finite infer struc binders sort nameopt cfs =
match x with match x with
| Vernacexpr.AssumExpr ((loc, Name id), _) -> Dumpglob.dump_definition (loc,id) false "proj" | Vernacexpr.AssumExpr ((loc, Name id), _) -> Dumpglob.dump_definition (loc,id) false "proj"
| _ -> ()) cfs); | _ -> ()) cfs);
ignore(Record.definition_structure (k,finite,infer,struc,binders,cfs,const,sort)) ignore(Record.definition_structure (k,poly,finite,infer,struc,binders,cfs,const,sort))


let vernac_inductive poly finite infer indl = let vernac_inductive poly finite infer indl =
if Dumpglob.dump () then if Dumpglob.dump () then
Expand Down

0 comments on commit 3d84c09

Please sign in to comment.