changeset 52709 | 0e4bacf21e77 |
parent 48985 | 5386df44a037 |
child 57512 | cc97b347b301 |
52708:13e6014ed42b | 52709:0e4bacf21e77 |
---|---|
185 oops |
185 oops |
186 |
186 |
187 |
187 |
188 text{*unification failure trace *} |
188 text{*unification failure trace *} |
189 |
189 |
190 ML "trace_unify_fail := true" |
190 declare [[unify_trace_failure = true]] |
191 |
191 |
192 lemma "P(a, f(b, g(e,a), b), a) \<Longrightarrow> P(a, f(b, g(c,a), b), a)" |
192 lemma "P(a, f(b, g(e,a), b), a) \<Longrightarrow> P(a, f(b, g(c,a), b), a)" |
193 txt{* |
193 txt{* |
194 @{subgoals[display,indent=0,margin=65]} |
194 @{subgoals[display,indent=0,margin=65]} |
195 apply assumption |
195 apply assumption |
210 Clash: == =/= Trueprop |
210 Clash: == =/= Trueprop |
211 Clash: == =/= Trueprop |
211 Clash: == =/= Trueprop |
212 *} |
212 *} |
213 oops |
213 oops |
214 |
214 |
215 ML "trace_unify_fail := false" |
215 declare [[unify_trace_failure = false]] |
216 |
216 |
217 |
217 |
218 text{*Quantifiers*} |
218 text{*Quantifiers*} |
219 |
219 |
220 text {* |
220 text {* |