remove two examples, now that the definition of "fst" and "snd" has changed
authorblanchet
Fri, 28 May 2010 22:51:04 +0200
changeset 37181 23ab9a5c41cf
parent 37180 d47fe9260c24
child 37182 71c8565dae38
remove two examples, now that the definition of "fst" and "snd" has changed
src/HOL/Nitpick_Examples/Core_Nits.thy
--- a/src/HOL/Nitpick_Examples/Core_Nits.thy	Fri May 28 22:34:21 2010 +0200
+++ b/src/HOL/Nitpick_Examples/Core_Nits.thy	Fri May 28 22:51:04 2010 +0200
@@ -638,14 +638,6 @@
 nitpick [expect = none]
 by (simp add: snd_def)
 
-lemma "fst p = (THE a. \<exists>b. p = Pair a b)"
-nitpick [expect = none]
-by (simp add: fst_def)
-
-lemma "snd p = (THE b. \<exists>a. p = Pair a b)"
-nitpick [expect = none]
-by (simp add: snd_def)
-
 lemma "I = (\<lambda>x. x) \<Longrightarrow> fst = (\<lambda>x. fst (I x))"
 nitpick [expect = none]
 by auto