src/Tools/eqsubst.ML
changeset 58318 f95754ca7082
parent 54742 7a86358a3c0b
child 58826 2ed2eaabe3df
--- a/src/Tools/eqsubst.ML	Thu Sep 11 20:01:29 2014 +0200
+++ b/src/Tools/eqsubst.ML	Thu Sep 11 21:11:03 2014 +0200
@@ -29,7 +29,7 @@
   val eqsubst_asm_tac': Proof.context ->
     (searchinfo -> int -> term -> match skipseq) -> int -> thm -> int -> tactic
   val eqsubst_tac: Proof.context ->
-    int list -> (* list of occurences to rewrite, use [0] for any *)
+    int list -> (* list of occurrences to rewrite, use [0] for any *)
     thm list -> int -> tactic
   val eqsubst_tac': Proof.context ->
     (searchinfo -> term -> match Seq.seq) (* search function *)
@@ -292,7 +292,7 @@
   in stepthms |> Seq.maps rewrite_with_thm end;
 
 
-(* General substitution of multiple occurances using one of
+(* General substitution of multiple occurrences using one of
    the given theorems *)
 
 fun skip_first_occs_search occ srchf sinfo lhs =
@@ -300,9 +300,9 @@
     SkipMore _ => Seq.empty
   | SkipSeq ss => Seq.flat ss);
 
-(* The "occs" argument is a list of integers indicating which occurence
+(* The "occs" argument is a list of integers indicating which occurrence
 w.r.t. the search order, to rewrite. Backtracking will also find later
-occurences, but all earlier ones are skipped. Thus you can use [0] to
+occurrences, but all earlier ones are skipped. Thus you can use [0] to
 just find all rewrites. *)
 
 fun eqsubst_tac ctxt occs thms i st =