src/HOL/Import/HOL/HOL4Base.thy
changeset 30971 7fbebf75b3ef
parent 30952 7ab2716dd93b
child 35416 d8d7d1b785af
equal deleted inserted replaced
30970:3fe2e418a071 30971:7fbebf75b3ef
  2792 
  2792 
  2793 lemma numeral_fact: "ALL n::nat. FACT n = (if n = 0 then 1 else n * FACT (PRE n))"
  2793 lemma numeral_fact: "ALL n::nat. FACT n = (if n = 0 then 1 else n * FACT (PRE n))"
  2794   by (import numeral numeral_fact)
  2794   by (import numeral numeral_fact)
  2795 
  2795 
  2796 lemma numeral_funpow: "ALL n::nat.
  2796 lemma numeral_funpow: "ALL n::nat.
  2797    ((f::'a::type => 'a::type) o^ n) (x::'a::type) =
  2797    ((f::'a::type => 'a::type) ^^ n) (x::'a::type) =
  2798    (if n = 0 then x else (f o^ (n - 1)) (f x))"
  2798    (if n = 0 then x else (f ^^ (n - 1)) (f x))"
  2799   by (import numeral numeral_funpow)
  2799   by (import numeral numeral_funpow)
  2800 
  2800 
  2801 ;end_setup
  2801 ;end_setup
  2802 
  2802 
  2803 ;setup_theory ind_type
  2803 ;setup_theory ind_type