diff -r ca6ca6fc28af -r 25d11b449e92 Nominal/Ex/Classical.thy --- a/Nominal/Ex/Classical.thy Tue Aug 07 18:53:50 2012 +0100 +++ b/Nominal/Ex/Classical.thy Tue Aug 07 18:54:52 2012 +0100 @@ -67,7 +67,7 @@ (if b=d then ImpR (x)..(M[d\c>e]) e else ImpR (x)..(M[d\c>e]) b)" | "atom a \ (d, e) \ (ImpL .M (x).N y)[d\c>e] = ImpL .(M[d\c>e]) (x).(N[d\c>e]) y" apply(simp only: eqvt_def) - apply(simp only: crename_graph_def) + apply(simp only: crename_graph_aux_def) apply (rule, perm_simp, rule) apply(rule TrueI) -- "covered all cases" @@ -272,7 +272,7 @@ | "atom x \ (u, v) \ (ImpL .M (x).N y)[u\n>v] = (if y=u then ImpL .(M[u\n>v]) (x).(N[u\n>v]) v else ImpL .(M[u\n>v]) (x).(N[u\n>v]) y)" apply(simp only: eqvt_def) - apply(simp only: nrename_graph_def) + apply(simp only: nrename_graph_aux_def) apply (rule, perm_simp, rule) apply(rule TrueI) -- "covered all cases" @@ -474,7 +474,7 @@ (if y=z then Cut .P (z').ImpL .(M{y:=.P}) (x).(N{y:=.P}) z' else ImpL .(M{y:=.P}) (x).(N{y:=.P}) z)" apply(simp only: eqvt_def) - apply(simp only: substn_graph_def) + apply(simp only: substn_graph_aux_def) apply (rule, perm_simp, rule) apply(rule TrueI) -- "covered all cases"