aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/class_tactics.ml4
diff options
context:
space:
mode:
authorGravatar serpyc <serpyc@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-04 10:40:03 +0000
committerGravatar serpyc <serpyc@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-04 10:40:03 +0000
commit88909c92cad0044dac83539b2b3d385242ed851e (patch)
treef8c946fc168920aab8c7e47cf875be8404f1bd10 /tactics/class_tactics.ml4
parent4b993912cc6c6135e41ea959f934fa73d1da05ab (diff)
Removal of trailing spaces.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12371 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/class_tactics.ml4')
-rw-r--r--tactics/class_tactics.ml48
1 files changed, 4 insertions, 4 deletions
diff --git a/tactics/class_tactics.ml4 b/tactics/class_tactics.ml4
index 6d1c91634..a5adb9169 100644
--- a/tactics/class_tactics.ml4
+++ b/tactics/class_tactics.ml4
@@ -82,7 +82,7 @@ let evars_to_goals p evm =
else
let goals = List.rev goals in
Some (goals, evm')
-
+
(** Typeclasses instance search tactic / eauto *)
let intersects s t =
@@ -281,7 +281,7 @@ let hints_tac hints =
in
if l = [] && !typeclasses_debug then
msgnl (pr_depth info.auto_depth ++ str": no match for " ++
- Printer.pr_constr_env (Evd.evar_env gl) concl ++
+ Printer.pr_constr_env (Evd.evar_env gl) concl ++
spc () ++ int (List.length poss) ++ str" possibilities");
List.map possible_resolve l
in
@@ -387,10 +387,10 @@ let run_on_evars ?(st=full_transparent_state) p evm tac =
Some (Evd.evars_reset_evd evm' evm)
-let eauto_tac hints = fix (or_tac intro_tac (hints_tac hints))
+let eauto_tac hints = fix (or_tac intro_tac (hints_tac hints))
let () = run_on_evars_forward := (fun hints st p evd -> run_on_evars ~st p evd (eauto_tac hints))
-
+
let eauto hints g =
let gl = { it = make_autogoal ~st:(Hint_db.transparent_state (List.hd hints)) g; sigma = project g } in
match run_tac (eauto_tac hints) gl with