doc-src/ZF/ZF_examples.thy
changeset 35416 d8d7d1b785af
parent 16417 9bc16273c2d4
child 46471 2289a3869c88
equal deleted inserted replaced
35342:4dc65845eab3 35416:d8d7d1b785af
    62 
    62 
    63 lemma n_nodes_aux_eq [rule_format]:
    63 lemma n_nodes_aux_eq [rule_format]:
    64      "t \<in> bt(A) ==> \<forall>k \<in> nat. n_nodes_aux(t)`k = n_nodes(t) #+ k"
    64      "t \<in> bt(A) ==> \<forall>k \<in> nat. n_nodes_aux(t)`k = n_nodes(t) #+ k"
    65   by (induct_tac t, simp_all) 
    65   by (induct_tac t, simp_all) 
    66 
    66 
    67 constdefs  n_nodes_tail :: "i => i"
    67 definition n_nodes_tail :: "i => i" where
    68    "n_nodes_tail(t) == n_nodes_aux(t) ` 0"
    68    "n_nodes_tail(t) == n_nodes_aux(t) ` 0"
    69 
    69 
    70 lemma "t \<in> bt(A) ==> n_nodes_tail(t) = n_nodes(t)"
    70 lemma "t \<in> bt(A) ==> n_nodes_tail(t) = n_nodes(t)"
    71  by (simp add: n_nodes_tail_def n_nodes_aux_eq) 
    71  by (simp add: n_nodes_tail_def n_nodes_aux_eq) 
    72 
    72