dropped redundant setup
authorhaftmann
Thu, 29 Dec 2011 10:47:56 +0100
changeset 46032 0da934e135b0
parent 46031 ac6bae9fdc2f
child 46033 6fc579c917b8
dropped redundant setup
src/HOL/Quickcheck_Narrowing.thy
--- a/src/HOL/Quickcheck_Narrowing.thy	Thu Dec 29 10:47:56 2011 +0100
+++ b/src/HOL/Quickcheck_Narrowing.thy	Thu Dec 29 10:47:56 2011 +0100
@@ -134,15 +134,10 @@
 lemma zero_code_int_code [code, code_unfold]:
   "(0\<Colon>code_int) = Numeral0"
   by (simp add: number_of_code_int_def Pls_def)
-lemma [code_post]: "Numeral0 = (0\<Colon>code_int)"
-  using zero_code_int_code ..
 
 lemma one_code_int_code [code, code_unfold]:
   "(1\<Colon>code_int) = Numeral1"
   by (simp add: number_of_code_int_def Pls_def Bit1_def)
-lemma [code_post]: "Numeral1 = (1\<Colon>code_int)"
-  using one_code_int_code ..
-
 
 definition div_mod_code_int :: "code_int \<Rightarrow> code_int \<Rightarrow> code_int \<times> code_int" where
   [code del]: "div_mod_code_int n m = (n div m, n mod m)"