src/HOL/Nominal/Nominal.thy
changeset 58318 f95754ca7082
parent 58310 91ea607a34d8
child 58372 bfd497f2f4c2
--- a/src/HOL/Nominal/Nominal.thy	Thu Sep 11 20:01:29 2014 +0200
+++ b/src/HOL/Nominal/Nominal.thy	Thu Sep 11 21:11:03 2014 +0200
@@ -3650,7 +3650,7 @@
 method_setup fresh_fun_simp = {*
   Scan.lift (Args.parens (Args.$$$ "no_asm") >> K true || Scan.succeed false) >>
     (fn b => fn ctxt => SIMPLE_METHOD' (fresh_fun_tac ctxt b))
-*} "delete one inner occurence of fresh_fun"
+*} "delete one inner occurrence of fresh_fun"
 
 
 (************************************************)