src/Doc/Tutorial/Rules/Basic.thy
changeset 52709 0e4bacf21e77
parent 48985 5386df44a037
child 57512 cc97b347b301
--- a/src/Doc/Tutorial/Rules/Basic.thy	Fri Jul 19 16:36:13 2013 +0200
+++ b/src/Doc/Tutorial/Rules/Basic.thy	Fri Jul 19 17:35:12 2013 +0200
@@ -187,7 +187,7 @@
 
 text{*unification failure trace *}
 
-ML "trace_unify_fail := true"
+declare [[unify_trace_failure = true]]
 
 lemma "P(a, f(b, g(e,a), b), a) \<Longrightarrow> P(a, f(b, g(c,a), b), a)"
 txt{*
@@ -212,7 +212,7 @@
 *}
 oops
 
-ML "trace_unify_fail := false"
+declare [[unify_trace_failure = false]]
 
 
 text{*Quantifiers*}