aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-22 20:23:05 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-22 20:23:05 +0000
commit287058532aefd848df5d83ee29707359672b626f (patch)
tree47c55470a6af179ce2ae5fa677bccdb774d32fb2 /toplevel
parent5a183ead91244c881df39bb817a9dded2769bd8f (diff)
Add the option to automatically introduce variables declared before the
colon in (mutual) proofs with [Set Automatic Introduction]. Fix a minor test-suite issue in ProgramWf due to new handling of the default obligation tactic. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12351 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/command.ml23
-rw-r--r--toplevel/vernacentries.ml8
2 files changed, 25 insertions, 6 deletions
diff --git a/toplevel/command.ml b/toplevel/command.ml
index 3b25f2fa6..1086e8419 100644
--- a/toplevel/command.ml
+++ b/toplevel/command.ml
@@ -1095,7 +1095,7 @@ let compute_proof_name = function
in
next (Pfedit.get_all_proof_names ()) default_thm_id
-let save_remaining_recthms (local,kind) body opaq i (id,(t_i,imps)) =
+let save_remaining_recthms (local,kind) body opaq i (id,(t_i,(_,imps))) =
match body with
| None ->
(match local with
@@ -1212,14 +1212,19 @@ let look_for_mutual_statements thms =
(* 4.2| General support for goals *)
let start_proof_com kind thms hook =
+ let evdref = ref (create_evar_defs Evd.empty) in
+ let env = Global.env () in
let thms = List.map (fun (sopt,(bl,t)) ->
- (compute_proof_name sopt,
- interp_type_evars_impls (Global.env()) (generalize_constr_expr t bl)))
+ let (env, ctx), imps = interp_context_evars evdref env bl in
+ let t', imps' = interp_type_evars_impls ~evdref env t in
+ let len = List.length ctx in
+ (compute_proof_name sopt,
+ (nf_isevar !evdref (it_mkProd_or_LetIn t' ctx), (len, imps @ lift_implicits len imps'))))
thms in
let rec_tac,thms = look_for_mutual_statements thms in
match thms with
| [] -> anomaly "No proof to start"
- | (id,(t,imps))::other_thms ->
+ | (id,(t,(len,imps)) as thm)::other_thms ->
let hook strength ref =
let other_thms_data =
if other_thms = [] then [] else
@@ -1230,8 +1235,14 @@ let start_proof_com kind thms hook =
List.iter (fun (strength,ref,imps) ->
maybe_declare_manual_implicits false ref imps;
hook strength ref) thms_data in
- start_proof id kind t ?init_tac:rec_tac
- ~compute_guard:(rec_tac<>None) hook
+ let init_tac =
+ let intro_tac (_, (_, (len, _))) = Refiner.tclDO len Tactics.intro in
+ if Flags.is_auto_intros () then
+ match rec_tac with
+ | None -> Some (intro_tac thm)
+ | Some tac -> Some (Tacticals.tclTHENS tac (List.map intro_tac thms))
+ else rec_tac
+ in start_proof id kind t ?init_tac hook ~compute_guard:(rec_tac<>None)
let check_anonymity id save_ident =
if atompart_of_id id <> "Unnamed_thm" then
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index 7cde4f637..5ee98db59 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -842,6 +842,14 @@ let _ =
let _ =
declare_bool_option
{ optsync = true;
+ optname = "automatic introduction of variables";
+ optkey = ["Automatic";"Introduction"];
+ optread = Flags.is_auto_intros;
+ optwrite = make_auto_intros }
+
+let _ =
+ declare_bool_option
+ { optsync = true;
optname = "coercion printing";
optkey = ["Printing";"Coercions"];
optread = (fun () -> !Constrextern.print_coercions);