# HG changeset patch # User wenzelm # Date 1450798497 -3600 # Node ID d5ead6bfa1ff34f58213b34fb9e537cc7e59dbaf # Parent a759f69db1f6fd8ecb84cdea2a714136492757f6 isabelle update_cartouches -c -t; diff -r a759f69db1f6 -r d5ead6bfa1ff src/HOL/Eisbach/Examples.thy --- a/src/HOL/Eisbach/Examples.thy Tue Dec 22 14:41:35 2015 +0000 +++ b/src/HOL/Eisbach/Examples.thy Tue Dec 22 16:34:57 2015 +0100 @@ -41,13 +41,13 @@ print_fact U\) lemma "\x. P x \ Q x \ A x \ B x \ R x y \ True" - apply match_test -- \Valid match, but not quite what we were expecting..\ - back -- \Can backtrack over matches, exploring all bindings\ + apply match_test \ \Valid match, but not quite what we were expecting..\ + back \ \Can backtrack over matches, exploring all bindings\ back back back back - back -- \Found the other conjunction\ + back \ \Found the other conjunction\ back back back @@ -57,7 +57,7 @@ lemma focus_test: shows "\x. \x. P x \ P x" - apply (my_spec "x :: 'a", assumption)? -- \Wrong x\ + apply (my_spec "x :: 'a", assumption)? \ \Wrong x\ apply (match conclusion in "P x" for x \ \my_spec x, assumption\) done @@ -102,7 +102,7 @@ print_term Q\) lemma "\x. P x \ Q x \ Q x \ Q x" - apply my_spec_guess2? -- \Fails. Note that both "P"s must match\ + apply my_spec_guess2? \ \Fails. Note that both "P"s must match\ oops lemma "\x. P x \ Q x \ P x \ Q x" @@ -141,7 +141,7 @@ subsection \Solves combinator\ lemma "A \ B \ A \ B" - apply (solves \rule conjI\)? -- \Doesn't solve the goal!\ + apply (solves \rule conjI\)? \ \Doesn't solve the goal!\ apply (solves \rule conjI, assumption, assumption\) done @@ -184,7 +184,7 @@ done lemma "(\x. P x \ Q x) \ P z \ P y \ Q y" - apply (solves \guess_all, prop_solver\) -- \Try it without solve\ + apply (solves \guess_all, prop_solver\) \ \Try it without solve\ done method guess_ex =