changeset 3842 | b55686a7b22c |
parent 3210 | e80db1660614 |
child 7295 | fe09a0c5cebe |
--- a/src/HOL/Modelcheck/MuCalculus.thy Fri Oct 10 18:37:49 1997 +0200 +++ b/src/HOL/Modelcheck/MuCalculus.thy Fri Oct 10 19:02:28 1997 +0200 @@ -18,7 +18,7 @@ defs -Charfun_def "Charfun == (% A.% x.x:A)" +Charfun_def "Charfun == (% A.% x. x:A)" monoP_def "monoP f == mono(Collect o f o Charfun)" mu_def "mu f == Charfun(lfp(Collect o f o Charfun))" nu_def "nu f == Charfun(gfp(Collect o f o Charfun))"