| author | wenzelm | 
| Tue, 23 Jan 2024 12:28:35 +0100 | |
| changeset 79517 | 0856026e2c88 | 
| parent 79489 | 1e19abf373ac | 
| child 79531 | 22a137a6de44 | 
| permissions | -rw-r--r-- | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1 | (* Title: HOL/Code_Numeral.thy | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 2 | Author: Florian Haftmann, TU Muenchen | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 3 | *) | 
| 24999 | 4 | |
| 60758 | 5 | section \<open>Numeric types for code generation onto target language numerals only\<close> | 
| 24999 | 6 | |
| 31205 
98370b26c2ce
String.literal replaces message_string, code_numeral replaces (code_)index
 haftmann parents: 
31203diff
changeset | 7 | theory Code_Numeral | 
| 78669 | 8 | imports Lifting Bit_Operations | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 9 | begin | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 10 | |
| 60758 | 11 | subsection \<open>Type of target language integers\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 12 | |
| 61076 | 13 | typedef integer = "UNIV :: int set" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 14 | morphisms int_of_integer integer_of_int .. | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 15 | |
| 59487 
adaa430fc0f7
default abstypes and default abstract equations make technical (no_code) annotation superfluous
 haftmann parents: 
58889diff
changeset | 16 | setup_lifting type_definition_integer | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 17 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 18 | lemma integer_eq_iff: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 19 | "k = l \<longleftrightarrow> int_of_integer k = int_of_integer l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 20 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 21 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 22 | lemma integer_eqI: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 23 | "int_of_integer k = int_of_integer l \<Longrightarrow> k = l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 24 | using integer_eq_iff [of k l] by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 25 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 26 | lemma int_of_integer_integer_of_int [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 27 | "int_of_integer (integer_of_int k) = k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 28 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 29 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 30 | lemma integer_of_int_int_of_integer [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 31 | "integer_of_int (int_of_integer k) = k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 32 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 33 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 34 | instantiation integer :: ring_1 | 
| 24999 | 35 | begin | 
| 36 | ||
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 37 | lift_definition zero_integer :: integer | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 38 | is "0 :: int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 39 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 40 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 41 | declare zero_integer.rep_eq [simp] | 
| 24999 | 42 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 43 | lift_definition one_integer :: integer | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 44 | is "1 :: int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 45 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 46 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 47 | declare one_integer.rep_eq [simp] | 
| 24999 | 48 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 49 | lift_definition plus_integer :: "integer \<Rightarrow> integer \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 50 | is "plus :: int \<Rightarrow> int \<Rightarrow> int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 51 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 52 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 53 | declare plus_integer.rep_eq [simp] | 
| 24999 | 54 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 55 | lift_definition uminus_integer :: "integer \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 56 | is "uminus :: int \<Rightarrow> int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 57 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 58 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 59 | declare uminus_integer.rep_eq [simp] | 
| 24999 | 60 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 61 | lift_definition minus_integer :: "integer \<Rightarrow> integer \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 62 | is "minus :: int \<Rightarrow> int \<Rightarrow> int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 63 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 64 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 65 | declare minus_integer.rep_eq [simp] | 
| 24999 | 66 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 67 | lift_definition times_integer :: "integer \<Rightarrow> integer \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 68 | is "times :: int \<Rightarrow> int \<Rightarrow> int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 69 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 70 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 71 | declare times_integer.rep_eq [simp] | 
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 72 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 73 | instance proof | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 74 | qed (transfer, simp add: algebra_simps)+ | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 75 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 76 | end | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 77 | |
| 64241 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 78 | instance integer :: Rings.dvd .. | 
| 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 79 | |
| 70927 | 80 | context | 
| 81 | includes lifting_syntax | |
| 82 | notes transfer_rule_numeral [transfer_rule] | |
| 83 | begin | |
| 64241 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 84 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 85 | lemma [transfer_rule]: | 
| 70927 | 86 | "(pcr_integer ===> pcr_integer ===> (\<longleftrightarrow>)) (dvd) (dvd)" | 
| 87 | by (unfold dvd_def) transfer_prover | |
| 88 | ||
| 89 | lemma [transfer_rule]: | |
| 90 | "((\<longleftrightarrow>) ===> pcr_integer) of_bool of_bool" | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 91 | by (unfold of_bool_def) transfer_prover | 
| 68010 | 92 | |
| 93 | lemma [transfer_rule]: | |
| 70927 | 94 | "((=) ===> pcr_integer) int of_nat" | 
| 64178 | 95 | by (rule transfer_rule_of_nat) transfer_prover+ | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 96 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 97 | lemma [transfer_rule]: | 
| 70927 | 98 | "((=) ===> pcr_integer) (\<lambda>k. k) of_int" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 99 | proof - | 
| 70927 | 100 | have "((=) ===> pcr_integer) of_int of_int" | 
| 64178 | 101 | by (rule transfer_rule_of_int) transfer_prover+ | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 102 | then show ?thesis by (simp add: id_def) | 
| 24999 | 103 | qed | 
| 104 | ||
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 105 | lemma [transfer_rule]: | 
| 70927 | 106 | "((=) ===> pcr_integer) numeral numeral" | 
| 107 | by transfer_prover | |
| 26140 | 108 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 109 | lemma [transfer_rule]: | 
| 70927 | 110 | "((=) ===> (=) ===> pcr_integer) Num.sub Num.sub" | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 111 | by (unfold Num.sub_def) transfer_prover | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 112 | |
| 68010 | 113 | lemma [transfer_rule]: | 
| 70927 | 114 | "(pcr_integer ===> (=) ===> pcr_integer) (^) (^)" | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 115 | by (unfold power_def) transfer_prover | 
| 68010 | 116 | |
| 70927 | 117 | end | 
| 118 | ||
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 119 | lemma int_of_integer_of_nat [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 120 | "int_of_integer (of_nat n) = of_nat n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 121 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 122 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 123 | lift_definition integer_of_nat :: "nat \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 124 | is "of_nat :: nat \<Rightarrow> int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 125 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 126 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 127 | lemma integer_of_nat_eq_of_nat [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 128 | "integer_of_nat = of_nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 129 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 130 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 131 | lemma int_of_integer_integer_of_nat [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 132 | "int_of_integer (integer_of_nat n) = of_nat n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 133 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 134 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 135 | lift_definition nat_of_integer :: "integer \<Rightarrow> nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 136 | is Int.nat | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 137 | . | 
| 26140 | 138 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 139 | lemma nat_of_integer_of_nat [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 140 | "nat_of_integer (of_nat n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 141 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 142 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 143 | lemma int_of_integer_of_int [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 144 | "int_of_integer (of_int k) = k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 145 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 146 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 147 | lemma nat_of_integer_integer_of_nat [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 148 | "nat_of_integer (integer_of_nat n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 149 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 150 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 151 | lemma integer_of_int_eq_of_int [simp, code_abbrev]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 152 | "integer_of_int = of_int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 153 | by transfer (simp add: fun_eq_iff) | 
| 26140 | 154 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 155 | lemma of_int_integer_of [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 156 | "of_int (int_of_integer k) = (k :: integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 157 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 158 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 159 | lemma int_of_integer_numeral [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 160 | "int_of_integer (numeral k) = numeral k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 161 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 162 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 163 | lemma int_of_integer_sub [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 164 | "int_of_integer (Num.sub k l) = Num.sub k l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 165 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 166 | |
| 66190 | 167 | definition integer_of_num :: "num \<Rightarrow> integer" | 
| 168 | where [simp]: "integer_of_num = numeral" | |
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 169 | |
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 170 | lemma integer_of_num [code]: | 
| 66190 | 171 | "integer_of_num Num.One = 1" | 
| 172 | "integer_of_num (Num.Bit0 n) = (let k = integer_of_num n in k + k)" | |
| 173 | "integer_of_num (Num.Bit1 n) = (let k = integer_of_num n in k + k + 1)" | |
| 174 | by (simp_all only: integer_of_num_def numeral.simps Let_def) | |
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 175 | |
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 176 | lemma integer_of_num_triv: | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 177 | "integer_of_num Num.One = 1" | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 178 | "integer_of_num (Num.Bit0 Num.One) = 2" | 
| 66190 | 179 | by simp_all | 
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 180 | |
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 181 | instantiation integer :: equal | 
| 26140 | 182 | begin | 
| 183 | ||
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 184 | lift_definition equal_integer :: \<open>integer \<Rightarrow> integer \<Rightarrow> bool\<close> | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 185 | is \<open>HOL.equal :: int \<Rightarrow> int \<Rightarrow> bool\<close> | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 186 | . | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 187 | |
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 188 | instance | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 189 | by (standard; transfer) (fact equal_eq) | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 190 | |
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 191 | end | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 192 | |
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 193 | instantiation integer :: linordered_idom | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 194 | begin | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 195 | |
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 196 | lift_definition abs_integer :: \<open>integer \<Rightarrow> integer\<close> | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 197 | is \<open>abs :: int \<Rightarrow> int\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 198 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 199 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 200 | declare abs_integer.rep_eq [simp] | 
| 26140 | 201 | |
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 202 | lift_definition sgn_integer :: \<open>integer \<Rightarrow> integer\<close> | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 203 | is \<open>sgn :: int \<Rightarrow> int\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 204 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 205 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 206 | declare sgn_integer.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 207 | |
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 208 | lift_definition less_eq_integer :: \<open>integer \<Rightarrow> integer \<Rightarrow> bool\<close> | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 209 | is \<open>less_eq :: int \<Rightarrow> int \<Rightarrow> bool\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 210 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 211 | |
| 69946 | 212 | lemma integer_less_eq_iff: | 
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 213 | \<open>k \<le> l \<longleftrightarrow> int_of_integer k \<le> int_of_integer l\<close> | 
| 69946 | 214 | by (fact less_eq_integer.rep_eq) | 
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 215 | |
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 216 | lift_definition less_integer :: \<open>integer \<Rightarrow> integer \<Rightarrow> bool\<close> | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 217 | is \<open>less :: int \<Rightarrow> int \<Rightarrow> bool\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 218 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 219 | |
| 69946 | 220 | lemma integer_less_iff: | 
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 221 | \<open>k < l \<longleftrightarrow> int_of_integer k < int_of_integer l\<close> | 
| 69946 | 222 | by (fact less_integer.rep_eq) | 
| 223 | ||
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 224 | instance | 
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 225 | by (standard; transfer) | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 226 | (simp_all add: algebra_simps less_le_not_le [symmetric] mult_strict_right_mono linear) | 
| 26140 | 227 | |
| 228 | end | |
| 229 | ||
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 230 | instance integer :: discrete_linordered_semidom | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 231 | by (standard; transfer) | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 232 | (fact less_iff_succ_less_eq) | 
| 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 233 | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 234 | context | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 235 | includes lifting_syntax | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 236 | begin | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 237 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 238 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 239 | \<open>(pcr_integer ===> pcr_integer ===> pcr_integer) min min\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 240 | by (unfold min_def) transfer_prover | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 241 | |
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 242 | lemma [transfer_rule]: | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 243 | \<open>(pcr_integer ===> pcr_integer ===> pcr_integer) max max\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 244 | by (unfold max_def) transfer_prover | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 245 | |
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 246 | end | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 247 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 248 | lemma int_of_integer_min [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 249 | "int_of_integer (min k l) = min (int_of_integer k) (int_of_integer l)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 250 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 251 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 252 | lemma int_of_integer_max [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 253 | "int_of_integer (max k l) = max (int_of_integer k) (int_of_integer l)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 254 | by transfer rule | 
| 26140 | 255 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 256 | lemma nat_of_integer_non_positive [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 257 | "k \<le> 0 \<Longrightarrow> nat_of_integer k = 0" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 258 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 259 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 260 | lemma of_nat_of_integer [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 261 | "of_nat (nat_of_integer k) = max 0 k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 262 | by transfer auto | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 263 | |
| 66817 | 264 | instantiation integer :: unique_euclidean_ring | 
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 265 | begin | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 266 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 267 | lift_definition divide_integer :: "integer \<Rightarrow> integer \<Rightarrow> integer" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 268 | is "divide :: int \<Rightarrow> int \<Rightarrow> int" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 269 | . | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 270 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 271 | declare divide_integer.rep_eq [simp] | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 272 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 273 | lift_definition modulo_integer :: "integer \<Rightarrow> integer \<Rightarrow> integer" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 274 | is "modulo :: int \<Rightarrow> int \<Rightarrow> int" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 275 | . | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 276 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 277 | declare modulo_integer.rep_eq [simp] | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 278 | |
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 279 | lift_definition euclidean_size_integer :: "integer \<Rightarrow> nat" | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 280 | is "euclidean_size :: int \<Rightarrow> nat" | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 281 | . | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 282 | |
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 283 | declare euclidean_size_integer.rep_eq [simp] | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 284 | |
| 66838 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 285 | lift_definition division_segment_integer :: "integer \<Rightarrow> integer" | 
| 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 286 | is "division_segment :: int \<Rightarrow> int" | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 287 | . | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 288 | |
| 66838 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 289 | declare division_segment_integer.rep_eq [simp] | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 290 | |
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 291 | instance | 
| 76053 | 292 | apply (standard; transfer) | 
| 293 | apply (use mult_le_mono2 [of 1] in \<open>auto simp add: sgn_mult_abs abs_mult sgn_mult abs_mod_less sgn_mod nat_mult_distrib | |
| 294 | division_segment_mult division_segment_mod\<close>) | |
| 295 | apply (simp add: division_segment_int_def split: if_splits) | |
| 296 | done | |
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 297 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 298 | end | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 299 | |
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 300 | lemma [code]: | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 301 | "euclidean_size = nat_of_integer \<circ> abs" | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 302 | by (simp add: fun_eq_iff nat_of_integer.rep_eq) | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 303 | |
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 304 | lemma [code]: | 
| 66838 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 305 | "division_segment (k :: integer) = (if k \<ge> 0 then 1 else - 1)" | 
| 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 306 | by transfer (simp add: division_segment_int_def) | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 307 | |
| 78937 
5e6b195eee83
slightly less technical formulation of very specific type class
 haftmann parents: 
78935diff
changeset | 308 | instance integer :: linordered_euclidean_semiring | 
| 66839 | 309 | by (standard; transfer) (simp_all add: of_nat_div division_segment_int_def) | 
| 66815 | 310 | |
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 311 | instantiation integer :: ring_bit_operations | 
| 71094 | 312 | begin | 
| 313 | ||
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 314 | lift_definition bit_integer :: \<open>integer \<Rightarrow> nat \<Rightarrow> bool\<close> | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 315 | is bit . | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 316 | |
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 317 | lift_definition not_integer :: \<open>integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 318 | is not . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 319 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 320 | lift_definition and_integer :: \<open>integer \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 321 | is \<open>and\<close> . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 322 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 323 | lift_definition or_integer :: \<open>integer \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 324 | is or . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 325 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 326 | lift_definition xor_integer :: \<open>integer \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 327 | is xor . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 328 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 329 | lift_definition mask_integer :: \<open>nat \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 330 | is mask . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 331 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 332 | lift_definition set_bit_integer :: \<open>nat \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 333 | is set_bit . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 334 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 335 | lift_definition unset_bit_integer :: \<open>nat \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 336 | is unset_bit . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 337 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 338 | lift_definition flip_bit_integer :: \<open>nat \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 339 | is flip_bit . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 340 | |
| 71094 | 341 | lift_definition push_bit_integer :: \<open>nat \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 342 | is push_bit . | 
| 71094 | 343 | |
| 344 | lift_definition drop_bit_integer :: \<open>nat \<Rightarrow> integer \<Rightarrow> integer\<close> | |
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 345 | is drop_bit . | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 346 | |
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 347 | lift_definition take_bit_integer :: \<open>nat \<Rightarrow> integer \<Rightarrow> integer\<close> | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 348 | is take_bit . | 
| 71094 | 349 | |
| 350 | instance by (standard; transfer) | |
| 79480 
c7cb1bf6efa0
consolidated name of lemma analogously to nat/int/word_bit_induct
 haftmann parents: 
79072diff
changeset | 351 | (fact bit_eq_rec bit_induct bit_iff_odd push_bit_eq_mult drop_bit_eq_div take_bit_eq_mod | 
| 79488 | 352 | bits_div_0 bits_div_by_0 bits_div_by_1 even_half_succ_eq | 
| 71413 | 353 | exp_div_exp_eq div_exp_eq mod_exp_eq mult_exp_mod_exp_eq div_exp_mod_exp_eq | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 354 | even_mask_div_iff even_mult_exp_div_exp_iff | 
| 79072 
a91050cd5c93
de-duplicated specification of class ring_bit_operations
 haftmann parents: 
79031diff
changeset | 355 | and_rec or_rec xor_rec mask_eq_exp_minus_1 | 
| 79489 | 356 | set_bit_eq_or unset_bit_eq_or_xor flip_bit_eq_xor not_eq_complement)+ | 
| 71094 | 357 | |
| 358 | end | |
| 68010 | 359 | |
| 78955 | 360 | instance integer :: linordered_euclidean_semiring_bit_operations .. | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 361 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 362 | context | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 363 | includes bit_operations_syntax | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 364 | begin | 
| 71094 | 365 | |
| 366 | lemma [code]: | |
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 367 | \<open>bit k n \<longleftrightarrow> odd (drop_bit n k)\<close> | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 368 | \<open>NOT k = - k - 1\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 369 | \<open>mask n = 2 ^ n - (1 :: integer)\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 370 | \<open>set_bit n k = k OR push_bit n 1\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 371 | \<open>unset_bit n k = k AND NOT (push_bit n 1)\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 372 | \<open>flip_bit n k = k XOR push_bit n 1\<close> | 
| 71094 | 373 | \<open>push_bit n k = k * 2 ^ n\<close> | 
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 374 | \<open>drop_bit n k = k div 2 ^ n\<close> | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 375 | \<open>take_bit n k = k mod 2 ^ n\<close> for k :: integer | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 376 | by (fact bit_iff_odd_drop_bit not_eq_complement mask_eq_exp_minus_1 | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 377 | set_bit_eq_or unset_bit_eq_and_not flip_bit_eq_xor push_bit_eq_mult drop_bit_eq_div take_bit_eq_mod)+ | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 378 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 379 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 380 | \<open>k AND l = (if k = 0 \<or> l = 0 then 0 else if k = - 1 then l else if l = - 1 then k | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 381 | else (k mod 2) * (l mod 2) + 2 * ((k div 2) AND (l div 2)))\<close> for k l :: integer | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 382 | by transfer (fact and_int_unfold) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 383 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 384 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 385 | \<open>k OR l = (if k = - 1 \<or> l = - 1 then - 1 else if k = 0 then l else if l = 0 then k | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 386 | else max (k mod 2) (l mod 2) + 2 * ((k div 2) OR (l div 2)))\<close> for k l :: integer | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 387 | by transfer (fact or_int_unfold) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 388 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 389 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 390 | \<open>k XOR l = (if k = - 1 then NOT l else if l = - 1 then NOT k else if k = 0 then l else if l = 0 then k | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 391 | else \<bar>k mod 2 - l mod 2\<bar> + 2 * ((k div 2) XOR (l div 2)))\<close> for k l :: integer | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 392 | by transfer (fact xor_int_unfold) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 393 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 394 | end | 
| 68010 | 395 | |
| 78937 
5e6b195eee83
slightly less technical formulation of very specific type class
 haftmann parents: 
78935diff
changeset | 396 | instantiation integer :: linordered_euclidean_semiring_division | 
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 397 | begin | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 398 | |
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 399 | definition divmod_integer :: "num \<Rightarrow> num \<Rightarrow> integer \<times> integer" | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 400 | where | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 401 | divmod_integer'_def: "divmod_integer m n = (numeral m div numeral n, numeral m mod numeral n)" | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 402 | |
| 75883 | 403 | definition divmod_step_integer :: "integer \<Rightarrow> integer \<times> integer \<Rightarrow> integer \<times> integer" | 
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 404 | where | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 405 | "divmod_step_integer l qr = (let (q, r) = qr | 
| 75936 | 406 | in if \<bar>l\<bar> \<le> \<bar>r\<bar> then (2 * q + 1, r - l) | 
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 407 | else (2 * q, r))" | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 408 | |
| 75936 | 409 | instance by standard | 
| 410 | (auto simp add: divmod_integer'_def divmod_step_integer_def integer_less_eq_iff) | |
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 411 | |
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 412 | end | 
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 413 | |
| 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 414 | declare divmod_algorithm_code [where ?'a = integer, | 
| 69946 | 415 | folded integer_of_num_def, unfolded integer_of_num_triv, | 
| 61275 
053ec04ea866
monomorphization of divmod wrt. code generation avoids costly dictionary unpacking at runtime
 haftmann parents: 
61274diff
changeset | 416 | code] | 
| 53069 
d165213e3924
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
 haftmann parents: 
52435diff
changeset | 417 | |
| 55427 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 418 | lemma integer_of_nat_0: "integer_of_nat 0 = 0" | 
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 419 | by transfer simp | 
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 420 | |
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 421 | lemma integer_of_nat_1: "integer_of_nat 1 = 1" | 
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 422 | by transfer simp | 
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 423 | |
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 424 | lemma integer_of_nat_numeral: | 
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 425 | "integer_of_nat (numeral n) = numeral n" | 
| 
ff54d22fe357
make integer_of_char and char_of_integer work with NBE and code_simp
 Andreas Lochbihler parents: 
54489diff
changeset | 426 | by transfer simp | 
| 26140 | 427 | |
| 68010 | 428 | |
| 60758 | 429 | subsection \<open>Code theorems for target language integers\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 430 | |
| 60758 | 431 | text \<open>Constructors\<close> | 
| 26140 | 432 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 433 | definition Pos :: "num \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 434 | where | 
| 61274 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 435 | [simp, code_post]: "Pos = numeral" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 436 | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 437 | context | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 438 | includes lifting_syntax | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 439 | begin | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 440 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 441 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 442 | \<open>((=) ===> pcr_integer) numeral Pos\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 443 | by simp transfer_prover | 
| 30245 
e67f42ac1157
consequent rewrite of index_size, size [index] to nat_of; support pseudo-primrec sepcifications with fun
 haftmann parents: 
29823diff
changeset | 444 | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 445 | end | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 446 | |
| 61274 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 447 | lemma Pos_fold [code_unfold]: | 
| 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 448 | "numeral Num.One = Pos Num.One" | 
| 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 449 | "numeral (Num.Bit0 k) = Pos (Num.Bit0 k)" | 
| 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 450 | "numeral (Num.Bit1 k) = Pos (Num.Bit1 k)" | 
| 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 451 | by simp_all | 
| 
0261eec37233
more selective preprocessing allows bare "numeral" occurences to be retained as real function in generated code
 haftmann parents: 
61076diff
changeset | 452 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 453 | definition Neg :: "num \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 454 | where | 
| 54489 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 haftmann parents: 
53069diff
changeset | 455 | [simp, code_abbrev]: "Neg n = - Pos n" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 456 | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 457 | context | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 458 | includes lifting_syntax | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 459 | begin | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 460 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 461 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 462 | \<open>((=) ===> pcr_integer) (\<lambda>n. - numeral n) Neg\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 463 | by (unfold Neg_def) transfer_prover | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 464 | |
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 465 | end | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 466 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 467 | code_datatype "0::integer" Pos Neg | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 468 | |
| 64994 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 469 | |
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 470 | text \<open>A further pair of constructors for generated computations\<close> | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 471 | |
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 472 | context | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 473 | begin | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 474 | |
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 475 | qualified definition positive :: "num \<Rightarrow> integer" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 476 | where [simp]: "positive = numeral" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 477 | |
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 478 | qualified definition negative :: "num \<Rightarrow> integer" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 479 | where [simp]: "negative = uminus \<circ> numeral" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 480 | |
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 481 | lemma [code_computation_unfold]: | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 482 | "numeral = positive" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 483 | "Pos = positive" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 484 | "Neg = negative" | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 485 | by (simp_all add: fun_eq_iff) | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 486 | |
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 487 | end | 
| 
6e4c05e8edbb
computation preprocessing rules to allow literals as input for computations
 haftmann parents: 
64848diff
changeset | 488 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 489 | |
| 60758 | 490 | text \<open>Auxiliary operations\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 491 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 492 | lift_definition dup :: "integer \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 493 | is "\<lambda>k::int. k + k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 494 | . | 
| 26140 | 495 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 496 | lemma dup_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 497 | "dup 0 = 0" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 498 | "dup (Pos n) = Pos (Num.Bit0 n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 499 | "dup (Neg n) = Neg (Num.Bit0 n)" | 
| 54489 
03ff4d1e6784
eliminiated neg_numeral in favour of - (numeral _)
 haftmann parents: 
53069diff
changeset | 500 | by (transfer, simp only: numeral_Bit0 minus_add_distrib)+ | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 501 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 502 | lift_definition sub :: "num \<Rightarrow> num \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 503 | is "\<lambda>m n. numeral m - numeral n :: int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 504 | . | 
| 26140 | 505 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 506 | lemma sub_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 507 | "sub Num.One Num.One = 0" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 508 | "sub (Num.Bit0 m) Num.One = Pos (Num.BitM m)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 509 | "sub (Num.Bit1 m) Num.One = Pos (Num.Bit0 m)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 510 | "sub Num.One (Num.Bit0 n) = Neg (Num.BitM n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 511 | "sub Num.One (Num.Bit1 n) = Neg (Num.Bit0 n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 512 | "sub (Num.Bit0 m) (Num.Bit0 n) = dup (sub m n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 513 | "sub (Num.Bit1 m) (Num.Bit1 n) = dup (sub m n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 514 | "sub (Num.Bit1 m) (Num.Bit0 n) = dup (sub m n) + 1" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 515 | "sub (Num.Bit0 m) (Num.Bit1 n) = dup (sub m n) - 1" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 516 | by (transfer, simp add: dbl_def dbl_inc_def dbl_dec_def)+ | 
| 28351 | 517 | |
| 24999 | 518 | |
| 60758 | 519 | text \<open>Implementations\<close> | 
| 24999 | 520 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 521 | lemma one_integer_code [code, code_unfold]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 522 | "1 = Pos Num.One" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 523 | by simp | 
| 24999 | 524 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 525 | lemma plus_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 526 | "k + 0 = (k::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 527 | "0 + l = (l::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 528 | "Pos m + Pos n = Pos (m + n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 529 | "Pos m + Neg n = sub m n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 530 | "Neg m + Pos n = sub n m" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 531 | "Neg m + Neg n = Neg (m + n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 532 | by (transfer, simp)+ | 
| 24999 | 533 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 534 | lemma uminus_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 535 | "uminus 0 = (0::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 536 | "uminus (Pos m) = Neg m" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 537 | "uminus (Neg m) = Pos m" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 538 | by simp_all | 
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 539 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 540 | lemma minus_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 541 | "k - 0 = (k::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 542 | "0 - l = uminus (l::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 543 | "Pos m - Pos n = sub m n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 544 | "Pos m - Neg n = Pos (m + n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 545 | "Neg m - Pos n = Neg (m + n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 546 | "Neg m - Neg n = sub n m" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 547 | by (transfer, simp)+ | 
| 46028 
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
 haftmann parents: 
45694diff
changeset | 548 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 549 | lemma abs_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 550 | "\<bar>k\<bar> = (if (k::integer) < 0 then - k else k)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 551 | by simp | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46664diff
changeset | 552 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 553 | lemma sgn_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 554 | "sgn k = (if k = 0 then 0 else if (k::integer) < 0 then - 1 else 1)" | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46664diff
changeset | 555 | by simp | 
| 46028 
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
 haftmann parents: 
45694diff
changeset | 556 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 557 | lemma times_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 558 | "k * 0 = (0::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 559 | "0 * l = (0::integer)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 560 | "Pos m * Pos n = Pos (m * n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 561 | "Pos m * Neg n = Neg (m * n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 562 | "Neg m * Pos n = Neg (m * n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 563 | "Neg m * Neg n = Pos (m * n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 564 | by simp_all | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 565 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 566 | definition divmod_integer :: "integer \<Rightarrow> integer \<Rightarrow> integer \<times> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 567 | where | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 568 | "divmod_integer k l = (k div l, k mod l)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 569 | |
| 66801 | 570 | lemma fst_divmod_integer [simp]: | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 571 | "fst (divmod_integer k l) = k div l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 572 | by (simp add: divmod_integer_def) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 573 | |
| 66801 | 574 | lemma snd_divmod_integer [simp]: | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 575 | "snd (divmod_integer k l) = k mod l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 576 | by (simp add: divmod_integer_def) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 577 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 578 | definition divmod_abs :: "integer \<Rightarrow> integer \<Rightarrow> integer \<times> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 579 | where | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 580 | "divmod_abs k l = (\<bar>k\<bar> div \<bar>l\<bar>, \<bar>k\<bar> mod \<bar>l\<bar>)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 581 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 582 | lemma fst_divmod_abs [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 583 | "fst (divmod_abs k l) = \<bar>k\<bar> div \<bar>l\<bar>" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 584 | by (simp add: divmod_abs_def) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 585 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 586 | lemma snd_divmod_abs [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 587 | "snd (divmod_abs k l) = \<bar>k\<bar> mod \<bar>l\<bar>" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 588 | by (simp add: divmod_abs_def) | 
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 589 | |
| 53069 
d165213e3924
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
 haftmann parents: 
52435diff
changeset | 590 | lemma divmod_abs_code [code]: | 
| 
d165213e3924
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
 haftmann parents: 
52435diff
changeset | 591 | "divmod_abs (Pos k) (Pos l) = divmod k l" | 
| 
d165213e3924
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
 haftmann parents: 
52435diff
changeset | 592 | "divmod_abs (Neg k) (Neg l) = divmod k l" | 
| 
d165213e3924
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
 haftmann parents: 
52435diff
changeset | 593 | "divmod_abs (Neg k) (Pos l) = divmod k l" | 
| 
d165213e3924
execution of int division by class semiring_numeral_div, replacing pdivmod by divmod_abs
 haftmann parents: 
52435diff
changeset | 594 | "divmod_abs (Pos k) (Neg l) = divmod k l" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 595 | "divmod_abs j 0 = (0, \<bar>j\<bar>)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 596 | "divmod_abs 0 j = (0, 0)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 597 | by (simp_all add: prod_eq_iff) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 598 | |
| 69946 | 599 | lemma divmod_integer_eq_cases: | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 600 | "divmod_integer k l = | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 601 | (if k = 0 then (0, 0) else if l = 0 then (0, k) else | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 602 | (apsnd \<circ> times \<circ> sgn) l (if sgn k = sgn l | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 603 | then divmod_abs k l | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 604 | else (let (r, s) = divmod_abs k l in | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 605 | if s = 0 then (- r, 0) else (- r - 1, \<bar>l\<bar> - s))))" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 606 | proof - | 
| 69946 | 607 | have *: "sgn k = sgn l \<longleftrightarrow> k = 0 \<and> l = 0 \<or> 0 < l \<and> 0 < k \<or> l < 0 \<and> k < 0" for k l :: int | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 608 | by (auto simp add: sgn_if) | 
| 69946 | 609 | have **: "- k = l * q \<longleftrightarrow> k = - (l * q)" for k l q :: int | 
| 610 | by auto | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 611 | show ?thesis | 
| 69946 | 612 | by (simp add: divmod_integer_def divmod_abs_def) | 
| 613 | (transfer, auto simp add: * ** not_less zdiv_zminus1_eq_if zmod_zminus1_eq_if div_minus_right mod_minus_right) | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 614 | qed | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 615 | |
| 69946 | 616 | lemma divmod_integer_code [code]: \<^marker>\<open>contributor \<open>René Thiemann\<close>\<close> \<^marker>\<open>contributor \<open>Akihisa Yamada\<close>\<close> | 
| 617 | "divmod_integer k l = | |
| 618 | (if k = 0 then (0, 0) | |
| 619 | else if l > 0 then | |
| 620 | (if k > 0 then Code_Numeral.divmod_abs k l | |
| 621 | else case Code_Numeral.divmod_abs k l of (r, s) \<Rightarrow> | |
| 622 | if s = 0 then (- r, 0) else (- r - 1, l - s)) | |
| 623 | else if l = 0 then (0, k) | |
| 624 | else apsnd uminus | |
| 625 | (if k < 0 then Code_Numeral.divmod_abs k l | |
| 626 | else case Code_Numeral.divmod_abs k l of (r, s) \<Rightarrow> | |
| 627 | if s = 0 then (- r, 0) else (- r - 1, - l - s)))" | |
| 628 | by (cases l "0 :: integer" rule: linorder_cases) | |
| 629 | (auto split: prod.splits simp add: divmod_integer_eq_cases) | |
| 630 | ||
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 631 | lemma div_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 632 | "k div l = fst (divmod_integer k l)" | 
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 633 | by simp | 
| 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 634 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 635 | lemma mod_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 636 | "k mod l = snd (divmod_integer k l)" | 
| 25767 | 637 | by simp | 
| 24999 | 638 | |
| 68028 | 639 | definition bit_cut_integer :: "integer \<Rightarrow> integer \<times> bool" | 
| 640 | where "bit_cut_integer k = (k div 2, odd k)" | |
| 641 | ||
| 642 | lemma bit_cut_integer_code [code]: | |
| 643 | "bit_cut_integer k = (if k = 0 then (0, False) | |
| 644 | else let (r, s) = Code_Numeral.divmod_abs k 2 | |
| 645 | in (if k > 0 then r else - r - s, s = 1))" | |
| 646 | proof - | |
| 647 | have "bit_cut_integer k = (let (r, s) = divmod_integer k 2 in (r, s = 1))" | |
| 648 | by (simp add: divmod_integer_def bit_cut_integer_def odd_iff_mod_2_eq_one) | |
| 649 | then show ?thesis | |
| 650 | by (simp add: divmod_integer_code) (auto simp add: split_def) | |
| 651 | qed | |
| 652 | ||
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 653 | lemma equal_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 654 | "HOL.equal 0 (0::integer) \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 655 | "HOL.equal 0 (Pos l) \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 656 | "HOL.equal 0 (Neg l) \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 657 | "HOL.equal (Pos k) 0 \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 658 | "HOL.equal (Pos k) (Pos l) \<longleftrightarrow> HOL.equal k l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 659 | "HOL.equal (Pos k) (Neg l) \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 660 | "HOL.equal (Neg k) 0 \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 661 | "HOL.equal (Neg k) (Pos l) \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 662 | "HOL.equal (Neg k) (Neg l) \<longleftrightarrow> HOL.equal k l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 663 | by (simp_all add: equal) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 664 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 665 | lemma equal_integer_refl [code nbe]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 666 | "HOL.equal (k::integer) k \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 667 | by (fact equal_refl) | 
| 31266 | 668 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 669 | lemma less_eq_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 670 | "0 \<le> (0::integer) \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 671 | "0 \<le> Pos l \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 672 | "0 \<le> Neg l \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 673 | "Pos k \<le> 0 \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 674 | "Pos k \<le> Pos l \<longleftrightarrow> k \<le> l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 675 | "Pos k \<le> Neg l \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 676 | "Neg k \<le> 0 \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 677 | "Neg k \<le> Pos l \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 678 | "Neg k \<le> Neg l \<longleftrightarrow> l \<le> k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 679 | by simp_all | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 680 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 681 | lemma less_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 682 | "0 < (0::integer) \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 683 | "0 < Pos l \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 684 | "0 < Neg l \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 685 | "Pos k < 0 \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 686 | "Pos k < Pos l \<longleftrightarrow> k < l" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 687 | "Pos k < Neg l \<longleftrightarrow> False" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 688 | "Neg k < 0 \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 689 | "Neg k < Pos l \<longleftrightarrow> True" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 690 | "Neg k < Neg l \<longleftrightarrow> l < k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 691 | by simp_all | 
| 26140 | 692 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 693 | lift_definition num_of_integer :: "integer \<Rightarrow> num" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 694 | is "num_of_nat \<circ> nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 695 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 696 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 697 | lemma num_of_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 698 | "num_of_integer k = (if k \<le> 1 then Num.One | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 699 | else let | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 700 | (l, j) = divmod_integer k 2; | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 701 | l' = num_of_integer l; | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 702 | l'' = l' + l' | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 703 | in if j = 0 then l'' else l'' + Num.One)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 704 | proof - | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 705 |   {
 | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 706 | assume "int_of_integer k mod 2 = 1" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 707 | then have "nat (int_of_integer k mod 2) = nat 1" by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 708 | moreover assume *: "1 < int_of_integer k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 709 | ultimately have **: "nat (int_of_integer k) mod 2 = 1" by (simp add: nat_mod_distrib) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 710 | have "num_of_nat (nat (int_of_integer k)) = | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 711 | num_of_nat (2 * (nat (int_of_integer k) div 2) + nat (int_of_integer k) mod 2)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 712 | by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 713 | then have "num_of_nat (nat (int_of_integer k)) = | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 714 | num_of_nat (nat (int_of_integer k) div 2 + nat (int_of_integer k) div 2 + nat (int_of_integer k) mod 2)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 715 | by (simp add: mult_2) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 716 | with ** have "num_of_nat (nat (int_of_integer k)) = | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 717 | num_of_nat (nat (int_of_integer k) div 2 + nat (int_of_integer k) div 2 + 1)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 718 | by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 719 | } | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 720 | note aux = this | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 721 | show ?thesis | 
| 55414 
eab03e9cee8a
renamed '{prod,sum,bool,unit}_case' to 'case_...'
 blanchet parents: 
54489diff
changeset | 722 | by (auto simp add: num_of_integer_def nat_of_integer_def Let_def case_prod_beta | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 723 | not_le integer_eq_iff less_eq_integer_def | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 724 | nat_mult_distrib nat_div_distrib num_of_nat_One num_of_nat_plus_distrib | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 725 | mult_2 [where 'a=nat] aux add_One) | 
| 25918 | 726 | qed | 
| 727 | ||
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 728 | lemma nat_of_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 729 | "nat_of_integer k = (if k \<le> 0 then 0 | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 730 | else let | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 731 | (l, j) = divmod_integer k 2; | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 732 | l' = nat_of_integer l; | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 733 | l'' = l' + l' | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 734 | in if j = 0 then l'' else l'' + 1)" | 
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 735 | proof - | 
| 66886 | 736 | obtain j where k: "k = integer_of_int j" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 737 | proof | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 738 | show "k = integer_of_int (int_of_integer k)" by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 739 | qed | 
| 66886 | 740 | have *: "nat j mod 2 = nat_of_integer (of_int j mod 2)" if "j \<ge> 0" | 
| 741 | using that by transfer (simp add: nat_mod_distrib) | |
| 742 | from k show ?thesis | |
| 743 | by (auto simp add: split_def Let_def nat_of_integer_def nat_div_distrib mult_2 [symmetric] | |
| 744 | minus_mod_eq_mult_div [symmetric] *) | |
| 33340 
a165b97f3658
moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
 haftmann parents: 
33318diff
changeset | 745 | qed | 
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 746 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 747 | lemma int_of_integer_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 748 | "int_of_integer k = (if k < 0 then - (int_of_integer (- k)) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 749 | else if k = 0 then 0 | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 750 | else let | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 751 | (l, j) = divmod_integer k 2; | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 752 | l' = 2 * int_of_integer l | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 753 | in if j = 0 then l' else l' + 1)" | 
| 64246 | 754 | by (auto simp add: split_def Let_def integer_eq_iff minus_mod_eq_mult_div [symmetric]) | 
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 755 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 756 | lemma integer_of_int_code [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 757 | "integer_of_int k = (if k < 0 then - (integer_of_int (- k)) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 758 | else if k = 0 then 0 | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 759 | else let | 
| 60868 
dd18c33c001e
direct bootstrap of integer division from natural division
 haftmann parents: 
60758diff
changeset | 760 | l = 2 * integer_of_int (k div 2); | 
| 
dd18c33c001e
direct bootstrap of integer division from natural division
 haftmann parents: 
60758diff
changeset | 761 | j = k mod 2 | 
| 
dd18c33c001e
direct bootstrap of integer division from natural division
 haftmann parents: 
60758diff
changeset | 762 | in if j = 0 then l else l + 1)" | 
| 64246 | 763 | by (auto simp add: split_def Let_def integer_eq_iff minus_mod_eq_mult_div [symmetric]) | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 764 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 765 | hide_const (open) Pos Neg sub dup divmod_abs | 
| 46547 
d1dcb91a512e
use qualified constant names instead of suffixes (from Florian Haftmann)
 huffman parents: 
46028diff
changeset | 766 | |
| 28708 
a1a436f09ec6
explicit check for pattern discipline before code translation
 haftmann parents: 
28562diff
changeset | 767 | |
| 60758 | 768 | subsection \<open>Serializer setup for target language integers\<close> | 
| 24999 | 769 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 770 | code_reserved Eval int Integer abs | 
| 25767 | 771 | |
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 772 | code_printing | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 773 | type_constructor integer \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 774 | (SML) "IntInf.int" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 775 | and (OCaml) "Z.t" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 776 | and (Haskell) "Integer" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 777 | and (Scala) "BigInt" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 778 | and (Eval) "int" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 779 | | class_instance integer :: equal \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 780 | (Haskell) - | 
| 24999 | 781 | |
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 782 | code_printing | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 783 | constant "0::integer" \<rightharpoonup> | 
| 58400 
d0d3c30806b4
always annotate potentially polymorphic Haskell numerals
 haftmann parents: 
58399diff
changeset | 784 | (SML) "!(0/ :/ IntInf.int)" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 785 | and (OCaml) "Z.zero" | 
| 58400 
d0d3c30806b4
always annotate potentially polymorphic Haskell numerals
 haftmann parents: 
58399diff
changeset | 786 | and (Haskell) "!(0/ ::/ Integer)" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 787 | and (Scala) "BigInt(0)" | 
| 47108 
2a1953f0d20d
merged fork with new numeral representation (see NEWS)
 huffman parents: 
46664diff
changeset | 788 | |
| 60758 | 789 | setup \<open> | 
| 58399 | 790 | fold (fn target => | 
| 69593 | 791 | Numeral.add_code \<^const_name>\<open>Code_Numeral.Pos\<close> I Code_Printer.literal_numeral target | 
| 792 | #> Numeral.add_code \<^const_name>\<open>Code_Numeral.Neg\<close> (~) Code_Printer.literal_numeral target) | |
| 58399 | 793 | ["SML", "OCaml", "Haskell", "Scala"] | 
| 60758 | 794 | \<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 795 | |
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 796 | code_printing | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 797 | constant "plus :: integer \<Rightarrow> _ \<Rightarrow> _" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 798 | (SML) "IntInf.+ ((_), (_))" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 799 | and (OCaml) "Z.add" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 800 | and (Haskell) infixl 6 "+" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 801 | and (Scala) infixl 7 "+" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 802 | and (Eval) infixl 8 "+" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 803 | | constant "uminus :: integer \<Rightarrow> _" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 804 | (SML) "IntInf.~" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 805 | and (OCaml) "Z.neg" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 806 | and (Haskell) "negate" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 807 | and (Scala) "!(- _)" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 808 | and (Eval) "~/ _" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 809 | | constant "minus :: integer \<Rightarrow> _" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 810 | (SML) "IntInf.- ((_), (_))" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 811 | and (OCaml) "Z.sub" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 812 | and (Haskell) infixl 6 "-" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 813 | and (Scala) infixl 7 "-" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 814 | and (Eval) infixl 8 "-" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 815 | | constant Code_Numeral.dup \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 816 | (SML) "IntInf.*/ (2,/ (_))" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 817 | and (OCaml) "Z.shift'_left/ _/ 1" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 818 | and (Haskell) "!(2 * _)" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 819 | and (Scala) "!(2 * _)" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 820 | and (Eval) "!(2 * _)" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 821 | | constant Code_Numeral.sub \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 822 | (SML) "!(raise/ Fail/ \"sub\")" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 823 | and (OCaml) "failwith/ \"sub\"" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 824 | and (Haskell) "error/ \"sub\"" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 825 | and (Scala) "!sys.error(\"sub\")" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 826 | | constant "times :: integer \<Rightarrow> _ \<Rightarrow> _" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 827 | (SML) "IntInf.* ((_), (_))" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 828 | and (OCaml) "Z.mul" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 829 | and (Haskell) infixl 7 "*" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 830 | and (Scala) infixl 8 "*" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 831 | and (Eval) infixl 9 "*" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 832 | | constant Code_Numeral.divmod_abs \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 833 | (SML) "IntInf.divMod/ (IntInf.abs _,/ IntInf.abs _)" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 834 | and (OCaml) "!(fun k l ->/ if Z.equal Z.zero l then/ (Z.zero, l) else/ Z.div'_rem/ (Z.abs k)/ (Z.abs l))" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 835 | and (Haskell) "divMod/ (abs _)/ (abs _)" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 836 | and (Scala) "!((k: BigInt) => (l: BigInt) =>/ if (l == 0)/ (BigInt(0), k) else/ (k.abs '/% l.abs))" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 837 | and (Eval) "Integer.div'_mod/ (abs _)/ (abs _)" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 838 | | constant "HOL.equal :: integer \<Rightarrow> _ \<Rightarrow> bool" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 839 | (SML) "!((_ : IntInf.int) = _)" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 840 | and (OCaml) "Z.equal" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 841 | and (Haskell) infix 4 "==" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 842 | and (Scala) infixl 5 "==" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 843 | and (Eval) infixl 6 "=" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 844 | | constant "less_eq :: integer \<Rightarrow> _ \<Rightarrow> bool" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 845 | (SML) "IntInf.<= ((_), (_))" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 846 | and (OCaml) "Z.leq" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 847 | and (Haskell) infix 4 "<=" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 848 | and (Scala) infixl 4 "<=" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 849 | and (Eval) infixl 6 "<=" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 850 | | constant "less :: integer \<Rightarrow> _ \<Rightarrow> bool" \<rightharpoonup> | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 851 | (SML) "IntInf.< ((_), (_))" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 852 | and (OCaml) "Z.lt" | 
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 853 | and (Haskell) infix 4 "<" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 854 | and (Scala) infixl 4 "<" | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 855 | and (Eval) infixl 6 "<" | 
| 61857 
542f2c6da692
add serialisation for abs on integer to target language operation
 Andreas Lochbihler parents: 
61275diff
changeset | 856 | | constant "abs :: integer \<Rightarrow> _" \<rightharpoonup> | 
| 
542f2c6da692
add serialisation for abs on integer to target language operation
 Andreas Lochbihler parents: 
61275diff
changeset | 857 | (SML) "IntInf.abs" | 
| 69906 
55534affe445
migrated from Nums to Zarith as library for OCaml integer arithmetic
 haftmann parents: 
69593diff
changeset | 858 | and (OCaml) "Z.abs" | 
| 61857 
542f2c6da692
add serialisation for abs on integer to target language operation
 Andreas Lochbihler parents: 
61275diff
changeset | 859 | and (Haskell) "Prelude.abs" | 
| 
542f2c6da692
add serialisation for abs on integer to target language operation
 Andreas Lochbihler parents: 
61275diff
changeset | 860 | and (Scala) "_.abs" | 
| 
542f2c6da692
add serialisation for abs on integer to target language operation
 Andreas Lochbihler parents: 
61275diff
changeset | 861 | and (Eval) "abs" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 862 | |
| 52435 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 863 | code_identifier | 
| 
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
 haftmann parents: 
51375diff
changeset | 864 | code_module Code_Numeral \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith | 
| 46547 
d1dcb91a512e
use qualified constant names instead of suffixes (from Florian Haftmann)
 huffman parents: 
46028diff
changeset | 865 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 866 | |
| 60758 | 867 | subsection \<open>Type of target language naturals\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 868 | |
| 61076 | 869 | typedef natural = "UNIV :: nat set" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 870 | morphisms nat_of_natural natural_of_nat .. | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 871 | |
| 59487 
adaa430fc0f7
default abstypes and default abstract equations make technical (no_code) annotation superfluous
 haftmann parents: 
58889diff
changeset | 872 | setup_lifting type_definition_natural | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 873 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 874 | lemma natural_eq_iff [termination_simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 875 | "m = n \<longleftrightarrow> nat_of_natural m = nat_of_natural n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 876 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 877 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 878 | lemma natural_eqI: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 879 | "nat_of_natural m = nat_of_natural n \<Longrightarrow> m = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 880 | using natural_eq_iff [of m n] by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 881 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 882 | lemma nat_of_natural_of_nat_inverse [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 883 | "nat_of_natural (natural_of_nat n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 884 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 885 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 886 | lemma natural_of_nat_of_natural_inverse [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 887 | "natural_of_nat (nat_of_natural n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 888 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 889 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 890 | instantiation natural :: "{comm_monoid_diff, semiring_1}"
 | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 891 | begin | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 892 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 893 | lift_definition zero_natural :: natural | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 894 | is "0 :: nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 895 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 896 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 897 | declare zero_natural.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 898 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 899 | lift_definition one_natural :: natural | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 900 | is "1 :: nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 901 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 902 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 903 | declare one_natural.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 904 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 905 | lift_definition plus_natural :: "natural \<Rightarrow> natural \<Rightarrow> natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 906 | is "plus :: nat \<Rightarrow> nat \<Rightarrow> nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 907 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 908 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 909 | declare plus_natural.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 910 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 911 | lift_definition minus_natural :: "natural \<Rightarrow> natural \<Rightarrow> natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 912 | is "minus :: nat \<Rightarrow> nat \<Rightarrow> nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 913 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 914 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 915 | declare minus_natural.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 916 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 917 | lift_definition times_natural :: "natural \<Rightarrow> natural \<Rightarrow> natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 918 | is "times :: nat \<Rightarrow> nat \<Rightarrow> nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 919 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 920 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 921 | declare times_natural.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 922 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 923 | instance proof | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 924 | qed (transfer, simp add: algebra_simps)+ | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 925 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 926 | end | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 927 | |
| 64241 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 928 | instance natural :: Rings.dvd .. | 
| 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 929 | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 930 | context | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 931 | includes lifting_syntax | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 932 | begin | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 933 | |
| 64241 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 934 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 935 | \<open>(pcr_natural ===> pcr_natural ===> (\<longleftrightarrow>)) (dvd) (dvd)\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 936 | by (unfold dvd_def) transfer_prover | 
| 64241 
430d74089d4d
transfer rules for divides relation on integer and natural
 haftmann parents: 
64178diff
changeset | 937 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 938 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 939 | \<open>((\<longleftrightarrow>) ===> pcr_natural) of_bool of_bool\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 940 | by (unfold of_bool_def) transfer_prover | 
| 68010 | 941 | |
| 942 | lemma [transfer_rule]: | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 943 | \<open>((=) ===> pcr_natural) (\<lambda>n. n) of_nat\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 944 | proof - | 
| 55945 | 945 | have "rel_fun HOL.eq pcr_natural (of_nat :: nat \<Rightarrow> nat) (of_nat :: nat \<Rightarrow> natural)" | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 946 | by (unfold of_nat_def) transfer_prover | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 947 | then show ?thesis by (simp add: id_def) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 948 | qed | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 949 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 950 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 951 | \<open>((=) ===> pcr_natural) numeral numeral\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 952 | proof - | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 953 | have \<open>((=) ===> pcr_natural) numeral (\<lambda>n. of_nat (numeral n))\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 954 | by transfer_prover | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 955 | then show ?thesis by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 956 | qed | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 957 | |
| 68010 | 958 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 959 | \<open>(pcr_natural ===> (=) ===> pcr_natural) (^) (^)\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 960 | by (unfold power_def) transfer_prover | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 961 | |
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 962 | end | 
| 68010 | 963 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 964 | lemma nat_of_natural_of_nat [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 965 | "nat_of_natural (of_nat n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 966 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 967 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 968 | lemma natural_of_nat_of_nat [simp, code_abbrev]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 969 | "natural_of_nat = of_nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 970 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 971 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 972 | lemma of_nat_of_natural [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 973 | "of_nat (nat_of_natural n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 974 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 975 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 976 | lemma nat_of_natural_numeral [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 977 | "nat_of_natural (numeral k) = numeral k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 978 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 979 | |
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 980 | instantiation natural :: "{linordered_semiring, equal}"
 | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 981 | begin | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 982 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 983 | lift_definition less_eq_natural :: "natural \<Rightarrow> natural \<Rightarrow> bool" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 984 | is "less_eq :: nat \<Rightarrow> nat \<Rightarrow> bool" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 985 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 986 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 987 | declare less_eq_natural.rep_eq [termination_simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 988 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 989 | lift_definition less_natural :: "natural \<Rightarrow> natural \<Rightarrow> bool" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 990 | is "less :: nat \<Rightarrow> nat \<Rightarrow> bool" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 991 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 992 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 993 | declare less_natural.rep_eq [termination_simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 994 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 995 | lift_definition equal_natural :: "natural \<Rightarrow> natural \<Rightarrow> bool" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 996 | is "HOL.equal :: nat \<Rightarrow> nat \<Rightarrow> bool" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 997 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 998 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 999 | instance proof | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1000 | qed (transfer, simp add: algebra_simps equal less_le_not_le [symmetric] linear)+ | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1001 | |
| 24999 | 1002 | end | 
| 46664 
1f6c140f9c72
moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
 haftmann parents: 
46638diff
changeset | 1003 | |
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1004 | context | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1005 | includes lifting_syntax | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1006 | begin | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1007 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1008 | lemma [transfer_rule]: | 
| 71535 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1009 | \<open>(pcr_natural ===> pcr_natural ===> pcr_natural) min min\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1010 | by (unfold min_def) transfer_prover | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1011 | |
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1012 | lemma [transfer_rule]: | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1013 | \<open>(pcr_natural ===> pcr_natural ===> pcr_natural) max max\<close> | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1014 | by (unfold max_def) transfer_prover | 
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1015 | |
| 
b612edee9b0c
more frugal simp rules for bit operations; more pervasive use of bit selector
 haftmann parents: 
71424diff
changeset | 1016 | end | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1017 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1018 | lemma nat_of_natural_min [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1019 | "nat_of_natural (min k l) = min (nat_of_natural k) (nat_of_natural l)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1020 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1021 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1022 | lemma nat_of_natural_max [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1023 | "nat_of_natural (max k l) = max (nat_of_natural k) (nat_of_natural l)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1024 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1025 | |
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1026 | instantiation natural :: unique_euclidean_semiring | 
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1027 | begin | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1028 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1029 | lift_definition divide_natural :: "natural \<Rightarrow> natural \<Rightarrow> natural" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1030 | is "divide :: nat \<Rightarrow> nat \<Rightarrow> nat" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1031 | . | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1032 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1033 | declare divide_natural.rep_eq [simp] | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1034 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1035 | lift_definition modulo_natural :: "natural \<Rightarrow> natural \<Rightarrow> natural" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1036 | is "modulo :: nat \<Rightarrow> nat \<Rightarrow> nat" | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1037 | . | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1038 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1039 | declare modulo_natural.rep_eq [simp] | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1040 | |
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1041 | lift_definition euclidean_size_natural :: "natural \<Rightarrow> nat" | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1042 | is "euclidean_size :: nat \<Rightarrow> nat" | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1043 | . | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1044 | |
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1045 | declare euclidean_size_natural.rep_eq [simp] | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1046 | |
| 66838 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 1047 | lift_definition division_segment_natural :: "natural \<Rightarrow> natural" | 
| 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 1048 | is "division_segment :: nat \<Rightarrow> nat" | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1049 | . | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1050 | |
| 66838 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 1051 | declare division_segment_natural.rep_eq [simp] | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1052 | |
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1053 | instance | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1054 | by (standard; transfer) | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1055 | (auto simp add: algebra_simps unit_factor_nat_def gr0_conv_Suc) | 
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1056 | |
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1057 | end | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1058 | |
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1059 | lemma [code]: | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1060 | "euclidean_size = nat_of_natural" | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1061 | by (simp add: fun_eq_iff) | 
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1062 | |
| 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1063 | lemma [code]: | 
| 66838 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 1064 | "division_segment (n::natural) = 1" | 
| 
17989f6bc7b2
clarified uniqueness criterion for euclidean rings
 haftmann parents: 
66836diff
changeset | 1065 | by (simp add: natural_eq_iff) | 
| 66806 
a4e82b58d833
abolished (semi)ring_div in favour of euclidean_(semi)ring_cancel
 haftmann parents: 
66801diff
changeset | 1066 | |
| 78935 
5e788ff7a489
explicit type class for discrete linordered semidoms
 haftmann parents: 
78669diff
changeset | 1067 | instance natural :: discrete_linordered_semidom | 
| 78937 
5e6b195eee83
slightly less technical formulation of very specific type class
 haftmann parents: 
78935diff
changeset | 1068 | by (standard; transfer) (simp_all add: Suc_le_eq) | 
| 67905 | 1069 | |
| 78937 
5e6b195eee83
slightly less technical formulation of very specific type class
 haftmann parents: 
78935diff
changeset | 1070 | instance natural :: linordered_euclidean_semiring | 
| 66839 | 1071 | by (standard; transfer) simp_all | 
| 66815 | 1072 | |
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1073 | instantiation natural :: semiring_bit_operations | 
| 71094 | 1074 | begin | 
| 1075 | ||
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1076 | lift_definition bit_natural :: \<open>natural \<Rightarrow> nat \<Rightarrow> bool\<close> | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1077 | is bit . | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1078 | |
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1079 | lift_definition and_natural :: \<open>natural \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1080 | is \<open>and\<close> . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1081 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1082 | lift_definition or_natural :: \<open>natural \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1083 | is or . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1084 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1085 | lift_definition xor_natural :: \<open>natural \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1086 | is xor . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1087 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1088 | lift_definition mask_natural :: \<open>nat \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1089 | is mask . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1090 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1091 | lift_definition set_bit_natural :: \<open>nat \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1092 | is set_bit . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1093 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1094 | lift_definition unset_bit_natural :: \<open>nat \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1095 | is unset_bit . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1096 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1097 | lift_definition flip_bit_natural :: \<open>nat \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1098 | is flip_bit . | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1099 | |
| 71094 | 1100 | lift_definition push_bit_natural :: \<open>nat \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1101 | is push_bit . | 
| 71094 | 1102 | |
| 1103 | lift_definition drop_bit_natural :: \<open>nat \<Rightarrow> natural \<Rightarrow> natural\<close> | |
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1104 | is drop_bit . | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1105 | |
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1106 | lift_definition take_bit_natural :: \<open>nat \<Rightarrow> natural \<Rightarrow> natural\<close> | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1107 | is take_bit . | 
| 71094 | 1108 | |
| 1109 | instance by (standard; transfer) | |
| 79480 
c7cb1bf6efa0
consolidated name of lemma analogously to nat/int/word_bit_induct
 haftmann parents: 
79072diff
changeset | 1110 | (fact bit_eq_rec bit_induct bit_iff_odd push_bit_eq_mult drop_bit_eq_div take_bit_eq_mod | 
| 79488 | 1111 | bits_div_0 bits_div_by_0 bits_div_by_1 even_half_succ_eq | 
| 71413 | 1112 | exp_div_exp_eq div_exp_eq mod_exp_eq mult_exp_mod_exp_eq div_exp_mod_exp_eq | 
| 79008 
74a4776f7a22
operations AND, OR, XOR are specified by characteristic recursive equation
 haftmann parents: 
78955diff
changeset | 1113 | even_mask_div_iff even_mult_exp_div_exp_iff and_rec or_rec xor_rec | 
| 79489 | 1114 | mask_eq_exp_minus_1 set_bit_eq_or unset_bit_eq_or_xor flip_bit_eq_xor)+ | 
| 71094 | 1115 | |
| 1116 | end | |
| 68010 | 1117 | |
| 78955 | 1118 | instance natural :: linordered_euclidean_semiring_bit_operations .. | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1119 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1120 | context | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1121 | includes bit_operations_syntax | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1122 | begin | 
| 71094 | 1123 | |
| 1124 | lemma [code]: | |
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1125 | \<open>bit m n \<longleftrightarrow> odd (drop_bit n m)\<close> | 
| 79016 | 1126 | \<open>mask n = 2 ^ n - (1 :: natural)\<close> | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1127 | \<open>set_bit n m = m OR push_bit n 1\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1128 | \<open>flip_bit n m = m XOR push_bit n 1\<close> | 
| 71094 | 1129 | \<open>push_bit n m = m * 2 ^ n\<close> | 
| 71965 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1130 | \<open>drop_bit n m = m div 2 ^ n\<close> | 
| 
d45f5d4c41bd
more class operations for the sake of efficient generated code
 haftmann parents: 
71535diff
changeset | 1131 | \<open>take_bit n m = m mod 2 ^ n\<close> for m :: natural | 
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1132 | by (fact bit_iff_odd_drop_bit mask_eq_exp_minus_1 | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1133 | set_bit_eq_or flip_bit_eq_xor push_bit_eq_mult drop_bit_eq_div take_bit_eq_mod)+ | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1134 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1135 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1136 | \<open>m AND n = (if m = 0 \<or> n = 0 then 0 | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1137 | else (m mod 2) * (n mod 2) + 2 * ((m div 2) AND (n div 2)))\<close> for m n :: natural | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1138 | by transfer (fact and_nat_unfold) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1139 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1140 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1141 | \<open>m OR n = (if m = 0 then n else if n = 0 then m | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1142 | else max (m mod 2) (n mod 2) + 2 * ((m div 2) OR (n div 2)))\<close> for m n :: natural | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1143 | by transfer (fact or_nat_unfold) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1144 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1145 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1146 | \<open>m XOR n = (if m = 0 then n else if n = 0 then m | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1147 | else (m mod 2 + n mod 2) mod 2 + 2 * ((m div 2) XOR (n div 2)))\<close> for m n :: natural | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1148 | by transfer (fact xor_nat_unfold) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1149 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1150 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1151 | \<open>unset_bit 0 m = 2 * (m div 2)\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1152 | \<open>unset_bit (Suc n) m = m mod 2 + 2 * unset_bit n (m div 2)\<close> for m :: natural | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1153 | by (transfer; simp add: unset_bit_Suc)+ | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1154 | |
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1155 | end | 
| 68010 | 1156 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1157 | lift_definition natural_of_integer :: "integer \<Rightarrow> natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1158 | is "nat :: int \<Rightarrow> nat" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1159 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1160 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1161 | lift_definition integer_of_natural :: "natural \<Rightarrow> integer" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1162 | is "of_nat :: nat \<Rightarrow> int" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1163 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1164 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1165 | lemma natural_of_integer_of_natural [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1166 | "natural_of_integer (integer_of_natural n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1167 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1168 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1169 | lemma integer_of_natural_of_integer [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1170 | "integer_of_natural (natural_of_integer k) = max 0 k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1171 | by transfer auto | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1172 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1173 | lemma int_of_integer_of_natural [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1174 | "int_of_integer (integer_of_natural n) = of_nat (nat_of_natural n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1175 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1176 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1177 | lemma integer_of_natural_of_nat [simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1178 | "integer_of_natural (of_nat n) = of_nat n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1179 | by transfer rule | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1180 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1181 | lemma [measure_function]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1182 | "is_measure nat_of_natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1183 | by (rule is_measure_trivial) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1184 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1185 | |
| 60758 | 1186 | subsection \<open>Inductive representation of target language naturals\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1187 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1188 | lift_definition Suc :: "natural \<Rightarrow> natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1189 | is Nat.Suc | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1190 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1191 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1192 | declare Suc.rep_eq [simp] | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1193 | |
| 58306 
117ba6cbe414
renamed 'rep_datatype' to 'old_rep_datatype' (HOL)
 blanchet parents: 
57512diff
changeset | 1194 | old_rep_datatype "0::natural" Suc | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1195 | by (transfer, fact nat.induct nat.inject nat.distinct)+ | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1196 | |
| 55416 | 1197 | lemma natural_cases [case_names nat, cases type: natural]: | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1198 | fixes m :: natural | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1199 | assumes "\<And>n. m = of_nat n \<Longrightarrow> P" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1200 | shows P | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1201 | using assms by transfer blast | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1202 | |
| 67332 | 1203 | instantiation natural :: size | 
| 1204 | begin | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1205 | |
| 67332 | 1206 | definition size_nat where [simp, code]: "size_nat = nat_of_natural" | 
| 1207 | ||
| 1208 | instance .. | |
| 1209 | ||
| 1210 | end | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1211 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1212 | lemma natural_decr [termination_simp]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1213 | "n \<noteq> 0 \<Longrightarrow> nat_of_natural n - Nat.Suc 0 < nat_of_natural n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1214 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1215 | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1216 | lemma natural_zero_minus_one: "(0::natural) - 1 = 0" | 
| 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1217 | by (rule zero_diff) | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1218 | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1219 | lemma Suc_natural_minus_one: "Suc n - 1 = n" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1220 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1221 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1222 | hide_const (open) Suc | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1223 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1224 | |
| 60758 | 1225 | subsection \<open>Code refinement for target language naturals\<close> | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1226 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1227 | lift_definition Nat :: "integer \<Rightarrow> natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1228 | is nat | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1229 | . | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1230 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1231 | lemma [code_post]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1232 | "Nat 0 = 0" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1233 | "Nat 1 = 1" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1234 | "Nat (numeral k) = numeral k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1235 | by (transfer, simp)+ | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1236 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1237 | lemma [code abstype]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1238 | "Nat (integer_of_natural n) = n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1239 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1240 | |
| 63174 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1241 | lemma [code]: | 
| 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1242 | "natural_of_nat n = natural_of_integer (integer_of_nat n)" | 
| 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1243 | by transfer simp | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1244 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1245 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1246 | "integer_of_natural (natural_of_integer k) = max 0 k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1247 | by simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1248 | |
| 74108 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1249 | lemma [code]: | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1250 | \<open>integer_of_natural (mask n) = mask n\<close> | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1251 | by transfer (simp add: mask_eq_exp_minus_1 of_nat_diff) | 
| 
3146646a43a7
simplified hierarchy of type classes for bit operations
 haftmann parents: 
74101diff
changeset | 1252 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1253 | lemma [code_abbrev]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1254 | "natural_of_integer (Code_Numeral.Pos k) = numeral k" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1255 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1256 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1257 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1258 | "integer_of_natural 0 = 0" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1259 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1260 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1261 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1262 | "integer_of_natural 1 = 1" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1263 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1264 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1265 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1266 | "integer_of_natural (Code_Numeral.Suc n) = integer_of_natural n + 1" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1267 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1268 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1269 | lemma [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1270 | "nat_of_natural = nat_of_integer \<circ> integer_of_natural" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1271 | by transfer (simp add: fun_eq_iff) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1272 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1273 | lemma [code, code_unfold]: | 
| 55416 | 1274 | "case_natural f g n = (if n = 0 then f else g (n - 1))" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1275 | by (cases n rule: natural.exhaust) (simp_all, simp add: Suc_def) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1276 | |
| 55642 
63beb38e9258
adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'
 blanchet parents: 
55428diff
changeset | 1277 | declare natural.rec [code del] | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1278 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1279 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1280 | "integer_of_natural (m + n) = integer_of_natural m + integer_of_natural n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1281 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1282 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1283 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1284 | "integer_of_natural (m - n) = max 0 (integer_of_natural m - integer_of_natural n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1285 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1286 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1287 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1288 | "integer_of_natural (m * n) = integer_of_natural m * integer_of_natural n" | 
| 64592 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1289 | by transfer simp | 
| 
7759f1766189
more fine-grained type class hierarchy for div and mod
 haftmann parents: 
64246diff
changeset | 1290 | |
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1291 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1292 | "integer_of_natural (m div n) = integer_of_natural m div integer_of_natural n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1293 | by transfer (simp add: zdiv_int) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1294 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1295 | lemma [code abstract]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1296 | "integer_of_natural (m mod n) = integer_of_natural m mod integer_of_natural n" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1297 | by transfer (simp add: zmod_int) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1298 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1299 | lemma [code]: | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1300 | "HOL.equal m n \<longleftrightarrow> HOL.equal (integer_of_natural m) (integer_of_natural n)" | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1301 | by transfer (simp add: equal) | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1302 | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1303 | lemma [code nbe]: "HOL.equal n (n::natural) \<longleftrightarrow> True" | 
| 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1304 | by (rule equal_class.equal_refl) | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1305 | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1306 | lemma [code]: "m \<le> n \<longleftrightarrow> integer_of_natural m \<le> integer_of_natural n" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1307 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1308 | |
| 58379 
c044539a2bda
reintroduced an instantiation of 'size' for 'numerals'
 blanchet parents: 
58377diff
changeset | 1309 | lemma [code]: "m < n \<longleftrightarrow> integer_of_natural m < integer_of_natural n" | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1310 | by transfer simp | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1311 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1312 | hide_const (open) Nat | 
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1313 | |
| 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1314 | code_reflect Code_Numeral | 
| 63174 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1315 | datatypes natural | 
| 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1316 | functions "Code_Numeral.Suc" "0 :: natural" "1 :: natural" | 
| 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1317 | "plus :: natural \<Rightarrow> _" "minus :: natural \<Rightarrow> _" | 
| 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1318 | "times :: natural \<Rightarrow> _" "divide :: natural \<Rightarrow> _" | 
| 63950 
cdc1e59aa513
syntactic type class for operation mod named after mod;
 haftmann parents: 
63174diff
changeset | 1319 | "modulo :: natural \<Rightarrow> _" | 
| 63174 
57c0d60e491c
do not export abstract constructors in code_reflect
 haftmann parents: 
61857diff
changeset | 1320 | integer_of_natural natural_of_integer | 
| 51143 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 haftmann parents: 
49962diff
changeset | 1321 | |
| 74101 | 1322 | lifting_update integer.lifting | 
| 1323 | lifting_forget integer.lifting | |
| 1324 | ||
| 1325 | lifting_update natural.lifting | |
| 1326 | lifting_forget natural.lifting | |
| 1327 | ||
| 1328 | end |