src/HOL/Nat.thy
changeset 20640 05e6042394b9
parent 20588 c847c56edf0c
child 20699 0cc77abb185a
equal deleted inserted replaced
20639:3aa960295c54 20640:05e6042394b9
  1060   "OperationalEquality.eq (Suc n) 0 = False" unfolding eq_def by auto
  1060   "OperationalEquality.eq (Suc n) 0 = False" unfolding eq_def by auto
  1061 
  1061 
  1062 lemma [code func]:
  1062 lemma [code func]:
  1063   "OperationalEquality.eq 0 (Suc m) = False" unfolding eq_def by auto
  1063   "OperationalEquality.eq 0 (Suc m) = False" unfolding eq_def by auto
  1064 
  1064 
       
  1065 code_typename
       
  1066   "nat" "IntDef.nat"
       
  1067 
       
  1068 code_constname
       
  1069   "0 \<Colon> nat" "IntDef.zero_nat"
       
  1070   "1 \<Colon> nat" "IntDef.one_nat"
       
  1071   Suc "IntDef.succ_nat"
       
  1072   "op + \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.plus_nat"
       
  1073   "op - \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.minus_nat"
       
  1074   "op * \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat" "IntDef.times_nat"
       
  1075   "op < \<Colon> nat \<Rightarrow> nat \<Rightarrow> bool" "IntDef.less_nat"
       
  1076   "op \<le> \<Colon> nat \<Rightarrow> nat \<Rightarrow> bool" "IntDef.less_eq_nat"
       
  1077   "OperationalEquality.eq \<Colon> nat \<Rightarrow> nat \<Rightarrow> bool" "IntDef.eq_nat"
       
  1078 
  1065 end
  1079 end