# HG changeset patch # User paulson # Date 982327626 -3600 # Node ID 0420158197740706b21cf4989bfa26ead1c5c107 # Parent 950ede59c05a8ca259ad91c57776db070ac3d43f for the change to LEAST diff -r 950ede59c05a -r 042015819774 doc-src/TutorialI/Rules/Basic.thy --- a/doc-src/TutorialI/Rules/Basic.thy Fri Feb 16 13:37:21 2001 +0100 +++ b/doc-src/TutorialI/Rules/Basic.thy Fri Feb 16 13:47:06 2001 +0100 @@ -228,7 +228,7 @@ theorem Least_equality: "\ P (k::nat); \x. P x \ k \ x \ \ (LEAST x. P(x)) = k" -apply (simp add: Least_def) +apply (simp add: Least_def LeastM_def) txt{*omit maybe? @{subgoals[display,indent=0,margin=65]} @@ -266,7 +266,7 @@ (*both can be done by blast, which however hasn't been introduced yet*) lemma "[| P (k::nat); \x. P x \ k \ x |] ==> (LEAST x. P(x)) = k"; -apply (simp add: Least_def) +apply (simp add: Least_def LeastM_def) by (blast intro: some_equality order_antisym); theorem axiom_of_choice: "(\x. \y. P x y) \ \f. \x. P x (f x)"